lean2/tests/lean/tst7.lean.expected.out
Leonardo de Moura a3bbd9fbb5 Minimize use the colors in tests. The colors make the diff hard to read
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-09-01 10:34:57 -07:00

15 lines
475 B
Text

Set option: pp::colors
Assumed: f
λ (A B : Type) (a : B), f B a
Error (line: 5, pos: 40) application type mismatch during term elaboration at term
f B a
Elaborator state
?M0 := [unassigned]
?M1 := [unassigned]
#0 ≈ lift:0:2 ?M0
Assumed: myeq
myeq (Π (A : Type) (a : A), A) (λ (A : Type) (a : A), a) (λ (B : Type) (b : B), b)
Bool
Assumed: R
Assumed: h
Bool → (Π (f1 g1 : Π A : Type, R A) (G : Π A : Type, myeq (R A) (f1 A) (g1 A)), Bool)