auto-minimizer should respect "isar_proofs = true"
authorblanchet
Wed, 20 Feb 2013 08:44:24 +0100
changeset 51191 89e9e945a005
parent 51190 2654b3965c8d
child 51192 4dc6bb65c3c3
auto-minimizer should respect "isar_proofs = true"
src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML	Wed Feb 20 08:44:24 2013 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML	Wed Feb 20 08:44:24 2013 +0100
@@ -295,7 +295,11 @@
             in
               (case Lazy.force preplay of
                  Played (reconstr as Metis _, timeout) =>
-                 if can_min_fast_enough timeout then
+                 if isar_proofs = SOME true then
+                   (* Cheat: Assume the original prover is as fast as "metis"
+                      for the goal it proved itself. *)
+                   (can_min_fast_enough timeout, (name, params))
+                 else if can_min_fast_enough timeout then
                    (true, extract_reconstructor params reconstr
                           ||> (fn override_params =>
                                   adjust_reconstructor_params override_params
@@ -303,7 +307,7 @@
                  else
                    (prover_fast_enough (), (name, params))
                | Played (SMT, timeout) =>
-                 (* Cheat: assume the original prover is as fast as "smt" for
+                 (* Cheat: Assume the original prover is as fast as "smt" for
                     the goal it proved itself *)
                  (can_min_fast_enough timeout, (name, params))
                | _ => (prover_fast_enough (), (name, params)),