src/HOL/Tools/Sledgehammer/sledgehammer.ML
changeset 39005 42fcb25de082
parent 39004 f1b465f889b5
child 39007 aae6a0d33c66
--- a/src/HOL/Tools/Sledgehammer/sledgehammer.ML	Wed Sep 01 23:04:47 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer.ML	Wed Sep 01 23:10:01 2010 +0200
@@ -31,8 +31,7 @@
     {ctxt: Proof.context,
      goal: thm,
      subgoal: int,
-     axiom_ts: term list,
-     prepared_axioms: ((string * locality) * fol_formula) option list}
+     axioms: (term * ((string * locality) * fol_formula) option) list}
   type prover_result =
     {outcome: failure option,
      message: string,
@@ -101,8 +100,7 @@
   {ctxt: Proof.context,
    goal: thm,
    subgoal: int,
-   axiom_ts: term list,
-   prepared_axioms: ((string * locality) * fol_formula) option list}
+   axioms: (term * ((string * locality) * fol_formula) option) list}
 
 type prover_result =
   {outcome: failure option,
@@ -220,13 +218,11 @@
          use_conjecture_for_hypotheses}
         ({debug, verbose, overlord, full_types, explicit_apply,
           max_relevant, isar_proof, isar_shrink_factor, timeout, ...} : params)
-        minimize_command
-        ({ctxt, goal, subgoal, axiom_ts, prepared_axioms} : problem) =
+        minimize_command ({ctxt, goal, subgoal, axioms} : problem) =
   let
     val (_, hyp_ts, concl_t) = strip_subgoal goal subgoal
     val max_relevant = the_default default_max_relevant max_relevant
-    val axiom_ts = take max_relevant axiom_ts
-    val prepared_axioms = take max_relevant prepared_axioms
+    val axioms = take max_relevant axioms
     (* path to unique problem file *)
     val the_dest_dir = if overlord then getenv "ISABELLE_HOME_USER"
                        else Config.get ctxt dest_dir
@@ -288,8 +284,7 @@
             val readable_names = debug andalso overlord
             val (problem, pool, conjecture_offset, axiom_names) =
               prepare_problem ctxt readable_names explicit_forall full_types
-                              explicit_apply hyp_ts concl_t axiom_ts
-                              prepared_axioms
+                              explicit_apply hyp_ts concl_t axioms
             val ss = strings_for_tptp_problem use_conjecture_for_hypotheses
                                               problem
             val _ = File.write_list probfile ss
@@ -368,8 +363,7 @@
       let
         val problem =
           {ctxt = ctxt, goal = goal, subgoal = i,
-           axiom_ts = map (prop_of o snd) axioms,
-           prepared_axioms = map (prepare_axiom ctxt) axioms}
+           axioms = map (prepare_axiom ctxt) axioms}
         val (outcome_code, message) =
           prover_fun atp_name prover params (minimize_command atp_name) problem
           |> (fn {outcome, message, ...} =>