lean2/tests/lean/induction1.lean.expected.out

15 lines
444 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Imported 'macros'
Using: Nat
Assumed: Induction
Proved: Comm1
Proved: Comm2
theorem Comm2 : ∀ n m : , n + m = m + n :=
λ n : ,
Induction
(λ x : , n + x == x + n)
(Nat::add::zeror n ⋈ symm (Nat::add::zerol n))
(λ (m : ) (iH : n + m = m + n),
Nat::add::succr n m ⋈ subst (refl (n + m + 1)) iH ⋈ symm (Nat::add::succl m n))