test(tests/lean/run/blast_simp4): add simp test
This commit is contained in:
parent
ac0bd539b0
commit
a35fd06a33
1 changed files with 15 additions and 0 deletions
15
tests/lean/run/blast_simp4.lean
Normal file
15
tests/lean/run/blast_simp4.lean
Normal file
|
@ -0,0 +1,15 @@
|
|||
import data.nat
|
||||
open nat
|
||||
|
||||
constant f : nat → nat
|
||||
definition g (a : nat) := a
|
||||
|
||||
|
||||
example (a b : nat) : a + 0 = 0 + g b → f (f b) = f (f a) :=
|
||||
suppose a + 0 = 0 + g b,
|
||||
assert a = b, by unfold g at *; simp,
|
||||
by simp
|
||||
|
||||
attribute g [reducible]
|
||||
example (a b : nat) : a + 0 = 0 + g b → f (f b) = f (f a) :=
|
||||
by simp
|
Loading…
Reference in a new issue