src/HOL/Tools/SMT/smt_datatypes.ML
changeset 42361 23f352990944
parent 41426 09615ed31f04
child 43385 9cd4b4ecb4dd
--- a/src/HOL/Tools/SMT/smt_datatypes.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/SMT/smt_datatypes.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -62,7 +62,7 @@
 fun get_record_decl ({ext_def, ...} : Record.info) T ctxt =
   let
     val (con, _) = Term.dest_Const (lhs_head_of ext_def)
-    val (fields, more) = Record.get_extT_fields (ProofContext.theory_of ctxt) T
+    val (fields, more) = Record.get_extT_fields (Proof_Context.theory_of ctxt) T
     val fieldTs = map snd fields @ [snd more]
 
     val constr = Const (con, fieldTs ---> T)
@@ -89,7 +89,7 @@
 fun declared declss T = exists (exists (equal T o fst)) declss
 
 fun get_decls T n Ts ctxt =
-  let val thy = ProofContext.theory_of ctxt
+  let val thy = Proof_Context.theory_of ctxt
   in
     (case Datatype.get_info thy n of
       SOME info => get_datatype_decl info n Ts ctxt