lean2/tests/lean/run/blast13.lean

16 lines
337 B
Text
Raw Normal View History

import data.list
open perm
set_option blast.strategy "cc"
example (p : Prop) (l : list nat) : ¬ l ~ l → p :=
by blast
example (a : nat) : ¬ a = a → false :=
by blast
example (A : Type) (p : Prop) (a b c : A) : a = b → ¬ b = a → p :=
by blast
example (A : Type) (p : Prop) (a b c : A) : a = b → b ≠ a → p :=
by blast