lean2/tests/lean/run/rewriter14.lean
2015-02-06 12:57:42 -08:00

12 lines
222 B
Text

import data.nat
open nat
definition f [unfold-c 2] (x y z : nat) : nat :=
x + y + z
attribute of_num [unfold-c 1]
example (x y : nat) (H1 : f x 0 0 = 0) : x = 0 :=
begin
rewrite [▸* at H1, 4>add_zero at H1, H1]
end