12 lines
264 B
Text
12 lines
264 B
Text
|
set_option blast.init_depth 10
|
|||
|
set_option blast.inc_depth 100
|
|||
|
set_option blast.trace 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
|