src/HOL/Tools/Sledgehammer/sledgehammer_atp_reconstruct.ML
changeset 42361 23f352990944
parent 42227 662b50b7126f
child 42449 494e4ac5b0f8
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_atp_reconstruct.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_atp_reconstruct.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -457,7 +457,7 @@
 
 fun check_formula ctxt =
   Type.constraint HOLogic.boolT
-  #> Syntax.check_term (ProofContext.set_mode ProofContext.mode_schematic ctxt)
+  #> Syntax.check_term (Proof_Context.set_mode Proof_Context.mode_schematic ctxt)
 
 
 (**** Translation of TSTP files to Isar Proofs ****)
@@ -467,7 +467,7 @@
 
 fun decode_line type_sys tfrees (Definition (name, phi1, phi2)) ctxt =
     let
-      val thy = ProofContext.theory_of ctxt
+      val thy = Proof_Context.theory_of ctxt
       val t1 = prop_from_formula thy type_sys tfrees phi1
       val vars = snd (strip_comb t1)
       val frees = map unvarify_term vars
@@ -483,7 +483,7 @@
     end
   | decode_line type_sys tfrees (Inference (name, u, deps)) ctxt =
     let
-      val thy = ProofContext.theory_of ctxt
+      val thy = Proof_Context.theory_of ctxt
       val t = u |> prop_from_formula thy type_sys tfrees
                 |> uncombine_term |> check_formula ctxt
     in