src/HOL/Tools/SMT/smt_normalize.ML
changeset 42361 23f352990944
parent 42190 b6b5846504cd
child 43116 e0add071fa10
--- a/src/HOL/Tools/SMT/smt_normalize.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/SMT/smt_normalize.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -170,7 +170,7 @@
     (case Term.strip_comb t of
       (Const c, ts as _ :: _) =>
         not (SMT_Builtin.is_builtin_fun_ext ctxt c ts) andalso
-        forall (is_constr_pat (ProofContext.theory_of ctxt)) ts
+        forall (is_constr_pat (Proof_Context.theory_of ctxt)) ts
     | _ => false)
 
   fun has_all_vars vs t =
@@ -218,7 +218,7 @@
       val (lhs, rhs) = dest_cond_eq ct
 
       val vs = map Thm.term_of cvs
-      val thy = ProofContext.theory_of ctxt
+      val thy = Proof_Context.theory_of ctxt
 
       fun get_mpats ct =
         if is_simp_lhs ctxt (Thm.term_of ct) then minimal_pats vs ct