lean2/tests/lean/run/blast_cc_missed.lean
Leonardo de Moura 19bfbe2df8 fix(library/blast/congruence_closure): uselist initialization (aka add_occurrence)
Make sure it matches the description in the paper.
2016-01-16 19:53:36 -08:00

13 lines
414 B
Text

set_option blast.strategy "cc"
example (C : nat → Type) (f : Π n, C n → C n) (n m : nat) (c : C n) (d : C m) :
f n == f m → c == d → n == m → f n c == f m d :=
by blast
example (f : nat → nat → nat) (a b c d : nat) :
c = d → f a = f b → f a c = f b d :=
by blast
example (f : nat → nat → nat) (a b c d : nat) :
c == d → f a == f b → f a c == f b d :=
by blast