weaken the "expect" flag so that it doesn't trigger errors if a prover is not installed
authorblanchet
Wed, 15 Dec 2010 11:26:28 +0100
changeset 41142 43e2b051339c
parent 41141 ad923cdd4a5d
child 41143 0b05cc14c2cb
weaken the "expect" flag so that it doesn't trigger errors if a prover is not installed
src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_run.ML	Wed Dec 15 11:26:28 2010 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_run.ML	Wed Dec 15 11:26:28 2010 +0100
@@ -86,7 +86,11 @@
                       ("unknown", "Internal error:\n" ^
                                   ML_Compiler.exn_message exn ^ "\n"))
         val _ =
-          if expect = "" orelse outcome_code = expect then
+          (* The "expect" argument is deliberately ignored if the prover is
+             missing so that the "Metis_Examples" can be processed on any
+             machine. *)
+          if expect = "" orelse outcome_code = expect orelse
+             not (is_prover_installed ctxt name) then
             ()
           else if blocking then
             error ("Unexpected outcome: " ^ quote outcome_code ^ ".")