src/HOL/Tools/SMT/smt_builtin.ML
changeset 42361 23f352990944
parent 41473 3717fc42ebe9
child 46042 ab32a87ba01a
--- a/src/HOL/Tools/SMT/smt_builtin.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/SMT/smt_builtin.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -73,7 +73,7 @@
   SMT_Utils.dict_merge (Ord_List.merge typ_ord) ttabp
 
 fun lookup_ttab ctxt ttab T =
-  let fun match (U, _) = Sign.typ_instance (ProofContext.theory_of ctxt) (T, U)
+  let fun match (U, _) = Sign.typ_instance (Proof_Context.theory_of ctxt) (T, U)
   in
     get_first (find_first match)
       (SMT_Utils.dict_lookup ttab (SMT_Config.solver_class_of ctxt))