src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML
changeset 39452 70a57e40f795
parent 39366 f58fbb959826
child 39491 2416666e6f94
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML	Thu Sep 16 09:59:32 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML	Thu Sep 16 11:12:08 2010 +0200
@@ -117,7 +117,7 @@
          val new_timeout =
            Int.min (msecs, Time.toMilliseconds time + fudge_msecs)
            |> Time.fromMilliseconds
-         val (min_thms, {proof, axiom_names, ...}) =
+         val (min_thms, {tstplike_proof, axiom_names, ...}) =
            sublinear_minimize (do_test new_timeout)
                (filter_used_facts used_thm_names axioms) ([], result)
          val n = length min_thms
@@ -130,8 +130,8 @@
          (SOME min_thms,
           proof_text isar_proof
               (pool, debug, isar_shrink_factor, ctxt, conjecture_shape)
-              ("Minimized command", full_types, K "", proof, axiom_names, goal,
-               i) |> fst)
+              ("Minimized command", full_types, K "", tstplike_proof,
+               axiom_names, goal, i) |> fst)
        end
      | {outcome = SOME TimedOut, ...} =>
        (NONE, "Timeout: You can increase the time limit using the \"timeout\" \