2014-01-07 13:24:46 -08:00
|
|
|
|
Set: pp::colors
|
|
|
|
|
Set: pp::unicode
|
|
|
|
|
Imported 'macros'
|
|
|
|
|
Using: Nat
|
|
|
|
|
Assumed: Induction
|
|
|
|
|
Failed to solve
|
2014-01-08 00:38:39 -08:00
|
|
|
|
⊢ ∀ m : ℕ, 0 + m == m + 0 ≺ ?M::3 0
|
2014-01-09 12:15:12 -08:00
|
|
|
|
induction2.lean:10:3: Type of argument 2 must be convertible to the expected type in the application of
|
2014-01-08 00:38:39 -08:00
|
|
|
|
Induction
|
|
|
|
|
with arguments:
|
|
|
|
|
?M::3
|
2014-01-09 08:33:52 -08:00
|
|
|
|
λ m : ℕ, Nat::add_zerol m ⋈ symm (Nat::add_zeror m)
|
2014-01-08 00:38:39 -08:00
|
|
|
|
λ (n : ℕ) (iH : ?M::3 n) (m : ℕ),
|
2014-01-09 08:33:52 -08:00
|
|
|
|
Nat::add_succl n m ⋈ subst (refl (n + m + 1)) iH ⋈ symm (Nat::add_succr m n)
|