src/HOL/Tools/Sledgehammer/clausifier.ML
changeset 37584 2e289dc13615
parent 37574 b8c1f4c46983
child 37616 c8d2d84d6011
--- a/src/HOL/Tools/Sledgehammer/clausifier.ML	Fri Jun 25 18:05:36 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/clausifier.ML	Fri Jun 25 18:34:06 2010 +0200
@@ -25,8 +25,8 @@
   val is_theorem_bad_for_atps: thm -> bool
   val type_has_topsort: typ -> bool
   val cnf_rules_pairs : theory -> (string * thm) list -> cnf_thm list
-  val saturate_skolem_cache: theory -> theory option
-  val auto_saturate_skolem_cache: bool Unsynchronized.ref
+  val saturate_cache: theory -> theory option
+  val auto_saturate_cache: bool Unsynchronized.ref
   val neg_clausify: thm -> thm list
   val neg_conjecture_clauses:
     Proof.context -> thm -> int -> thm list list * (string * typ) list
@@ -504,7 +504,7 @@
 
 in
 
-fun saturate_skolem_cache thy =
+fun saturate_cache thy =
   let
     val facts = PureThy.facts_of thy;
     val new_facts = (facts, []) |-> Facts.fold_static (fn (name, ths) =>
@@ -536,10 +536,10 @@
 end;
 
 (* For emergency use where the Skolem cache causes problems. *)
-val auto_saturate_skolem_cache = Unsynchronized.ref true
+val auto_saturate_cache = Unsynchronized.ref true
 
-fun conditionally_saturate_skolem_cache thy =
-  if !auto_saturate_skolem_cache then saturate_skolem_cache thy else NONE
+fun conditionally_saturate_cache thy =
+  if !auto_saturate_cache then saturate_cache thy else NONE
 
 
 (*** Converting a subgoal into negated conjecture clauses. ***)
@@ -565,7 +565,7 @@
 (** setup **)
 
 val setup =
-  perhaps conditionally_saturate_skolem_cache
-  #> Theory.at_end conditionally_saturate_skolem_cache
+  perhaps conditionally_saturate_cache
+  #> Theory.at_end conditionally_saturate_cache
 
 end;