2013-09-02 19:29:21 +00:00
|
|
|
Set: pp::colors
|
2013-09-03 17:44:51 +00:00
|
|
|
Set: pp::unicode
|
2013-09-01 02:15:48 +00:00
|
|
|
Assumed: f
|
2013-09-01 17:34:57 +00:00
|
|
|
λ (A B : Type) (a : B), f B a
|
2013-10-25 02:08:35 +00:00
|
|
|
Failed to solve
|
2014-02-07 01:25:33 +00:00
|
|
|
A : Type, a : ?M::0, B : Type ⊢ ?M::0[lift:0 2] ≺ B
|
2014-01-09 20:15:12 +00:00
|
|
|
tst7.lean:4:42: Type of argument 2 must be convertible to the expected type in the application of
|
2013-10-25 02:08:35 +00:00
|
|
|
f
|
|
|
|
with arguments:
|
|
|
|
B
|
|
|
|
a
|
2013-09-01 02:15:48 +00:00
|
|
|
Assumed: myeq
|
2014-01-08 08:38:39 +00:00
|
|
|
myeq (∀ (A : Type), A → A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b)
|
|
|
|
myeq (∀ (A : Type), A → A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b) : Bool
|
2013-09-01 02:15:48 +00:00
|
|
|
Assumed: R
|
|
|
|
Assumed: h
|
2014-01-08 08:38:39 +00: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)
|