2015-02-06 20:57:42 +00:00
|
|
|
import data.nat
|
|
|
|
open nat
|
|
|
|
|
2015-07-07 23:37:06 +00:00
|
|
|
definition f [unfold 2] (x y z : nat) : nat :=
|
2015-02-06 20:57:42 +00:00
|
|
|
x + y + z
|
|
|
|
|
2015-07-07 23:37:06 +00:00
|
|
|
attribute of_num [unfold 1]
|
2015-02-06 20:57:42 +00:00
|
|
|
|
|
|
|
example (x y : nat) (H1 : f x 0 0 = 0) : x = 0 :=
|
|
|
|
begin
|
2015-10-14 19:27:09 +00:00
|
|
|
rewrite [↑f at H1, 4>nat.add_zero at H1, H1]
|
2015-02-06 20:57:42 +00:00
|
|
|
end
|