2015-12-06 22:33:21 +00:00
|
|
|
set_option blast.strategy "cc"
|
|
|
|
|
2015-12-03 07:28:57 +00:00
|
|
|
constant R : nat → nat → Prop
|
|
|
|
axiom R_trans : ∀ a b c, R a b → R b c → R a c
|
|
|
|
attribute R_trans [trans]
|
|
|
|
|
|
|
|
set_option blast.subst false
|
|
|
|
|
|
|
|
example (a b c : nat) : a = b → R a b → R a a :=
|
|
|
|
by blast
|