lean2/tests/lean/run/blast_cc1.lean
2015-12-09 12:23:00 -08:00

24 lines
569 B
Text

import data.list
constant f {A : Type} : A → A → A
constant g : nat → nat
set_option blast.strategy "cc"
example (a b c : nat) : a = b → g a == g b :=
by blast
example (a b c : nat) : a = b → c = b → f (f a b) (g c) = f (f c a) (g b) :=
by blast
example (a b c d e x y : nat) : a = b → a = x → b = y → c = d → c = e → c = b → a = e :=
by blast
open perm
example (a b c d : list nat) : a ~ b → c ~ b → d ~ c → a ~ d :=
by blast
set_option trace.cc true
example (a b c d : list nat) : a ~ b → c ~ b → d = c → a ~ d :=
by blast