--- a/src/HOL/Tools/recdef.ML Thu Jan 21 12:20:28 2010 +0100
+++ b/src/HOL/Tools/recdef.ML Thu Jan 21 14:13:21 2010 +0100
@@ -204,18 +204,13 @@
val simp_att =
if null tcs then [Simplifier.simp_add, Nitpick_Simps.add, Code.add_default_eqn_attribute]
else [];
- fun specs_of simps =
- let
- fun dest_eqn th = fst (strip_comb (fst (HOLogic.dest_eq (HOLogic.dest_Trueprop (prop_of th)))))
- val ts = distinct (op =) (map dest_eqn simps)
- in (ts, simps) end
val ((simps' :: rules', [induct']), thy) =
thy
|> Sign.add_path bname
|> PureThy.add_thmss
(((Binding.name "simps", flat rules), simp_att) :: ((eq_names ~~ rules) ~~ eq_atts))
||>> PureThy.add_thms [((Binding.name "induct", induct), [])]
- ||> Spec_Rules.add_global Spec_Rules.Equational (specs_of (flat rules));
+ ||> Spec_Rules.add_global Spec_Rules.Equational (tcs, flat rules);
val result = {simps = simps', rules = rules', induct = induct', tcs = tcs};
val thy =
thy