src/HOL/ex/sledgehammer_tactics.ML
changeset 42361 23f352990944
parent 42106 ed1d40888b1b
child 42443 724e612ba248
--- a/src/HOL/ex/sledgehammer_tactics.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/ex/sledgehammer_tactics.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -55,7 +55,7 @@
 fun thms_of_name ctxt name =
   let
     val lex = Keyword.get_lexicons
-    val get = maps (ProofContext.get_fact ctxt o fst)
+    val get = maps (Proof_Context.get_fact ctxt o fst)
   in
     Source.of_string name
     |> Symbol.source
@@ -77,7 +77,7 @@
 
 fun generic_sledgehammer_as_oracle_tac force_full_types ctxt i th =
   let
-    val thy = ProofContext.theory_of ctxt
+    val thy = Proof_Context.theory_of ctxt
     val timeout = Time.fromSeconds 30
     val xs = run_atp force_full_types timeout i i ctxt th atp
   in if is_some xs then Skip_Proof.cheat_tac thy th else Seq.empty end