Skip to content

Commit

Permalink
test
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 committed Apr 1, 2019
1 parent 3e21b01 commit d56fd56
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/data/nat/basic.lean
Expand Up @@ -17,7 +17,7 @@ variables {m n k : ℕ}
-- mediated operations.
@[simp] theorem add_def {a b : ℕ} : nat.add a b = a + b := rfl
@[simp] theorem mul_def {a b : ℕ} : nat.mul a b = a * b := rfl

lemma two_add_Two : 2 + 2 = 4 := rfl
attribute [simp] nat.add_sub_cancel nat.add_sub_cancel_left
attribute [simp] nat.sub_self

Expand Down

0 comments on commit d56fd56

Please sign in to comment.