src/Tools/coherent.ML
changeset 42361 23f352990944
parent 41228 e1fce873b814
child 42488 4638622bcaa1
--- a/src/Tools/coherent.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/Tools/coherent.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -82,7 +82,7 @@
   | valid_conj ctxt facts env (t :: ts) =
       Seq.maps (fn (u, x) => Seq.map (apsnd (cons x))
         (valid_conj ctxt facts
-           (Pattern.match (ProofContext.theory_of ctxt) (t, u) env) ts
+           (Pattern.match (Proof_Context.theory_of ctxt) (t, u) env) ts
          handle Pattern.MATCH => Seq.empty))
           (Seq.of_list (sort (int_ord o pairself snd) (Net.unify_term facts t)));
 
@@ -219,7 +219,7 @@
            (mk_dom xs) Net.empty 0 0 of
          NONE => no_tac
        | SOME prf =>
-           rtac (thm_of_cl_prf (ProofContext.theory_of context) concl [] prf) 1
+           rtac (thm_of_cl_prf (Proof_Context.theory_of context) concl [] prf) 1
     end) context 1) ctxt;
 
 val setup = Method.setup @{binding coherent}