lean2/tests/lean/tst7.lean.expected.out
Leonardo de Moura fdeb457a81 feat(kernel/pos_info_provider): add support for file names in pos_info_provider
The idea is to include the file name when displaying justification objects.

Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-09 12:19:30 -08:00

18 lines
717 B
Text

Set: pp::colors
Set: pp::unicode
Assumed: f
λ (A B : Type) (a : B), f B a
Failed to solve
A : Type, a : ?M::0, B : Type ⊢ ?M::0[lift:0:2] ≺ B
tst7.lean:4:42: Type of argument 2 must be convertible to the expected type in the application of
f
with arguments:
B
a
Assumed: myeq
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
Assumed: R
Assumed: h
λ (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)