lean2/tests/lean/run/blast16.lean

10 lines
202 B
Text
Raw Normal View History

2015-12-09 04:06:43 +00:00
set_option trace.blast true
example (p q : Prop) : p q → q p :=
by blast
definition lemma1 (p q r s : Prop) (a b : nat) : r s → p q → a = b → q p :=
by blast
print lemma1