lean2/tests/lean/elab1.lean.expected.out

58 lines
1.6 KiB
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Assumed: f
Failed to solve
⊢ Bool ≺
(line: 2: pos: 6) Type of argument 3 must be convertible to the expected type in the application of
@f
with arguments:
10
Assumed: g
Error (line: 5, pos: 8) invalid expression, it still contains metavariables after elaboration, metavariable: ?M::1, type:
Type
Assumed: h
Failed to solve
x : ?M::0, A : Type ⊢ ?M::0 ≺ A
(line: 9: pos: 27) Type of argument 2 must be convertible to the expected type in the application of
h
with arguments:
A
x
Assumed: my_eq
Failed to solve
A : Type, B : Type, a : ?M::0, b : ?M::1, C : Type ⊢ ?M::0[lift:0:3] ≺ C
(line: 13: pos: 51) Type of argument 2 must be convertible to the expected type in the application of
my_eq
with arguments:
C
a
b
Assumed: a
Assumed: b
Assumed: H
Failed to solve
⊢ ∀ H1 : ?M::0, ?M::1 ∧ a ≺ b
(line: 18: pos: 18) Type of definition 't1' must be convertible to expected type.
Failed to solve
⊢ b == b ≺ a == b
(line: 20: pos: 22) Type of argument 6 must be convertible to the expected type in the application of
@trans
with arguments:
?M::1
a
a
b
refl a
refl b
Failed to solve
⊢ ?M::1 ≺ Type
(line: 22: pos: 6) Type of argument 1 must be convertible to the expected type in the application of
@f
with arguments:
?M::0
Bool
Bool
Error (line: 25, pos: 19) unknown identifier 'EM'