85409a59d3
closes #511
14 lines
370 B
Text
14 lines
370 B
Text
import data.nat
|
|
open nat
|
|
|
|
example (a b : nat) (f : nat → nat) (h : f (succ a) = 0) : f (a+1) = 0 :=
|
|
by rewrite [add_one, h]
|
|
|
|
example (a b : nat) (f : nat → nat) (h : f (succ a) = 0) : f (a+1) = 0 :=
|
|
by xrewrite h
|
|
|
|
definition g (a : nat) := a + 1
|
|
definition h (a : nat) := a
|
|
|
|
example (a b : nat) (f : nat → nat) (h : f (g (h a)) = 0) : f (a+1) = 0 :=
|
|
by krewrite h
|