lean2/tests/lean/run/blast_ematch2.lean

13 lines
219 B
Text
Raw Normal View History

import data.nat
open nat
constant f : nat → nat
constant g : nat → nat
definition lemma1 [forward] : ∀ x, g (f x) = x :=
sorry
set_option blast.ematch true
example (a b : nat) : f a = f b → a = b :=
by blast