2015-02-06 19:03:36 +00:00
|
|
|
import data.nat
|
2015-10-14 19:27:09 +00:00
|
|
|
open nat algebra
|
2015-02-06 19:03:36 +00:00
|
|
|
constant f : nat → nat
|
|
|
|
|
|
|
|
example (x y : nat) (H1 : (λ z, z + 0) x = y) : f x = f y :=
|
2015-10-13 22:39:03 +00:00
|
|
|
by rewrite [▸* at H1, add_zero at H1, H1]
|
2015-02-06 19:03:36 +00:00
|
|
|
|
|
|
|
example (x y : nat) (H1 : (λ z, z + 0) x = y) : f x = f y :=
|
2015-10-13 22:39:03 +00:00
|
|
|
by rewrite [▸* at H1, add_zero at H1, H1]
|