85379b7706
not (not (not a)) -> not a
29 lines
601 B
Text
29 lines
601 B
Text
constants a b c d : Prop
|
||
|
||
set_option blast.strategy "unit"
|
||
|
||
example (H : ¬ a → ¬ b → ¬ c ∨ ¬ d) : ¬ a → c → d → ¬ b → false :=
|
||
by blast
|
||
|
||
set_option blast.strategy "preprocess"
|
||
|
||
example : ¬¬¬¬¬a → ¬¬a → false :=
|
||
by blast
|
||
|
||
example : ¬¬¬¬¬a → ¬¬¬¬a → false :=
|
||
by blast
|
||
|
||
example : ¬¬¬¬¬a → a → false :=
|
||
by blast
|
||
|
||
example : ¬¬a → ¬¬¬¬¬a → false :=
|
||
by blast
|
||
|
||
example : ¬¬¬¬¬a → ¬¬¬¬¬¬¬¬a → false :=
|
||
by blast
|
||
|
||
example : ¬¬¬¬¬a → a → false :=
|
||
by blast
|
||
|
||
example : ¬¬¬¬¬¬¬¬a → ¬¬¬¬¬a → false :=
|
||
by blast
|