src/HOL/Tools/inductive_set.ML
changeset 54895 515630483010
parent 51717 9e7d1c139569
child 55990 41c6b99c5fb7
--- a/src/HOL/Tools/inductive_set.ML	Wed Jan 01 13:24:23 2014 +0100
+++ b/src/HOL/Tools/inductive_set.ML	Wed Jan 01 14:29:22 2014 +0100
@@ -406,8 +406,10 @@
 
 (**** preprocessor for code generator ****)
 
-fun codegen_preproc thy =
+(* FIXME unused!? *)
+fun codegen_preproc thy =  (* FIXME proper context!? *)
   let
+    val ctxt = Proof_Context.init_global thy;
     val {to_pred_simps, set_arities, pred_arities, ...} =
       Data.get (Context.Theory thy);
     fun preproc thm =
@@ -417,7 +419,7 @@
             forall is_none xs) arities) (prop_of thm)
       then
         thm |>
-        Simplifier.full_simplify (Simplifier.global_context thy HOL_basic_ss addsimprocs
+        Simplifier.full_simplify (put_simpset HOL_basic_ss ctxt addsimprocs
           [to_pred_simproc (mem_Collect_eq :: @{thm split_conv} :: to_pred_simps)]) |>
         eta_contract_thm (is_pred pred_arities)
       else thm