lean2/tests/lean/induction2.lean.expected.out

31 lines
1.1 KiB
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Imported 'macros'
Using: Nat
Assumed: Induction
Failed to solve
⊢ ∀ m : , 0 + m = m + 0 ≺ ?M::3 0
induction2.lean:10:3: Type of argument 2 must be convertible to the expected type in the application of
Induction
with arguments:
?M::3
λ m : , trans (Nat::add_zerol m) (symm (Nat::add_zeror m))
λ (n : ) (iH : (?M::3[lift:0:1]) n) (m : ),
@trans
(n + 1 + m)
(m + n + 1)
(m + (n + 1))
(@trans
(n + 1 + m)
(n + m + 1)
(m + n + 1)
(Nat::add_succl n m)
(@subst ?M::14
?M::15
?M::16
(λ x : ?M::14,
@eq ((?M::48[lift:0:1]) x) ((?M::49[lift:0:1]) x) ((?M::50[lift:0:1]) x))
(refl (n + m + 1))
iH))
(symm (Nat::add_succr m n))