Files
NNG/Game/MyNat/PeanoAxioms.lean
2023-10-11 17:53:51 +01:00

16 lines
454 B
Lean4
Raw Blame History

This file contains ambiguous Unicode characters
This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.
import Game.MyNat.Definition
import Mathlib.Tactic
namespace MyNat
-- KB note: I have not thought about simp at all and perhaps this
-- comes from some earlier NNG3 port?
attribute [-simp] MyNat.succ.injEq
-- example (a b : ) (h : (succ a) = b) : succ (succ a) = succ b := by
-- simp
-- sorry
theorem succ_inj (a b : ) : succ a = succ b a = b := by rintro h; rfl
theorem zero_ne_succ (a : ) : 0 succ a := by rintro h