lean2/tests/lean/run/rewrite8.lean

6 lines
166 B
Text

import data.nat
open nat
constant f : nat → nat
theorem tst1 (x y : nat) (H1 : (λ z, z + 0) x = y) : f x = f y :=
by rewrite [▸* at H1, nat.add_zero at H1, H1]