src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
changeset 62093 bd73a2279fcd
parent 61877 276ad4354069
child 62095 7edf47be2baf
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML	Thu Jan 07 15:50:09 2016 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML	Thu Jan 07 15:53:39 2016 +0100
@@ -83,9 +83,6 @@
 
 val backquote = enclose "\<open>" "\<close>"
 
-(* unfolding these can yield really huge terms *)
-val risky_defs = @{thms Bit0_def Bit1_def}
-
 fun is_rec_eq lhs = Term.exists_subterm (curry (op =) (head_of lhs))
 
 fun is_rec_def (@{const Trueprop} $ t) = is_rec_def t
@@ -324,7 +321,6 @@
         val (rec_defs, nonrec_defs) = specs
           |> filter (curry (op =) Spec_Rules.Equational o fst)
           |> maps (snd o snd)
-          |> filter_out (member Thm.eq_thm_prop risky_defs)
           |> List.partition (is_rec_def o Thm.prop_of)
         val spec_intros = specs
           |> filter (member (op =) [Spec_Rules.Inductive, Spec_Rules.Co_Inductive] o fst)