doc-src/Sledgehammer/sledgehammer.tex
changeset 45048 59ca831deef4
parent 44816 efa1f532508b
child 45063 b3b50d8b535a
equal deleted inserted replaced
45047:3aa8d3c391a4 45048:59ca831deef4
   174 \item[$\bullet$] If you prefer to build E or SPASS yourself, or obtained a
   174 \item[$\bullet$] If you prefer to build E or SPASS yourself, or obtained a
   175 Vampire executable from somewhere (e.g., \url{http://www.vprover.org/}),
   175 Vampire executable from somewhere (e.g., \url{http://www.vprover.org/}),
   176 set the environment variable \texttt{E\_HOME}, \texttt{SPASS\_HOME}, or
   176 set the environment variable \texttt{E\_HOME}, \texttt{SPASS\_HOME}, or
   177 \texttt{VAMPIRE\_HOME} to the directory that contains the \texttt{eproof},
   177 \texttt{VAMPIRE\_HOME} to the directory that contains the \texttt{eproof},
   178 \texttt{SPASS}, or \texttt{vampire} executable. Sledgehammer has been tested
   178 \texttt{SPASS}, or \texttt{vampire} executable. Sledgehammer has been tested
   179 with E 1.0 to 1.3, SPASS 3.5 and 3.7, and Vampire 0.6, 1.0, and 1.8%
   179 with E 1.0 to 1.4, SPASS 3.5 and 3.7, and Vampire 0.6, 1.0, and 1.8%
   180 \footnote{Following the rewrite of Vampire, the counter for version numbers was
   180 \footnote{Following the rewrite of Vampire, the counter for version numbers was
   181 reset to 0; hence the (new) Vampire versions 0.6, 1.0, and 1.8 are more recent
   181 reset to 0; hence the (new) Vampire versions 0.6, 1.0, and 1.8 are more recent
   182 than, say, Vampire 9.0 or 11.5.}%
   182 than, say, Vampire 9.0 or 11.5.}%
   183 . Since the ATPs' output formats are neither documented nor stable, other
   183 . Since the ATPs' output formats are neither documented nor stable, other
   184 versions of the ATPs might or might not work well with Sledgehammer. Ideally,
   184 versions of the ATPs might or might not work well with Sledgehammer. Ideally,
   263 %
   263 %
   264 Sledgehammer: ``\textit{remote\_waldmeister}'' on goal \\
   264 Sledgehammer: ``\textit{remote\_waldmeister}'' on goal \\
   265 $[a] = [b] \,\Longrightarrow\, a = b$ \\
   265 $[a] = [b] \,\Longrightarrow\, a = b$ \\
   266 Try this: \textbf{by} (\textit{metis hd.simps}) (15 ms). \\[3\smallskipamount]
   266 Try this: \textbf{by} (\textit{metis hd.simps}) (15 ms). \\[3\smallskipamount]
   267 %
   267 %
   268 Sledgehammer: ``\textit{remote\_e\_sine}'' on goal \\
       
   269 $[a] = [b] \,\Longrightarrow\, a = b$ \\
       
   270 Try this: \textbf{by} (\textit{metis hd.simps}) (18 ms). \\[3\smallskipamount]
       
   271 %
       
   272 Sledgehammer: ``\textit{remote\_z3}'' on goal \\
   268 Sledgehammer: ``\textit{remote\_z3}'' on goal \\
   273 $[a] = [b] \,\Longrightarrow\, a = b$ \\
   269 $[a] = [b] \,\Longrightarrow\, a = b$ \\
   274 Try this: \textbf{by} (\textit{metis list.inject}) (20 ms).
   270 Try this: \textbf{by} (\textit{metis list.inject}) (20 ms).
   275 \postw
   271 \postw
   276 
   272 
   277 Sledgehammer ran E, E-SInE, SPASS, Vampire, Waldmeister, and Z3 in parallel.
   273 Sledgehammer ran E, SPASS, Vampire, Waldmeister, and Z3 in parallel.
   278 Depending on which provers are installed and how many processor cores are
   274 Depending on which provers are installed and how many processor cores are
   279 available, some of the provers might be missing or present with a
   275 available, some of the provers might be missing or present with a
   280 \textit{remote\_} prefix. Waldmeister is run only for unit equational problems,
   276 \textit{remote\_} prefix. Waldmeister is run only for unit equational problems,
   281 where the goal's conclusion is a (universally quantified) equation.
   277 where the goal's conclusion is a (universally quantified) equation.
   282 
   278 
   503 \prew
   499 \prew
   504 \slshape
   500 \slshape
   505 Metis: Falling back on ``\textit{metis} (\textit{full\_types})''.
   501 Metis: Falling back on ``\textit{metis} (\textit{full\_types})''.
   506 \postw
   502 \postw
   507 
   503 
   508 in a successful Metis proof, you can advantageously pass the
   504 for a successful Metis proof, you can advantageously pass the
   509 \textit{full\_types} option to \textit{metis} directly.
   505 \textit{full\_types} option to \textit{metis} directly.
   510 
   506 
   511 \point{Are generated proofs minimal?}
   507 \point{Are generated proofs minimal?}
   512 
   508 
   513 Automatic provers frequently use many more facts than are necessary.
   509 Automatic provers frequently use many more facts than are necessary.
   816 
   812 
   817 \item[$\bullet$] \textbf{\textit{remote\_z3\_tptp}:} The remote version of ``Z3
   813 \item[$\bullet$] \textbf{\textit{remote\_z3\_tptp}:} The remote version of ``Z3
   818 with TPTP syntax'' runs on Geoff Sutcliffe's Miami servers.
   814 with TPTP syntax'' runs on Geoff Sutcliffe's Miami servers.
   819 \end{enum}
   815 \end{enum}
   820 
   816 
   821 By default, Sledgehammer runs E, E-SInE, SPASS, Vampire, Z3 (or whatever
   817 By default, Sledgehammer runs E, SPASS, Vampire, Z3 (or whatever
   822 the SMT module's \textit{smt\_solver} configuration option is set to), and (if
   818 the SMT module's \textit{smt\_solver} configuration option is set to), and (if
   823 appropriate) Waldmeister in parallel---either locally or remotely, depending on
   819 appropriate) Waldmeister in parallel---either locally or remotely, depending on
   824 the number of processor cores available. For historical reasons, the default
   820 the number of processor cores available. For historical reasons, the default
   825 value of this option can be overridden using the option ``Sledgehammer:
   821 value of this option can be overridden using the option ``Sledgehammer:
   826 Provers'' in Proof General's ``Isabelle'' menu.
   822 Provers'' in Proof General's ``Isabelle'' menu.