src/HOL/Tools/Sledgehammer/sledgehammer_proof_methods.ML
changeset 58074 87a8cc594bf6
parent 58073 1cd45fec98e2
child 58075 95bab16eac45
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_proof_methods.ML	Thu Aug 28 16:58:27 2014 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_proof_methods.ML	Thu Aug 28 16:58:27 2014 +0200
@@ -32,7 +32,6 @@
   type one_line_params =
     ((string * stature) list * (proof_method * play_outcome)) * string * int * int
 
-  val skolem_tac : Proof.context -> int -> tactic
   val is_proof_method_direct : proof_method -> bool
   val string_of_proof_method : Proof.context -> string list -> proof_method -> string
   val tac_of_proof_method : Proof.context -> thm list * thm list -> proof_method -> int -> tactic
@@ -49,10 +48,6 @@
 open ATP_Problem_Generate
 open ATP_Proof_Reconstruct
 
-fun skolem_tac ctxt =
-  TRY o Atomize_Elim.atomize_elim_tac ctxt THEN'
-  SELECT_GOAL (Clasimp.auto_tac (ctxt addSIs @{thms choice}) THEN ALLGOALS (blast_tac ctxt))
-
 datatype proof_method =
   Metis_Method of string option * string option |
   Meson_Method |