author | blanchet |
Thu, 10 Feb 2011 16:38:12 +0100 | |
changeset 41747 | f58d4d202924 |
parent 41740 | 4b09f8b9e012 |
child 42180 | a6c141925a8a |
permissions | -rw-r--r-- |
36926 | 1 |
\documentclass[a4paper,12pt]{article} |
2 |
\usepackage[T1]{fontenc} |
|
3 |
\usepackage{amsmath} |
|
4 |
\usepackage{amssymb} |
|
5 |
\usepackage[english,french]{babel} |
|
6 |
\usepackage{color} |
|
7 |
\usepackage{footmisc} |
|
8 |
\usepackage{graphicx} |
|
9 |
%\usepackage{mathpazo} |
|
10 |
\usepackage{multicol} |
|
11 |
\usepackage{stmaryrd} |
|
12 |
%\usepackage[scaled=.85]{beramono} |
|
40689 | 13 |
\usepackage{../isabelle,../iman,../pdfsetup} |
36926 | 14 |
|
15 |
%\oddsidemargin=4.6mm |
|
16 |
%\evensidemargin=4.6mm |
|
17 |
%\textwidth=150mm |
|
18 |
%\topmargin=4.6mm |
|
19 |
%\headheight=0mm |
|
20 |
%\headsep=0mm |
|
21 |
%\textheight=234mm |
|
22 |
||
23 |
\def\Colon{\mathord{:\mkern-1.5mu:}} |
|
24 |
%\def\lbrakk{\mathopen{\lbrack\mkern-3.25mu\lbrack}} |
|
25 |
%\def\rbrakk{\mathclose{\rbrack\mkern-3.255mu\rbrack}} |
|
26 |
\def\lparr{\mathopen{(\mkern-4mu\mid}} |
|
27 |
\def\rparr{\mathclose{\mid\mkern-4mu)}} |
|
28 |
||
29 |
\def\unk{{?}} |
|
30 |
\def\undef{(\lambda x.\; \unk)} |
|
31 |
%\def\unr{\textit{others}} |
|
32 |
\def\unr{\ldots} |
|
33 |
\def\Abs#1{\hbox{\rm{\flqq}}{\,#1\,}\hbox{\rm{\frqq}}} |
|
34 |
\def\Q{{\smash{\lower.2ex\hbox{$\scriptstyle?$}}}} |
|
35 |
||
36 |
\urlstyle{tt} |
|
37 |
||
38 |
\begin{document} |
|
39 |
||
40 |
\selectlanguage{english} |
|
41 |
||
42 |
\title{\includegraphics[scale=0.5]{isabelle_sledgehammer} \\[4ex] |
|
43 |
Hammering Away \\[\smallskipamount] |
|
44 |
\Large A User's Guide to Sledgehammer for Isabelle/HOL} |
|
45 |
\author{\hbox{} \\ |
|
46 |
Jasmin Christian Blanchette \\ |
|
47 |
{\normalsize Institut f\"ur Informatik, Technische Universit\"at M\"unchen} \\ |
|
48 |
\hbox{}} |
|
49 |
||
50 |
\maketitle |
|
51 |
||
52 |
\tableofcontents |
|
53 |
||
54 |
\setlength{\parskip}{.7em plus .2em minus .1em} |
|
55 |
\setlength{\parindent}{0pt} |
|
56 |
\setlength{\abovedisplayskip}{\parskip} |
|
57 |
\setlength{\abovedisplayshortskip}{.9\parskip} |
|
58 |
\setlength{\belowdisplayskip}{\parskip} |
|
59 |
\setlength{\belowdisplayshortskip}{.9\parskip} |
|
60 |
||
61 |
% General-purpose enum environment with correct spacing |
|
62 |
\newenvironment{enum}% |
|
63 |
{\begin{list}{}{% |
|
64 |
\setlength{\topsep}{.1\parskip}% |
|
65 |
\setlength{\partopsep}{.1\parskip}% |
|
66 |
\setlength{\itemsep}{\parskip}% |
|
67 |
\advance\itemsep by-\parsep}} |
|
68 |
{\end{list}} |
|
69 |
||
70 |
\def\pre{\begingroup\vskip0pt plus1ex\advance\leftskip by\leftmargin |
|
71 |
\advance\rightskip by\leftmargin} |
|
72 |
\def\post{\vskip0pt plus1ex\endgroup} |
|
73 |
||
74 |
\def\prew{\pre\advance\rightskip by-\leftmargin} |
|
75 |
\def\postw{\post} |
|
76 |
||
77 |
\section{Introduction} |
|
78 |
\label{introduction} |
|
79 |
||
80 |
Sledgehammer is a tool that applies first-order automatic theorem provers (ATPs) |
|
40942 | 81 |
and satisfiability-modulo-theories (SMT) solvers on the current goal. The |
40073 | 82 |
supported ATPs are E \cite{schulz-2002}, SPASS \cite{weidenbach-et-al-2009}, |
83 |
Vampire \cite{riazanov-voronkov-2002}, SInE-E \cite{sine}, and SNARK |
|
84 |
\cite{snark}. The ATPs are run either locally or remotely via the |
|
85 |
System\-On\-TPTP web service \cite{sutcliffe-2000}. In addition to the ATPs, the |
|
40942 | 86 |
SMT solvers Z3 \cite{z3} is used, and you can tell Sledgehammer to try Yices |
87 |
\cite{yices} and CVC3 \cite{cvc3} as well. |
|
36926 | 88 |
|
40073 | 89 |
The problem passed to the automatic provers consists of your current goal |
90 |
together with a heuristic selection of hundreds of facts (theorems) from the |
|
91 |
current theory context, filtered by relevance. Because jobs are run in the |
|
92 |
background, you can continue to work on your proof by other means. Provers can |
|
93 |
be run in parallel. Any reply (which may arrive half a minute later) will appear |
|
94 |
in the Proof General response buffer. |
|
37517
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
95 |
|
40073 | 96 |
The result of a successful proof search is some source text that usually (but |
97 |
not always) reconstructs the proof within Isabelle. For ATPs, the reconstructed |
|
98 |
proof relies on the general-purpose Metis prover \cite{metis}, which is fully |
|
99 |
integrated into Isabelle/HOL, with explicit inferences going through the kernel. |
|
100 |
Thus its results are correct by construction. |
|
36926 | 101 |
|
39320 | 102 |
In this manual, we will explicitly invoke the \textbf{sledgehammer} command. |
103 |
Sledgehammer also provides an automatic mode that can be enabled via the |
|
104 |
``Auto Sledgehammer'' option from the ``Isabelle'' menu in Proof General. In |
|
105 |
this mode, Sledgehammer is run on every newly entered theorem. The time limit |
|
106 |
for Auto Sledgehammer and other automatic tools can be set using the ``Auto |
|
107 |
Tools Time Limit'' option. |
|
108 |
||
36926 | 109 |
\newbox\boxA |
110 |
\setbox\boxA=\hbox{\texttt{nospam}} |
|
111 |
||
40689 | 112 |
To run Sledgehammer, you must make sure that the theory \textit{Sledgehammer} is |
113 |
imported---this is rarely a problem in practice since it is part of |
|
114 |
\textit{Main}. Examples of Sledgehammer use can be found in Isabelle's |
|
36926 | 115 |
\texttt{src/HOL/Metis\_Examples} directory. |
116 |
Comments and bug reports concerning Sledgehammer or this manual should be |
|
117 |
directed to |
|
118 |
\texttt{blan{\color{white}nospam}\kern-\wd\boxA{}chette@\allowbreak |
|
119 |
in.\allowbreak tum.\allowbreak de}. |
|
120 |
||
121 |
\vskip2.5\smallskipamount |
|
122 |
||
123 |
%\textbf{Acknowledgment.} The author would like to thank Mark Summerfield for |
|
124 |
%suggesting several textual improvements. |
|
125 |
||
126 |
\section{Installation} |
|
127 |
\label{installation} |
|
128 |
||
129 |
Sledgehammer is part of Isabelle, so you don't need to install it. However, it |
|
40073 | 130 |
relies on third-party automatic theorem provers (ATPs) and SAT solvers. |
131 |
Currently, E, SPASS, and Vampire can be run locally; in addition, E, Vampire, |
|
132 |
SInE-E, and SNARK are available remotely via SystemOnTPTP \cite{sutcliffe-2000}. |
|
133 |
If you want better performance, you should install E and SPASS locally. |
|
36926 | 134 |
|
38043 | 135 |
There are three main ways to install ATPs on your machine: |
36926 | 136 |
|
137 |
\begin{enum} |
|
138 |
\item[$\bullet$] If you installed an official Isabelle package with everything |
|
139 |
inside, it should already include properly setup executables for E and SPASS, |
|
38043 | 140 |
ready to use.% |
141 |
\footnote{Vampire's license prevents us from doing the same for this otherwise |
|
142 |
wonderful tool.} |
|
36926 | 143 |
|
38043 | 144 |
\item[$\bullet$] Alternatively, you can download the Isabelle-aware E and SPASS |
36926 | 145 |
binary packages from Isabelle's download page. Extract the archives, then add a |
41747
f58d4d202924
fix path to etc/settings and etc/components in doc
blanchet
parents:
41740
diff
changeset
|
146 |
line to your \texttt{\$ISABELLE\_HOME\_USER/etc/components}% |
f58d4d202924
fix path to etc/settings and etc/components in doc
blanchet
parents:
41740
diff
changeset
|
147 |
\footnote{The variable \texttt{\$ISABELLE\_HOME\_USER} is set by Isabelle at |
f58d4d202924
fix path to etc/settings and etc/components in doc
blanchet
parents:
41740
diff
changeset
|
148 |
startup. Its value can be retrieved by invoking \texttt{isabelle} |
f58d4d202924
fix path to etc/settings and etc/components in doc
blanchet
parents:
41740
diff
changeset
|
149 |
\texttt{getenv} \texttt{ISABELLE\_HOME\_USER} on the command line.} |
f58d4d202924
fix path to etc/settings and etc/components in doc
blanchet
parents:
41740
diff
changeset
|
150 |
file with the absolute |
40203 | 151 |
path to E or SPASS. For example, if the \texttt{components} does not exist yet |
152 |
and you extracted SPASS to \texttt{/usr/local/spass-3.7}, create the |
|
153 |
\texttt{components} file with the single line |
|
36926 | 154 |
|
155 |
\prew |
|
156 |
\texttt{/usr/local/spass-3.7} |
|
157 |
\postw |
|
158 |
||
38043 | 159 |
in it. |
160 |
||
161 |
\item[$\bullet$] If you prefer to build E or SPASS yourself, or obtained a |
|
162 |
Vampire executable from somewhere (e.g., \url{http://www.vprover.org/}), |
|
163 |
set the environment variable \texttt{E\_HOME}, \texttt{SPASS\_HOME}, or |
|
164 |
\texttt{VAMPIRE\_HOME} to the directory that contains the \texttt{eproof}, |
|
38063 | 165 |
\texttt{SPASS}, or \texttt{vampire} executable. Sledgehammer has been tested |
166 |
with E 1.0 and 1.2, SPASS 3.5 and 3.7, and Vampire 1.0% |
|
167 |
\footnote{Following the rewrite of Vampire, the counter for version numbers was |
|
168 |
reset to 0; hence the new Vampire 1.0 is more recent than Vampire 11.5.}% |
|
169 |
. Since the ATPs' output formats are neither documented nor stable, other |
|
170 |
versions of the ATPs might or might not work well with Sledgehammer. |
|
36926 | 171 |
\end{enum} |
172 |
||
173 |
To check whether E and SPASS are installed, follow the example in |
|
174 |
\S\ref{first-steps}. |
|
175 |
||
37517
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
176 |
Remote ATP invocation via the SystemOnTPTP web service requires Perl with the |
39152
f09b378cb252
make remote ATP invocation work for those people who need to go through a proxy;
blanchet
parents:
38997
diff
changeset
|
177 |
World Wide Web Library (\texttt{libwww-perl}) installed. If you must use a proxy |
f09b378cb252
make remote ATP invocation work for those people who need to go through a proxy;
blanchet
parents:
38997
diff
changeset
|
178 |
server to access the Internet, set the \texttt{http\_proxy} environment variable |
39153 | 179 |
to the proxy, either in the environment in which Isabelle is launched or in your |
41747
f58d4d202924
fix path to etc/settings and etc/components in doc
blanchet
parents:
41740
diff
changeset
|
180 |
\texttt{\char`\~/\$ISABELLE\_HOME\_USER/etc/settings} file. Here are a few examples: |
39152
f09b378cb252
make remote ATP invocation work for those people who need to go through a proxy;
blanchet
parents:
38997
diff
changeset
|
181 |
|
f09b378cb252
make remote ATP invocation work for those people who need to go through a proxy;
blanchet
parents:
38997
diff
changeset
|
182 |
\prew |
39153 | 183 |
\texttt{http\_proxy=http://proxy.example.org} \\ |
184 |
\texttt{http\_proxy=http://proxy.example.org:8080} \\ |
|
185 |
\texttt{http\_proxy=http://joeblow:pAsSwRd@proxy.example.org} |
|
39152
f09b378cb252
make remote ATP invocation work for those people who need to go through a proxy;
blanchet
parents:
38997
diff
changeset
|
186 |
\postw |
37517
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
187 |
|
36926 | 188 |
\section{First Steps} |
189 |
\label{first-steps} |
|
190 |
||
191 |
To illustrate Sledgehammer in context, let us start a theory file and |
|
192 |
attempt to prove a simple lemma: |
|
193 |
||
194 |
\prew |
|
195 |
\textbf{theory}~\textit{Scratch} \\ |
|
196 |
\textbf{imports}~\textit{Main} \\ |
|
197 |
\textbf{begin} \\[2\smallskipamount] |
|
198 |
% |
|
199 |
\textbf{lemma} ``$[a] = [b] \,\longleftrightarrow\, a = b$'' \\ |
|
200 |
\textbf{sledgehammer} |
|
201 |
\postw |
|
202 |
||
37517
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
203 |
Instead of issuing the \textbf{sledgehammer} command, you can also find |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
204 |
Sledgehammer in the ``Commands'' submenu of the ``Isabelle'' menu in Proof |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
205 |
General or press the Emacs key sequence C-c C-a C-s. |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
206 |
Either way, Sledgehammer produces the following output after a few seconds: |
36926 | 207 |
|
208 |
\prew |
|
209 |
\slshape |
|
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
210 |
Sledgehammer: ``\textit{e}'' for subgoal 1: \\ |
36926 | 211 |
$([a] = [b]) = (a = b)$ \\ |
212 |
Try this command: \textbf{by} (\textit{metis hd.simps}). \\ |
|
38043 | 213 |
To minimize the number of lemmas, try this: \\ |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
214 |
\textbf{sledgehammer} \textit{minimize} [\textit{prover} = \textit{e}] (\textit{hd.simps}). \\[3\smallskipamount] |
36926 | 215 |
% |
40060
5ef6747aa619
first step in adding support for an SMT backend to Sledgehammer
blanchet
parents:
40059
diff
changeset
|
216 |
Sledgehammer: ``\textit{spass}'' for subgoal 1: \\ |
36926 | 217 |
$([a] = [b]) = (a = b)$ \\ |
218 |
Try this command: \textbf{by} (\textit{metis insert\_Nil last\_ConsL}). \\ |
|
38043 | 219 |
To minimize the number of lemmas, try this: \\ |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
220 |
\textbf{sledgehammer} \textit{minimize} [\textit{prover} = \textit{spass}] (\textit{insert\_Nil last\_ConsL}). \\[3\smallskipamount] |
36926 | 221 |
% |
40073 | 222 |
Sledgehammer: ``\textit{vampire}'' for subgoal 1: \\ |
36926 | 223 |
$([a] = [b]) = (a = b)$ \\ |
40073 | 224 |
Try this command: \textbf{by} (\textit{metis eq\_commute last\_snoc}) \\ |
38043 | 225 |
To minimize the number of lemmas, try this: \\ |
40073 | 226 |
\textbf{sledgehammer} \textit{minimize} [\textit{prover} = \textit{vampire}]~(\textit{eq\_commute last\_snoc}). \\[3\smallskipamount] |
227 |
% |
|
228 |
Sledgehammer: ``\textit{remote\_sine\_e}'' for subgoal 1: \\ |
|
229 |
$([a] = [b]) = (a = b)$ \\ |
|
230 |
Try this command: \textbf{by} (\textit{metis hd.simps}) \\ |
|
231 |
To minimize the number of lemmas, try this: \\ |
|
40203 | 232 |
\textbf{sledgehammer} \textit{minimize} [\textit{prover} = \textit{remote\_sine\_e}]~(\textit{hd.simps}). |
40942 | 233 |
% |
234 |
Sledgehammer: ``\textit{remote\_z3}'' for subgoal 1: \\ |
|
235 |
$([a] = [b]) = (a = b)$ \\ |
|
236 |
Try this command: \textbf{by} (\textit{metis hd.simps}) \\ |
|
237 |
To minimize the number of lemmas, try this: \\ |
|
238 |
\textbf{sledgehammer} \textit{minimize} [\textit{prover} = \textit{remote\_sine\_e}]~(\textit{hd.simps}). |
|
36926 | 239 |
\postw |
240 |
||
40942 | 241 |
Sledgehammer ran E, SPASS, Vampire, SInE-E, and Z3 in parallel. Depending on |
242 |
which provers are installed and how many processor cores are available, some of |
|
243 |
the provers might be missing or present with a \textit{remote\_} prefix. |
|
36926 | 244 |
|
40073 | 245 |
For each successful prover, Sledgehammer gives a one-liner proof that uses the |
246 |
\textit{metis} or \textit{smt} method. You can click the proof to insert it into |
|
247 |
the theory text. You can click the ``\textbf{sledgehammer} \textit{minimize}'' |
|
248 |
command if you want to look for a shorter (and probably faster) proof. But here |
|
249 |
the proof found by E looks perfect, so click it to finish the proof. |
|
36926 | 250 |
|
251 |
You can ask Sledgehammer for an Isar text proof by passing the |
|
252 |
\textit{isar\_proof} option: |
|
253 |
||
254 |
\prew |
|
255 |
\textbf{sledgehammer} [\textit{isar\_proof}] |
|
256 |
\postw |
|
257 |
||
258 |
When Isar proof construction is successful, it can yield proofs that are more |
|
259 |
readable and also faster than the \textit{metis} one-liners. This feature is |
|
40073 | 260 |
experimental and is only available for ATPs. |
36926 | 261 |
|
37517
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
262 |
\section{Hints} |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
263 |
\label{hints} |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
264 |
|
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
265 |
For best results, first simplify your problem by calling \textit{auto} or at |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
266 |
least \textit{safe} followed by \textit{simp\_all}. None of the ATPs contain |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
267 |
arithmetic decision procedures. They are not especially good at heavy rewriting, |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
268 |
but because they regard equations as undirected, they often prove theorems that |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
269 |
require the reverse orientation of a \textit{simp} rule. Higher-order problems |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
270 |
can be tackled, but the success rate is better for first-order problems. Hence, |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
271 |
you may get better results if you first simplify the problem to remove |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
272 |
higher-order features. |
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
273 |
|
39320 | 274 |
Note that problems can be easy for \textit{auto} and difficult for ATPs, but the |
275 |
reverse is also true, so don't be discouraged if your first attempts fail. |
|
276 |
Because the system refers to all theorems known to Isabelle, it is particularly |
|
277 |
suitable when your goal has a short proof from lemmas that you don't know about. |
|
37517
19ba7ec5f1e3
steal some of http://isabelle.in.tum.de/sledgehammer.html and add it to the docs
blanchet
parents:
37498
diff
changeset
|
278 |
|
36926 | 279 |
\section{Command Syntax} |
280 |
\label{command-syntax} |
|
281 |
||
282 |
Sledgehammer can be invoked at any point when there is an open goal by entering |
|
283 |
the \textbf{sledgehammer} command in the theory file. Its general syntax is as |
|
284 |
follows: |
|
285 |
||
286 |
\prew |
|
287 |
\textbf{sledgehammer} \textit{subcommand\/$^?$ options\/$^?$ facts\_override\/$^?$ num\/$^?$} |
|
288 |
\postw |
|
289 |
||
290 |
For convenience, Sledgehammer is also available in the ``Commands'' submenu of |
|
291 |
the ``Isabelle'' menu in Proof General or by pressing the Emacs key sequence C-c |
|
292 |
C-a C-s. This is equivalent to entering the \textbf{sledgehammer} command with |
|
293 |
no arguments in the theory text. |
|
294 |
||
295 |
In the general syntax, the \textit{subcommand} may be any of the following: |
|
296 |
||
297 |
\begin{enum} |
|
40203 | 298 |
\item[$\bullet$] \textbf{\textit{run} (the default):} Runs Sledgehammer on |
299 |
subgoal number \textit{num} (1 by default), with the given options and facts. |
|
36926 | 300 |
|
301 |
\item[$\bullet$] \textbf{\textit{minimize}:} Attempts to minimize the provided facts |
|
302 |
(specified in the \textit{facts\_override} argument) to obtain a simpler proof |
|
303 |
involving fewer facts. The options and goal number are as for \textit{run}. |
|
304 |
||
40203 | 305 |
\item[$\bullet$] \textbf{\textit{messages}:} Redisplays recent messages issued |
306 |
by Sledgehammer. This allows you to examine results that might have been lost |
|
307 |
due to Sledgehammer's asynchronous nature. The \textit{num} argument specifies a |
|
36926 | 308 |
limit on the number of messages to display (5 by default). |
309 |
||
41727
ab3f6d76fb23
available_provers ~> supported_provers (for clarity)
blanchet
parents:
41724
diff
changeset
|
310 |
\item[$\bullet$] \textbf{\textit{supported\_provers}:} Prints the list of |
41724 | 311 |
automatic provers supported by Sledgehammer. See \S\ref{installation} and |
312 |
\S\ref{mode-of-operation} for more information on how to install automatic |
|
313 |
provers. |
|
36926 | 314 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
315 |
\item[$\bullet$] \textbf{\textit{running\_provers}:} Prints information about |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
316 |
currently running automatic provers, including elapsed runtime and remaining |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
317 |
time until timeout. |
36926 | 318 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
319 |
\item[$\bullet$] \textbf{\textit{kill\_provers}:} Terminates all running |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
320 |
automatic provers. |
36926 | 321 |
|
322 |
\item[$\bullet$] \textbf{\textit{refresh\_tptp}:} Refreshes the list of remote |
|
323 |
ATPs available at System\-On\-TPTP \cite{sutcliffe-2000}. |
|
324 |
\end{enum} |
|
325 |
||
326 |
Sledgehammer's behavior can be influenced by various \textit{options}, which can |
|
327 |
be specified in brackets after the \textbf{sledgehammer} command. The |
|
328 |
\textit{options} are a list of key--value pairs of the form ``[$k_1 = v_1, |
|
329 |
\ldots, k_n = v_n$]''. For Boolean options, ``= \textit{true}'' is optional. For |
|
330 |
example: |
|
331 |
||
332 |
\prew |
|
333 |
\textbf{sledgehammer} [\textit{isar\_proof}, \,\textit{timeout} = 120$\,s$] |
|
334 |
\postw |
|
335 |
||
336 |
Default values can be set using \textbf{sledgehammer\_\allowbreak params}: |
|
337 |
||
338 |
\prew |
|
339 |
\textbf{sledgehammer\_params} \textit{options} |
|
340 |
\postw |
|
341 |
||
342 |
The supported options are described in \S\ref{option-reference}. |
|
343 |
||
344 |
The \textit{facts\_override} argument lets you alter the set of facts that go |
|
345 |
through the relevance filter. It may be of the form ``(\textit{facts})'', where |
|
346 |
\textit{facts} is a space-separated list of Isabelle facts (theorems, local |
|
347 |
assumptions, etc.), in which case the relevance filter is bypassed and the given |
|
39320 | 348 |
facts are used. It may also be of the form ``(\textit{add}:\ \textit{facts}$_1$)'', |
349 |
``(\textit{del}:\ \textit{facts}$_2$)'', or ``(\textit{add}:\ \textit{facts}$_1$\ |
|
350 |
\textit{del}:\ \textit{facts}$_2$)'', where the relevance filter is instructed to |
|
36926 | 351 |
proceed as usual except that it should consider \textit{facts}$_1$ |
352 |
highly-relevant and \textit{facts}$_2$ fully irrelevant. |
|
353 |
||
39320 | 354 |
You can instruct Sledgehammer to run automatically on newly entered theorems by |
355 |
enabling the ``Auto Sledgehammer'' option from the ``Isabelle'' menu in Proof |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
356 |
General. For automatic runs, only the first prover set using \textit{provers} |
39320 | 357 |
(\S\ref{mode-of-operation}) is considered, \textit{verbose} |
358 |
(\S\ref{output-format}) and \textit{debug} (\S\ref{output-format}) are disabled, |
|
40073 | 359 |
fewer facts are passed to the prover, and \textit{timeout} |
360 |
(\S\ref{mode-of-operation}) is superseded by the ``Auto Tools Time Limit'' in |
|
361 |
Proof General's ``Isabelle'' menu. Sledgehammer's output is also more concise. |
|
39320 | 362 |
|
36926 | 363 |
\section{Option Reference} |
364 |
\label{option-reference} |
|
365 |
||
366 |
\def\flushitem#1{\item[]\noindent\kern-\leftmargin \textbf{#1}} |
|
367 |
\def\qty#1{$\left<\textit{#1}\right>$} |
|
368 |
\def\qtybf#1{$\mathbf{\left<\textbf{\textit{#1}}\right>}$} |
|
369 |
\def\optrue#1#2{\flushitem{\textit{#1} $\bigl[$= \qtybf{bool}$\bigr]$\quad [\textit{true}]\hfill (neg.: \textit{#2})}\nopagebreak\\[\parskip]} |
|
370 |
\def\opfalse#1#2{\flushitem{\textit{#1} $\bigl[$= \qtybf{bool}$\bigr]$\quad [\textit{false}]\hfill (neg.: \textit{#2})}\nopagebreak\\[\parskip]} |
|
371 |
\def\opsmart#1#2{\flushitem{\textit{#1} $\bigl[$= \qtybf{bool\_or\_smart}$\bigr]$\quad [\textit{smart}]\hfill (neg.: \textit{#2})}\nopagebreak\\[\parskip]} |
|
372 |
\def\opsmartx#1#2{\flushitem{\textit{#1} $\bigl[$= \qtybf{bool\_or\_smart}$\bigr]$\quad [\textit{smart}]\hfill\\\hbox{}\hfill (neg.: \textit{#2})}\nopagebreak\\[\parskip]} |
|
373 |
\def\opnodefault#1#2{\flushitem{\textit{#1} = \qtybf{#2}} \nopagebreak\\[\parskip]} |
|
374 |
\def\opdefault#1#2#3{\flushitem{\textit{#1} = \qtybf{#2}\quad [\textit{#3}]} \nopagebreak\\[\parskip]} |
|
375 |
\def\oparg#1#2#3{\flushitem{\textit{#1} \qtybf{#2} = \qtybf{#3}} \nopagebreak\\[\parskip]} |
|
376 |
\def\opargbool#1#2#3{\flushitem{\textit{#1} \qtybf{#2} $\bigl[$= \qtybf{bool}$\bigr]$\hfill (neg.: \textit{#3})}\nopagebreak\\[\parskip]} |
|
377 |
\def\opargboolorsmart#1#2#3{\flushitem{\textit{#1} \qtybf{#2} $\bigl[$= \qtybf{bool\_or\_smart}$\bigr]$\hfill (neg.: \textit{#3})}\nopagebreak\\[\parskip]} |
|
378 |
||
379 |
Sledgehammer's options are categorized as follows:\ mode of operation |
|
38984 | 380 |
(\S\ref{mode-of-operation}), problem encoding (\S\ref{problem-encoding}), |
381 |
relevance filter (\S\ref{relevance-filter}), output format |
|
382 |
(\S\ref{output-format}), and authentication (\S\ref{authentication}). |
|
36926 | 383 |
|
384 |
The descriptions below refer to the following syntactic quantities: |
|
385 |
||
386 |
\begin{enum} |
|
387 |
\item[$\bullet$] \qtybf{string}: A string. |
|
388 |
\item[$\bullet$] \qtybf{bool\/}: \textit{true} or \textit{false}. |
|
40203 | 389 |
\item[$\bullet$] \qtybf{bool\_or\_smart\/}: \textit{true}, \textit{false}, or |
390 |
\textit{smart}. |
|
36926 | 391 |
\item[$\bullet$] \qtybf{int\/}: An integer. |
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
392 |
\item[$\bullet$] \qtybf{float\_pair\/}: A pair of floating-point numbers |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
393 |
(e.g., 0.6 0.95). |
38591 | 394 |
\item[$\bullet$] \qtybf{int\_or\_smart\/}: An integer or \textit{smart}. |
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
395 |
\item[$\bullet$] \qtybf{float\_or\_none\/}: An integer (e.g., 60) or |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
396 |
floating-point number (e.g., 0.5) expressing a number of seconds, or the keyword |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
397 |
\textit{none} ($\infty$ seconds). |
36926 | 398 |
\end{enum} |
399 |
||
400 |
Default values are indicated in square brackets. Boolean options have a negated |
|
38984 | 401 |
counterpart (e.g., \textit{blocking} vs.\ \textit{non\_blocking}). When setting |
36926 | 402 |
Boolean options, ``= \textit{true}'' may be omitted. |
403 |
||
404 |
\subsection{Mode of Operation} |
|
405 |
\label{mode-of-operation} |
|
406 |
||
407 |
\begin{enum} |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
408 |
\opnodefault{provers}{string} |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
409 |
Specifies the automatic provers to use as a space-separated list (e.g., |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
410 |
``\textit{e}~\textit{spass}''). The following provers are supported: |
36926 | 411 |
|
412 |
\begin{enum} |
|
413 |
\item[$\bullet$] \textbf{\textit{e}:} E is an ATP developed by Stephan Schulz |
|
414 |
\cite{schulz-2002}. To use E, set the environment variable |
|
415 |
\texttt{E\_HOME} to the directory that contains the \texttt{eproof} executable, |
|
416 |
or install the prebuilt E package from Isabelle's download page. See |
|
417 |
\S\ref{installation} for details. |
|
418 |
||
419 |
\item[$\bullet$] \textbf{\textit{spass}:} SPASS is an ATP developed by Christoph |
|
420 |
Weidenbach et al.\ \cite{weidenbach-et-al-2009}. To use SPASS, set the |
|
421 |
environment variable \texttt{SPASS\_HOME} to the directory that contains the |
|
422 |
\texttt{SPASS} executable, or install the prebuilt SPASS package from Isabelle's |
|
37414
d0cea0796295
expect SPASS 3.7, and give a friendly warning if an older version is used
blanchet
parents:
36926
diff
changeset
|
423 |
download page. Sledgehammer requires version 3.5 or above. See |
d0cea0796295
expect SPASS 3.7, and give a friendly warning if an older version is used
blanchet
parents:
36926
diff
changeset
|
424 |
\S\ref{installation} for details. |
36926 | 425 |
|
426 |
\item[$\bullet$] \textbf{\textit{vampire}:} Vampire is an ATP developed by |
|
427 |
Andrei Voronkov and his colleagues \cite{riazanov-voronkov-2002}. To use |
|
428 |
Vampire, set the environment variable \texttt{VAMPIRE\_HOME} to the directory |
|
40942 | 429 |
that contains the \texttt{vampire} executable. Sledgehammer has been tested with |
430 |
versions 11, 0.6, and 1.0. |
|
431 |
||
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
432 |
\item[$\bullet$] \textbf{\textit{cvc3}:} CVC3 is an SMT solver developed by |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
433 |
Clark Barrett, Cesare Tinelli, and their colleagues \cite{cvc3}. To use CVC3, |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
434 |
set the environment variable \texttt{CVC3\_SOLVER} to the complete path of the |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
435 |
executable, including the file name. Sledgehammer has been tested with version |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
436 |
2.2. |
36926 | 437 |
|
40942 | 438 |
\item[$\bullet$] \textbf{\textit{yices}:} Yices is an SMT solver developed at |
439 |
SRI \cite{yices}. To use Yices, set the environment variable |
|
440 |
\texttt{YICES\_SOLVER} to the complete path of the executable, including the |
|
441 |
file name. Sledgehammer has been tested with version 1.0. |
|
442 |
||
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
443 |
\item[$\bullet$] \textbf{\textit{z3}:} Z3 is an SMT solver developed at |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
444 |
Microsoft Research \cite{z3}. To use Z3, set the environment variable |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
445 |
\texttt{Z3\_SOLVER} to the complete path of the executable, including the file |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
446 |
name. Sledgehammer has been tested with versions 2.7 to 2.18. |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
447 |
|
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
448 |
\item[$\bullet$] \textbf{\textit{z3\_atp}:} This version of Z3 pretends to be an |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
449 |
ATP, exploiting Z3's undocumented support for the TPTP format. It is included |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
450 |
for experimental purposes. It requires versions 2.18 or above. |
40073 | 451 |
|
38601 | 452 |
\item[$\bullet$] \textbf{\textit{remote\_e}:} The remote version of E runs |
36926 | 453 |
on Geoff Sutcliffe's Miami servers \cite{sutcliffe-2000}. |
454 |
||
455 |
\item[$\bullet$] \textbf{\textit{remote\_vampire}:} The remote version of |
|
38601 | 456 |
Vampire runs on Geoff Sutcliffe's Miami servers. Version 9 is used. |
36926 | 457 |
|
38601 | 458 |
\item[$\bullet$] \textbf{\textit{remote\_sine\_e}:} SInE-E is a metaprover |
459 |
developed by Kry\v stof Hoder \cite{sine} based on E. The remote version of |
|
460 |
SInE runs on Geoff Sutcliffe's Miami servers. |
|
461 |
||
462 |
\item[$\bullet$] \textbf{\textit{remote\_snark}:} SNARK is a prover |
|
463 |
developed by Stickel et al.\ \cite{snark}. The remote version of |
|
464 |
SNARK runs on Geoff Sutcliffe's Miami servers. |
|
40073 | 465 |
|
41738
eb98c60a6cf0
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
blanchet
parents:
41727
diff
changeset
|
466 |
\item[$\bullet$] \textbf{\textit{remote\_cvc3}:} The remote version of CVC3 runs |
eb98c60a6cf0
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
blanchet
parents:
41727
diff
changeset
|
467 |
on servers at the TU M\"unchen (or wherever \texttt{REMOTE\_SMT\_URL} is set to |
eb98c60a6cf0
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
blanchet
parents:
41727
diff
changeset
|
468 |
point). |
eb98c60a6cf0
added experimental "remote_z3_atp", Sutcliffe's TPTP-syntax-aware wrapper for Z3 -- allows to do head-to-head comparison of Sledgehammer's ATP translation and of Sascha's SMT translation
blanchet
parents:
41727
diff
changeset
|
469 |
|
40942 | 470 |
\item[$\bullet$] \textbf{\textit{remote\_z3}:} The remote version of Z3 runs on |
471 |
servers at the TU M\"unchen (or wherever \texttt{REMOTE\_SMT\_URL} is set to |
|
472 |
point). |
|
40073 | 473 |
|
41740
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
474 |
\item[$\bullet$] \textbf{\textit{remote\_z3\_atp}:} The remote version of ``Z3 |
4b09f8b9e012
added "Z3 as an ATP" support to Sledgehammer locally
blanchet
parents:
41738
diff
changeset
|
475 |
as an ATP'' runs on Geoff Sutcliffe's Miami servers. |
36926 | 476 |
\end{enum} |
477 |
||
40942 | 478 |
By default, Sledgehammer will run E, SPASS, Vampire, SInE-E, and Z3 (or whatever |
479 |
the SMT module's \emph{smt\_solver} configuration option is set to) in |
|
40073 | 480 |
parallel---either locally or remotely, depending on the number of processor |
481 |
cores available. For historical reasons, the default value of this option can be |
|
482 |
overridden using the option ``Sledgehammer: Provers'' from the ``Isabelle'' menu |
|
483 |
in Proof General. |
|
36926 | 484 |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
485 |
It is a good idea to run several provers in parallel, although it could slow |
40073 | 486 |
down your machine. Running E, SPASS, Vampire, and SInE-E together for 5 seconds |
487 |
yields a better success rate than running the most effective of these (Vampire) |
|
488 |
for 120 seconds \cite{boehme-nipkow-2010}. |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
489 |
|
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
490 |
\opnodefault{prover}{string} |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
491 |
Alias for \textit{provers}. |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
492 |
|
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
493 |
\opnodefault{atps}{string} |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
494 |
Legacy alias for \textit{provers}. |
36926 | 495 |
|
496 |
\opnodefault{atp}{string} |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
497 |
Legacy alias for \textit{provers}. |
36926 | 498 |
|
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
499 |
\opdefault{timeout}{float\_or\_none}{\upshape 30} |
40341
03156257040f
standardize on seconds for Nitpick and Sledgehammer timeouts
blanchet
parents:
40203
diff
changeset
|
500 |
Specifies the maximum number of seconds that the automatic provers should spend |
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
501 |
searching for a proof. For historical reasons, the default value of this option |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
502 |
can be overridden using the option ``Sledgehammer: Time Limit'' from the |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
503 |
``Isabelle'' menu in Proof General. |
38984 | 504 |
|
38983 | 505 |
\opfalse{blocking}{non\_blocking} |
506 |
Specifies whether the \textbf{sledgehammer} command should operate |
|
507 |
synchronously. The asynchronous (non-blocking) mode lets the user start proving |
|
508 |
the putative theorem manually while Sledgehammer looks for a proof, but it can |
|
509 |
also be more confusing. |
|
510 |
||
36926 | 511 |
\opfalse{overlord}{no\_overlord} |
512 |
Specifies whether Sledgehammer should put its temporary files in |
|
513 |
\texttt{\$ISA\-BELLE\_\allowbreak HOME\_\allowbreak USER}, which is useful for |
|
514 |
debugging Sledgehammer but also unsafe if several instances of the tool are run |
|
515 |
simultaneously. The files are identified by the prefix \texttt{prob\_}; you may |
|
516 |
safely remove them after Sledgehammer has run. |
|
517 |
||
518 |
\nopagebreak |
|
519 |
{\small See also \textit{debug} (\S\ref{output-format}).} |
|
520 |
\end{enum} |
|
521 |
||
522 |
\subsection{Problem Encoding} |
|
523 |
\label{problem-encoding} |
|
524 |
||
525 |
\begin{enum} |
|
526 |
\opfalse{explicit\_apply}{implicit\_apply} |
|
527 |
Specifies whether function application should be encoded as an explicit |
|
40073 | 528 |
``apply'' operator in ATP problems. If the option is set to \textit{false}, each |
529 |
function will be directly applied to as many arguments as possible. Enabling |
|
530 |
this option can sometimes help discover higher-order proofs that otherwise would |
|
531 |
not be found. |
|
36926 | 532 |
|
533 |
\opfalse{full\_types}{partial\_types} |
|
40073 | 534 |
Specifies whether full-type information is encoded in ATP problems. Enabling |
535 |
this option can prevent the discovery of type-incorrect proofs, but it also |
|
536 |
tends to slow down the ATPs significantly. For historical reasons, the default |
|
537 |
value of this option can be overridden using the option ``Sledgehammer: Full |
|
538 |
Types'' from the ``Isabelle'' menu in Proof General. |
|
38591 | 539 |
\end{enum} |
36926 | 540 |
|
38591 | 541 |
\subsection{Relevance Filter} |
542 |
\label{relevance-filter} |
|
543 |
||
544 |
\begin{enum} |
|
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
545 |
\opdefault{relevance\_thresholds}{float\_pair}{\upshape 0.45~0.85} |
38746 | 546 |
Specifies the thresholds above which facts are considered relevant by the |
547 |
relevance filter. The first threshold is used for the first iteration of the |
|
548 |
relevance filter and the second threshold is used for the last iteration (if it |
|
549 |
is reached). The effective threshold is quadratically interpolated for the other |
|
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
550 |
iterations. Each threshold ranges from 0 to 1, where 0 means that all theorems |
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
551 |
are relevant and 1 only theorems that refer to previously seen constants. |
36926 | 552 |
|
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
553 |
\opsmart{max\_relevant}{int\_or\_smart} |
38746 | 554 |
Specifies the maximum number of facts that may be returned by the relevance |
555 |
filter. If the option is set to \textit{smart}, it is set to a value that was |
|
40059
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
556 |
empirically found to be appropriate for the prover. A typical value would be |
6ad9081665db
use consistent terminology in Sledgehammer: "prover = ATP or SMT solver or ..."
blanchet
parents:
39335
diff
changeset
|
557 |
300. |
36926 | 558 |
\end{enum} |
559 |
||
560 |
\subsection{Output Format} |
|
561 |
\label{output-format} |
|
562 |
||
563 |
\begin{enum} |
|
564 |
||
565 |
\opfalse{verbose}{quiet} |
|
566 |
Specifies whether the \textbf{sledgehammer} command should explain what it does. |
|
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
40942
diff
changeset
|
567 |
This option is implicitly disabled for automatic runs. |
36926 | 568 |
|
569 |
\opfalse{debug}{no\_debug} |
|
40203 | 570 |
Specifies whether Sledgehammer should display additional debugging information |
571 |
beyond what \textit{verbose} already displays. Enabling \textit{debug} also |
|
41208
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
40942
diff
changeset
|
572 |
enables \textit{verbose} and \textit{blocking} (\S\ref{mode-of-operation}) |
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
40942
diff
changeset
|
573 |
behind the scenes. The \textit{debug} option is implicitly disabled for |
1b28c43a7074
make "debug" imply "blocking", since in blocking mode the exceptions flow through and are more instructive
blanchet
parents:
40942
diff
changeset
|
574 |
automatic runs. |
36926 | 575 |
|
576 |
\nopagebreak |
|
577 |
{\small See also \textit{overlord} (\S\ref{mode-of-operation}).} |
|
578 |
||
579 |
\opfalse{isar\_proof}{no\_isar\_proof} |
|
580 |
Specifies whether Isar proofs should be output in addition to one-liner |
|
581 |
\textit{metis} proofs. Isar proof construction is still experimental and often |
|
582 |
fails; however, they are usually faster and sometimes more robust than |
|
583 |
\textit{metis} proofs. |
|
584 |
||
40343
4521d56aef63
use floating-point numbers for Sledgehammer's "thresholds" option rather than percentages;
blanchet
parents:
40341
diff
changeset
|
585 |
\opdefault{isar\_shrink\_factor}{int}{\upshape 1} |
36926 | 586 |
Specifies the granularity of the Isar proof. A value of $n$ indicates that each |
587 |
Isar proof step should correspond to a group of up to $n$ consecutive proof |
|
588 |
steps in the ATP proof. |
|
589 |
||
590 |
\end{enum} |
|
591 |
||
38984 | 592 |
\subsection{Authentication} |
593 |
\label{authentication} |
|
594 |
||
595 |
\begin{enum} |
|
596 |
\opnodefault{expect}{string} |
|
597 |
Specifies the expected outcome, which must be one of the following: |
|
36926 | 598 |
|
599 |
\begin{enum} |
|
40203 | 600 |
\item[$\bullet$] \textbf{\textit{some}:} Sledgehammer found a (potentially |
601 |
unsound) proof. |
|
38984 | 602 |
\item[$\bullet$] \textbf{\textit{none}:} Sledgehammer found no proof. |
40203 | 603 |
\item[$\bullet$] \textbf{\textit{unknown}:} Sledgehammer encountered some |
604 |
problem. |
|
38984 | 605 |
\end{enum} |
606 |
||
607 |
Sledgehammer emits an error (if \textit{blocking} is enabled) or a warning |
|
608 |
(otherwise) if the actual outcome differs from the expected outcome. This option |
|
609 |
is useful for regression testing. |
|
610 |
||
611 |
\nopagebreak |
|
612 |
{\small See also \textit{blocking} (\S\ref{mode-of-operation}).} |
|
36926 | 613 |
\end{enum} |
614 |
||
615 |
\let\em=\sl |
|
616 |
\bibliography{../manual}{} |
|
617 |
\bibliographystyle{abbrv} |
|
618 |
||
619 |
\end{document} |