Skip to content

Commit

Permalink
mynat simp lemmas have 0 in so move from zero to 0
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Nov 1, 2023
1 parent 96be0b3 commit d29d187
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 5 deletions.
1 change: 0 additions & 1 deletion Game/MyNat/DecidableEq.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,6 @@ example : 4 ≠ 5 := by
example : (0 : ℕ) + 0 = 0 := by
MyDecide

set_option pp.all true in
example : (2 : ℕ) + 2 = 4 := by
MyDecide

Expand Down
5 changes: 1 addition & 4 deletions Game/MyNat/Definition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -33,11 +33,8 @@ instance instofNat {n : Nat} : OfNat MyNat n where
instance : ToString MyNat where
toString p := toString (toNat p)

@[simp]
theorem zero_eq_0 : MyNat.zero = 0 := rfl

@[MyNat_decide]
theorem zero_eq_zero : (0 : ℕ) = MyNat.zero := rfl
theorem zero_eq_0 : MyNat.zero = 0 := rfl

def one : MyNat := MyNat.succ 0

Expand Down

0 comments on commit d29d187

Please sign in to comment.