merged
authorwenzelm
Mon, 22 Mar 2010 22:56:46 +0100
changeset 35909 a4ed7aaa7d03
parent 35901 12f09bf2c77f (current diff)
parent 35899 e810f73c8ee2 (diff)
child 35910 400822011088
merged
--- a/src/HOL/Predicate_Compile.thy	Mon Mar 22 13:27:35 2010 -0700
+++ b/src/HOL/Predicate_Compile.thy	Mon Mar 22 22:56:46 2010 +0100
@@ -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 13:27:35 2010 -0700
+++ b/src/HOL/Tools/Datatype/datatype_codegen.ML	Mon Mar 22 22:56:46 2010 +0100
@@ -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;