imported patch sledge_doc_metis_as_prover
authorblanchet
Mon, 30 May 2011 17:00:38 +0200
changeset 43053 da6f459a7021
parent 43052 8d6a4978cc65
child 43054 f1864c0bd165
imported patch sledge_doc_metis_as_prover
doc-src/Sledgehammer/sledgehammer.tex
--- a/doc-src/Sledgehammer/sledgehammer.tex	Mon May 30 17:00:38 2011 +0200
+++ b/doc-src/Sledgehammer/sledgehammer.tex	Mon May 30 17:00:38 2011 +0200
@@ -750,6 +750,11 @@
 \item[$\bullet$] \textbf{\textit{z3\_atp}:} This version of Z3 pretends to be an
 ATP, exploiting Z3's undocumented support for the TPTP format. It is included
 for experimental purposes. It requires version 2.18 or above.
+
+\item[$\bullet$] \textbf{\textit{metis}:} Although it is much less powerful than
+the external provers, Metis itself can be used for proof search.
+
+\item[$\bullet$] \textbf{\textit{metisFT}:} Fully typed version of Metis.
 \end{enum}
 
 In addition, the following remote provers are supported:
@@ -814,6 +819,9 @@
 success rate to running the most effective of these for 120~seconds
 \cite{boehme-nipkow-2010}.
 
+For the \textit{min} subcommand, the default prover is \textit{metis}. If
+several provers are set, the first one is used.
+
 \opnodefault{prover}{string}
 Alias for \textit{provers}.