2015-03-26 00:42:34 +00:00
|
|
|
import data.nat
|
|
|
|
open nat
|
|
|
|
|
|
|
|
attribute nat.add [unfold-c 2]
|
|
|
|
attribute nat.rec_on [unfold-c 2]
|
|
|
|
|
|
|
|
example (a b c : nat) : a + 0 = 0 + a ∧ b + 0 = 0 + b :=
|
|
|
|
begin
|
|
|
|
apply and.intro,
|
2015-03-28 00:26:06 +00:00
|
|
|
all_goals esimp[of_num],
|
2015-03-26 00:42:34 +00:00
|
|
|
all_goals (state; rewrite zero_add)
|
|
|
|
end
|