Skip to content

Commit

Permalink
remove dead code
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Nov 12, 2023
1 parent 2bf6c63 commit 0acd296
Showing 1 changed file with 0 additions and 6 deletions.
6 changes: 0 additions & 6 deletions Game/MyNat/Addition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -22,9 +22,3 @@ If `a` and `d` are natural numbers, then `add_succ a d` is the proof that
-/
@[MyNat_decide]
axiom add_succ (a d : MyNat) : a + (succ d) = succ (a + d)

-- -- don't tell the viewers, we cheat with decide because
-- -- we used axioms to define nat
-- @[MyNat_decide]
-- theorem toNat_add (m n : MyNat) : (m + n).toNat = m.toNat + n.toNat := by
-- induction n <;> simp [MyNat_decide, Nat.add_succ, *];

0 comments on commit 0acd296

Please sign in to comment.