src/HOL/Tools/Sledgehammer/clausifier.ML
changeset 37616 c8d2d84d6011
parent 37584 2e289dc13615
child 37617 f73cd4069f69
--- a/src/HOL/Tools/Sledgehammer/clausifier.ML	Mon Jun 28 13:36:21 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/clausifier.ML	Mon Jun 28 17:31:38 2010 +0200
@@ -9,12 +9,7 @@
 sig
   type cnf_thm = thm * ((string * int) * thm)
 
-  val sledgehammer_prefix: string
-  val chained_prefix: string
   val trace: bool Unsynchronized.ref
-  val trace_msg: (unit -> string) -> unit
-  val name_thms_pair_from_ref :
-    Proof.context -> thm list -> Facts.ref -> string * thm list
   val skolem_theory_name: string
   val skolem_prefix: string
   val skolem_infix: string
@@ -38,23 +33,10 @@
 
 type cnf_thm = thm * ((string * int) * thm)
 
-val sledgehammer_prefix = "Sledgehammer" ^ Long_Name.separator
-
-(* Used to label theorems chained into the goal. *)
-val chained_prefix = sledgehammer_prefix ^ "chained_"
-
 val trace = Unsynchronized.ref false;
 fun trace_msg msg = if !trace then tracing (msg ()) else ();
 
-fun name_thms_pair_from_ref ctxt chained_ths xref =
-  let
-    val ths = ProofContext.get_fact ctxt xref
-    val name = Facts.string_of_ref xref
-               |> forall (member Thm.eq_thm chained_ths) ths
-                  ? prefix chained_prefix
-  in (name, ths) end
-
-val skolem_theory_name = sledgehammer_prefix ^ "Sko"
+val skolem_theory_name = "Sledgehammer" ^ Long_Name.separator ^ "Sko"
 val skolem_prefix = "sko_"
 val skolem_infix = "$"
 
@@ -409,6 +391,7 @@
   end
 
 (* FIXME: put other record thms here, or declare as "no_atp" *)
+(* FIXME: move to "Sledgehammer_Fact_Filter" *)
 val multi_base_blacklist =
   ["defs", "select_defs", "update_defs", "induct", "inducts", "split", "splits",
    "split_asm", "cases", "ext_cases"];