merged
authorhuffman
Mon, 22 Mar 2010 16:02:51 -0700
changeset 35913 6943a36453e8
parent 35912 b0e300bd3a2c (current diff)
parent 35911 2062295537e0 (diff)
child 35914 91a7311177c4
merged
--- a/src/HOL/Predicate_Compile.thy	Mon Mar 22 15:53:25 2010 -0700
+++ b/src/HOL/Predicate_Compile.thy	Mon Mar 22 16:02:51 2010 -0700
@@ -1,4 +1,3 @@
-
 (*  Title:      HOL/Predicate_Compile.thy
     Author:     Stefan Berghofer, Lukas Bulwahn, Florian Haftmann, TU Muenchen
 *)
--- a/src/HOL/Tools/Datatype/datatype_codegen.ML	Mon Mar 22 15:53:25 2010 -0700
+++ b/src/HOL/Tools/Datatype/datatype_codegen.ML	Mon Mar 22 16:02:51 2010 -0700
@@ -358,7 +358,7 @@
       [trueprop $ false_eq (t1, t2), trueprop $ false_eq (t2, t1)];
     val distincts = maps prep_distinct (snd (nth (Datatype_Prop.make_distincts [descr] vs) index));
     val refl = HOLogic.mk_Trueprop (true_eq (Free ("x", ty), Free ("x", ty)));
-    val simpset = Simplifier.context (ProofContext.init thy) (HOL_basic_ss addsimps 
+    val simpset = Simplifier.global_context thy (HOL_basic_ss addsimps 
       (map Simpdata.mk_eq (@{thm eq} :: @{thm eq_True} :: inject_thms @ distinct_thms)));
     fun prove prop = Skip_Proof.prove_global thy [] [] prop (K (ALLGOALS (simp_tac simpset)))
       |> Simpdata.mk_eq;