merged
authorblanchet
Wed, 23 Feb 2011 11:18:10 +0100
changeset 41825 49d5af6a3d1b
parent 41823 81d64ec48427 (current diff)
parent 41824 1b447261865e (diff)
child 41826 18d4d2b60016
merged
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML	Wed Feb 23 11:16:56 2011 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_minimize.ML	Wed Feb 23 11:18:10 2011 +0100
@@ -178,12 +178,6 @@
        (NONE, "Timeout: You can increase the time limit using the \"timeout\" \
               \option (e.g., \"timeout = " ^
               string_of_int (10 + msecs div 1000) ^ "\").")
-     | {outcome = SOME (UnknownError _), ...} =>
-       (* Failure sometimes mean timeout, unfortunately. *)
-       (NONE, "Failure: No proof was found with the current time limit. You \
-              \can increase the time limit using the \"timeout\" \
-              \option (e.g., \"timeout = " ^
-              string_of_int (10 + msecs div 1000) ^ "\").")
      | {message, ...} => (NONE, "Prover error: " ^ message))
     handle ERROR msg => (NONE, "Error: " ^ msg)
   end