src/HOL/Tools/ATP/atp_proof.ML
changeset 45301 866b075aa99b
parent 45235 7187bce94e88
child 45551 a62c7a21f4ab
--- a/src/HOL/Tools/ATP/atp_proof.ML	Sat Oct 29 13:15:58 2011 +0200
+++ b/src/HOL/Tools/ATP/atp_proof.ML	Sat Oct 29 13:15:58 2011 +0200
@@ -24,8 +24,6 @@
     TimedOut |
     Inappropriate |
     OutOfResources |
-    SpassTooOld |
-    VampireTooOld |
     NoPerl |
     NoLibwwwPerl |
     MalformedInput |
@@ -81,8 +79,6 @@
   TimedOut |
   Inappropriate |
   OutOfResources |
-  SpassTooOld |
-  VampireTooOld |
   NoPerl |
   NoLibwwwPerl |
   MalformedInput |
@@ -134,17 +130,6 @@
   | string_for_failure Inappropriate =
     "The problem lies outside the prover's scope."
   | string_for_failure OutOfResources = "The prover ran out of resources."
-  | string_for_failure SpassTooOld =
-    "Isabelle requires a more recent version of SPASS with support for the \
-    \TPTP syntax. To install it, download and extract the package \
-    \\"http://isabelle.in.tum.de/dist/contrib/spass-3.7.tar.gz\" and add the \
-    \\"spass-3.7\" directory's absolute path to " ^
-    Path.print (Path.expand (Path.explode "$ISABELLE_HOME_USER/etc/components")) ^
-    " on a line of its own."
-  | string_for_failure VampireTooOld =
-    "Isabelle requires a more recent version of Vampire. To install it, follow \
-    \the instructions from the Sledgehammer manual (\"isabelle doc\
-    \ sledgehammer\")."
   | string_for_failure NoPerl = "Perl" ^ missing_message_tail
   | string_for_failure NoLibwwwPerl =
     "The Perl module \"libwww-perl\"" ^ missing_message_tail