lean2/tests/lean/run/all_goals.lean
2015-03-27 17:54:48 -07:00

12 lines
245 B
Text

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,
all_goals esimp[of_num],
all_goals (state; rewrite zero_add)
end