src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy
changeset 60649 e007aa6a8aa2
parent 59720 f893472fff31
child 60925 90659d0215bd
--- a/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy	Sun Jul 05 22:07:09 2015 +0200
+++ b/src/HOL/TPTP/TPTP_Proof_Reconstruction_Test.thy	Sun Jul 05 22:32:14 2015 +0200
@@ -329,10 +329,8 @@
 *}
 
 ML {*
-(*given a thm, show us the axioms in its thy*)
-val axms_of_thy_of_thm =
-  Thm.theory_of_thm
-  #> ` Theory.axioms_of
+val axms_of_thy =
+  `Theory.axioms_of
   #> apsnd cterm_of
   #> swap
   #> apsnd (map snd)
@@ -351,14 +349,8 @@
   *}
 
 ML {*
-fun leo2_tac_wrap prob_name step i = fn st =>
-  let
-    val ctxt =
-      Thm.theory_of_thm st
-      |> Proof_Context.init_global
-  in
-    rtac (interpret_leo2_inference ctxt prob_name step) i st
-  end
+fun leo2_tac_wrap ctxt prob_name step i st =
+  rtac (interpret_leo2_inference ctxt prob_name step) i st
 *}
 
 (*FIXME move these examples elsewhere*)