src/HOL/Tools/lin_arith.ML
changeset 42361 23f352990944
parent 41468 0e4f6cf20cdf
child 42439 9efdd0af15ac
--- a/src/HOL/Tools/lin_arith.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/lin_arith.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -267,7 +267,7 @@
 
 fun decomp ctxt : term -> decomp option =
   let
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val {discrete, inj_consts, ...} = get_arith_data ctxt
   in decomp_negation (thy, discrete, inj_consts) end;
 
@@ -336,7 +336,7 @@
 fun split_once_items ctxt (Ts : typ list, terms : term list) :
                      (typ list * term list) list option =
 let
-  val thy = ProofContext.theory_of ctxt
+  val thy = Proof_Context.theory_of ctxt
   (* takes a list  [t1, ..., tn]  to the term                                *)
   (*   tn' --> ... --> t1' --> False  ,                                      *)
   (* where ti' = HOLogic.dest_Trueprop ti                                    *)
@@ -709,7 +709,7 @@
 fun split_once_tac ss split_thms =
   let
     val ctxt = Simplifier.the_context ss
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val cond_split_tac = SUBGOAL (fn (subgoal, i) =>
       let
         val Ts = rev (map snd (Logic.strip_params subgoal))