src/HOL/Tools/Function/scnp_reconstruct.ML
changeset 42361 23f352990944
parent 41493 f05976d69141
child 42774 6c999448c2bb
--- a/src/HOL/Tools/Function/scnp_reconstruct.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/Function/scnp_reconstruct.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -155,7 +155,7 @@
 
 fun reconstruct_tac ctxt D cs (GP (_, gs)) certificate =
   let
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val Multiset
           { msetT, mk_mset,
             mset_regroup_conv, mset_pwleq_tac, set_of_simps,
@@ -300,7 +300,7 @@
 
 fun single_scnp_tac use_tags orders ctxt D = Termination.CALLS (fn (cs, i) =>
   let
-    val ms_configured = is_some (Multiset_Setup.get (ProofContext.theory_of ctxt))
+    val ms_configured = is_some (Multiset_Setup.get (Proof_Context.theory_of ctxt))
     val orders' = if ms_configured then orders
                   else filter_out (curry op = MS) orders
     val gp = gen_probl D cs