src/Tools/Code/code_preproc.ML
changeset 42361 23f352990944
parent 41346 6673f6fa94ca
child 42383 0ae4ad40d7b5
--- a/src/Tools/Code/code_preproc.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/Tools/Code/code_preproc.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -90,7 +90,7 @@
 
 fun add_unfold_post raw_thm thy =
   let
-    val thm = Local_Defs.meta_rewrite_rule (ProofContext.init_global thy) raw_thm;
+    val thm = Local_Defs.meta_rewrite_rule (Proof_Context.init_global thy) raw_thm;
     val thm_sym = Thm.symmetric thm;
   in
     thy |> map_pre_post (fn (pre, post) =>
@@ -165,7 +165,7 @@
 
 fun preprocess_conv thy =
   let
-    val ctxt = ProofContext.init_global thy;
+    val ctxt = Proof_Context.init_global thy;
     val pre = (Simplifier.global_context thy o #pre o the_thmproc) thy;
   in
     Simplifier.rewrite pre
@@ -186,7 +186,7 @@
 
 fun print_codeproc thy =
   let
-    val ctxt = ProofContext.init_global thy;
+    val ctxt = Proof_Context.init_global thy;
     val pre = (#pre o the_thmproc) thy;
     val post = (#post o the_thmproc) thy;
     val functrans = (map fst o #functrans o the_thmproc) thy;