src/HOL/Tools/Sledgehammer/sledgehammer_minimize_isar.ML
changeset 54813 c8b04da1bd01
parent 54754 6b0ca7f79e93
child 54826 79745ba60a5a
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_minimize_isar.ML	Wed Dec 18 22:55:43 2013 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_minimize_isar.ML	Thu Dec 19 09:28:20 2013 +0100
@@ -28,8 +28,7 @@
   | min_deps_of_step {get_preplay_time, set_preplay_time, preplay_quietly, ...}
       (step as Prove (qs, xs, l, t, subproofs, ((lfs, gfs), meth))) =
     (case get_preplay_time l of
-      (* don't touch steps that time out or fail; minimizing won't help (not true -- FIXME) *)
-      (true, _) => step
+      (true, _) => step (* don't touch steps that time out or fail *)
     | (false, time) =>
       let
         fun mk_step_lfs_gfs lfs gfs = Prove (qs, xs, l, t, subproofs, ((lfs, gfs), meth))
@@ -69,12 +68,12 @@
       (case label_of_step step of
         NONE => (refed, step :: accu)
       | SOME l =>
-          if Ord_List.member label_ord refed l then
-            do_refed_step step
-            |>> Ord_List.union label_ord refed
-            ||> (fn x => x :: accu)
-          else
-            (refed, accu))
+        if Ord_List.member label_ord refed l then
+          do_refed_step step
+          |>> Ord_List.union label_ord refed
+          ||> (fn x => x :: accu)
+        else
+          (refed, accu))
     and do_refed_step step = step |> postproc_step |> do_refed_step'
     and do_refed_step' (Let _) = raise Fail "Sledgehammer_Minimize_Isar"
       | do_refed_step' (Prove (qs, xs, l, t, subproofs, ((lfs, gfs), m))) =