src/HOL/TPTP/TPTP_Proof_Reconstruction.thy
changeset 59639 f596ed647018
parent 59621 291934bac95e
child 59755 f8d164ab0dc1
--- a/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy	Fri Mar 06 23:54:05 2015 +0100
+++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction.thy	Fri Mar 06 23:54:36 2015 +0100
@@ -806,8 +806,6 @@
 ML {*
 fun instantiate_skols ctxt consts_candidates i = fn st =>
   let
-    val thy = Proof_Context.theory_of ctxt
-
     val gls =
       Thm.prop_of st
       |> Logic.strip_horn
@@ -917,7 +915,7 @@
     (* val contextualise = fold absdummy (map snd params) *)
     val contextualise = fold absfree params
 
-    val skolem_cts = map (contextualise #> Thm.global_cterm_of thy) skolem_terms
+    val skolem_cts = map (contextualise #> Thm.cterm_of ctxt) skolem_terms
 
 
 (*now the instantiation code*)
@@ -937,7 +935,7 @@
         fun make_var pre_var =
           the_single pre_var
           |> Var
-          |> Thm.global_cterm_of thy
+          |> Thm.cterm_of ctxt
           |> SOME
       in
         if null pre_var then NONE
@@ -2003,7 +2001,7 @@
      thy
      prob_name (#meta pannot) n
       |> the
-      |> (fn {inference_fmla, ...} => Thm.global_cterm_of thy inference_fmla)
+      |> (fn {inference_fmla, ...} => Thm.cterm_of ctxt inference_fmla)
       |> oracle_iinterp
   end
 *}