2013-09-02 12:29:21 -07:00
|
|
|
Set: pp::colors
|
2013-09-03 10:44:51 -07:00
|
|
|
Set: pp::unicode
|
2013-08-31 19:15:48 -07:00
|
|
|
Assumed: f
|
2013-09-01 10:34:57 -07:00
|
|
|
λ (A B : Type) (a : B), f B a
|
2013-09-04 13:21:57 -07:00
|
|
|
Error (line: 4, pos: 40) application type mismatch during term elaboration
|
2013-08-31 19:15:48 -07:00
|
|
|
f B a
|
2013-09-04 13:21:57 -07:00
|
|
|
Function type:
|
2013-09-08 11:04:07 -07:00
|
|
|
Π (A : Type), A → Bool
|
2013-09-04 13:21:57 -07:00
|
|
|
Arguments types:
|
|
|
|
B : Type
|
|
|
|
a : lift:0:2 ?M0
|
2013-08-31 19:15:48 -07:00
|
|
|
Elaborator state
|
2013-09-01 10:34:57 -07:00
|
|
|
#0 ≈ lift:0:2 ?M0
|
2013-08-31 19:15:48 -07:00
|
|
|
Assumed: myeq
|
2013-09-08 11:04:07 -07:00
|
|
|
myeq (Π (A : Type), A → A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b)
|
2013-09-08 22:54:22 -07:00
|
|
|
myeq (Π (A : Type), A → A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b) : Bool
|
2013-08-31 19:15:48 -07:00
|
|
|
Assumed: R
|
|
|
|
Assumed: h
|
2013-09-08 22:54:22 -07:00
|
|
|
λ (H : Bool) (f1 g1 : Π A : Type, R A) (G : Π A : Type, myeq (R A) (f1 A) (g1 A)), h f1 :
|
|
|
|
Bool → (Π (f1 g1 : Π A : Type, R A), (Π A : Type, myeq (R A) (f1 A) (g1 A)) → Bool)
|