src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML
changeset 50267 1da2e67242d6
parent 50266 e8173d1fa725
child 50269 20a01c3e8072
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Wed Nov 28 12:25:43 2012 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_reconstruct.ML	Wed Nov 28 12:25:43 2012 +0100
@@ -28,7 +28,6 @@
 
   val smtN : string
   val string_for_reconstructor : reconstructor -> string
-  val thms_of_name : Proof.context -> string -> thm list
   val lam_trans_from_atp_proof : string proof -> string -> string
   val is_typed_helper_used_in_atp_proof : string proof -> bool
   val used_facts_in_atp_proof :
@@ -82,19 +81,6 @@
     metis_call type_enc lam_trans
   | string_for_reconstructor SMT = smtN
 
-fun thms_of_name ctxt name =
-  let
-    val lex = Keyword.get_lexicons
-    val get = maps (Proof_Context.get_fact ctxt o fst)
-  in
-    Source.of_string name
-    |> Symbol.source
-    |> Token.source {do_recover = SOME false} lex Position.start
-    |> Token.source_proper
-    |> Source.source Token.stopper (Parse_Spec.xthms1 >> get) NONE
-    |> Source.exhaust
-  end
-
 
 (** fact extraction from ATP proofs **)