2015-11-30 16:43:08 +00:00
|
|
|
import data.nat
|
|
|
|
open nat
|
|
|
|
constant f : nat → nat
|
|
|
|
constant g : nat → nat
|
|
|
|
|
|
|
|
definition lemma1 [forward] : ∀ x, (:g (f x):) = x :=
|
|
|
|
sorry
|
|
|
|
|
2015-12-06 23:01:49 +00:00
|
|
|
set_option blast.strategy "ematch"
|
2015-11-30 16:43:08 +00:00
|
|
|
|
|
|
|
example (a b c : nat) : a = f b → a = f c → g a ≠ b → false :=
|
|
|
|
by blast
|