lean2/tests/lean/run/blast_ematch10.lean

8 lines
187 B
Text

attribute iff [reducible]
set_option blast.strategy "ematch"
definition lemma1 (p : nat → Prop) (a b c : nat) : p a → a = b → p b :=
by blast
set_option pp.beta true
print lemma1