src/HOL/TPTP/CASC/SysDesc_Isabelle.html
author blanchet
Thu, 15 Dec 2016 15:05:35 +0100
changeset 64561 a7664ca9ffc5
parent 60719 b6713e04889e
permissions -rw-r--r--
updated CASC instructions + tuning
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     1
<HR><!------------------------------------------------------------------------>
64561
a7664ca9ffc5 updated CASC instructions + tuning
blanchet
parents: 60719
diff changeset
     2
<H2>Isabelle/HOL 2016-1</H2>
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     3
Jasmin C. Blanchette<sup>1</sup>, Lawrence C. Paulson<sup>2</sup>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     4
Tobias Nipkow<sup>1</sup>, Makarius Wenzel<sup>3</sup> <BR>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     5
<sup>1</sup>Technische Universit&auml;t M&uuml;nchen, Germany <BR>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     6
<sup>2</sup>University of Cambridge, United Kingdom <BR>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     7
<sup>3</sup>Universit&eacute; Paris Sud, France <BR>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     8
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
     9
<H3>Architecture</H3>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    10
64561
a7664ca9ffc5 updated CASC instructions + tuning
blanchet
parents: 60719
diff changeset
    11
Isabelle/HOL 2016-1 [<A HREF="#References">NPW13</A>] is the higher-order
a7664ca9ffc5 updated CASC instructions + tuning
blanchet
parents: 60719
diff changeset
    12
logic incarnation of the generic proof assistant
a7664ca9ffc5 updated CASC instructions + tuning
blanchet
parents: 60719
diff changeset
    13
<A HREF="http://www.cl.cam.ac.uk/research/hvg/Isabelle/">Isabelle2016-1</A>.
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    14
Isabelle/HOL provides several automatic proof tactics, notably an equational
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    15
reasoner [<A HREF="#References">Nip89</A>], a classical reasoner [<A
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    16
HREF="#References">Pau94</A>], and a tableau prover [<A
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    17
HREF="#References">Pau99</A>]. It also integrates external first- and
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    18
higher-order provers via its subsystem Sledgehammer [<A
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    19
HREF="#References">PB10</A>, <A HREF="#References">BBP11</A>].
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    20
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    21
<P>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    22
Isabelle includes a parser for the TPTP syntaxes CNF, FOF, TFF0, and THF0, due
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    23
to Nik Sultana. It also includes TPTP versions of its popular tools, invokable
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    24
on the command line as <tt>isabelle tptp_<em>tool</em> <em>max_secs</em>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    25
<em>file.p</em></tt>. For example:
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    26
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    27
<blockquote><pre>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    28
isabelle tptp_isabelle_hot 100 SEU/SEU824^3.p
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    29
</pre></blockquote>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    30
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    31
<P>
60719
b6713e04889e tuned description
blanchet
parents: 60717
diff changeset
    32
Isabelle is available in two versions. The <em>demo</em> (or HOT) version
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    33
includes its competitors LEO-II [<A HREF="#References">BPTF08</A>] and Satallax
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    34
[<A HREF="#References">Bro12</A>] as Sledgehammer backends, whereas the
60719
b6713e04889e tuned description
blanchet
parents: 60717
diff changeset
    35
<em>competition</em> version leaves them out. As the name suggests,
b6713e04889e tuned description
blanchet
parents: 60717
diff changeset
    36
only the competition version takes part in the competition.
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    37
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    38
<H3>Strategies</H3>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    39
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    40
The <em>Isabelle</em> tactic submitted to the competition simply tries the
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    41
following tactics sequentially:
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    42
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    43
<DL>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    44
<DT> <tt>sledgehammer</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    45
<DD> Invokes the following sequence of provers as oracles via Sledgehammer:
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    46
	<UL>
60717
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    47
	<LI> <tt>satallax</tt>&mdash;Satallax 2.7 [<A HREF="#References">Bro12</A>] (<em>demo only</em>);
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    48
	<LI> <tt>leo2</tt>&mdash;LEO-II 1.6.2 [<A HREF="#References">BPTF08</A>] (<em>demo only</em>);
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    49
	<LI> <tt>spass</tt>&mdash;SPASS 3.8ds [<A HREF="#References">BPWW12</A>];
60717
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    50
	<LI> <tt>vampire</tt>&mdash;Vampire 3.0 (revision 1803) [<A HREF="#References">RV02</A>];
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    51
	<LI> <tt>e</tt>&mdash;E 1.8 [<A HREF="#References">Sch04</A>];
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    52
	</UL>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    53
<DT> <tt>nitpick</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    54
<DD> For problems involving only the type <tt>$o</tt> of Booleans, checks
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    55
	 whether a finite model exists using Nitpick [<A HREF="#References">BN10</A>].
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    56
<DT> <tt>simp</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    57
<DD> Performs equational reasoning using rewrite rules [<A HREF="#References">Nip89</A>].
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    58
<DT> <tt>blast</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    59
<DD> Searches for a proof using a fast untyped tableau prover and then
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    60
     attempts to reconstruct the proof using Isabelle tactics
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    61
     [<A HREF="#References">Pau99</A>].
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    62
<DT> <tt>auto+spass</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    63
<DD> Combines simplification and classical reasoning
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    64
	 [<A HREF="#References">Pau94</A>] under one roof; then invoke Sledgehammer
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    65
     with SPASS on any subgoals that emerge.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    66
<DT> <tt>z3</tt>
60717
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    67
<DD> Invokes the SMT solver Z3 4.4.0-prerelease [<A HREF="#References">dMB08</A>].
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    68
<DT> <tt>cvc4</tt>
9a14d574ea65 updated Isabelle description to CASC
blanchet
parents: 60716
diff changeset
    69
<DD> Invokes the SMT solver CVC4 1.5-prerelease [<A HREF="#References">BT07</A>].
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    70
<DT> <tt>fast</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    71
<DD> Searches for a proof using sequent-style reasoning, performing a
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    72
     depth-first search [<A HREF="#References">Pau94</A>]. Unlike
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    73
     <tt>blast</tt>, it construct proofs directly in Isabelle. That makes it
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    74
     slower but enables it to work in the presence of the more unusual features
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    75
     of HOL, such as type classes and function unknowns.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    76
<DT> <tt>best</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    77
<DD> Similar to <tt>fast</tt>, except that it performs a best-first search.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    78
<DT> <tt>force</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    79
<DD> Similar to <tt>auto</tt>, but more exhaustive.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    80
<DT> <tt>meson</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    81
<DD> Implements Loveland's MESON procedure [<A HREF="#References">Lov78</A>].
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    82
Constructs proofs directly in Isabelle.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    83
<DT> <tt>fastforce</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    84
<DD> Combines <tt>fast</tt> and <tt>force</tt>.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    85
</DL>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    86
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    87
<H3>Implementation</H3>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    88
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    89
Isabelle is a generic theorem prover written in Standard ML. Its meta-logic,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    90
Isabelle/Pure, provides an intuitionistic fragment of higher-order logic. The
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    91
HOL object logic extends pure with a more elaborate version of higher-order
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    92
logic, complete with the familiar connectives and quantifiers. Other object
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    93
logics are available, notably FOL (first-order logic) and ZF
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    94
(Zermelo&ndash;Fraenkel set theory).
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    95
<P>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    96
The implementation of Isabelle relies on a small LCF-style kernel, meaning that
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    97
inferences are implemented as operations on an abstract <tt>theorem</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    98
datatype. Assuming the kernel is correct, all values of type <tt>theorem</tt>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
    99
are correct by construction.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   100
<P>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   101
Most of the code for Isabelle was written by the Isabelle teams at the
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   102
University of Cambridge and the Technische Universit&auml;t M&uuml;nchen.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   103
Isabelle/HOL is available for all major platforms under a BSD-style license
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   104
from
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   105
<PRE>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   106
    <A HREF="http:////www.cl.cam.ac.uk/research/hvg/Isabelle/">http://www.cl.cam.ac.uk/research/hvg/Isabelle</A></PRE>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   107
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   108
<H3>Expected Competition Performance</H3>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   109
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   110
<P>
60716
8e82a83757df imported patch up_casc
blanchet
parents: 52098
diff changeset
   111
Thanks to the addition of CVC4 and a new version of Vampire,
8e82a83757df imported patch up_casc
blanchet
parents: 52098
diff changeset
   112
Isabelle might have become now strong enough to take on Satallax
8e82a83757df imported patch up_casc
blanchet
parents: 52098
diff changeset
   113
and its various declensions. But we expect Isabelle to end in
8e82a83757df imported patch up_casc
blanchet
parents: 52098
diff changeset
   114
second or third place, to be honest.
52098
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   115
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   116
<H3>References</H3>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   117
<DL>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   118
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   119
<DT> BBP11
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   120
<DD> Blanchette J. C., B&ouml;hme S., Paulson L. C. (2011),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   121
     <STRONG>Extending Sledgehammer with SMT Solvers</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   122
     CADE-23, LNAI 6803, pp. 116&ndash;130, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   123
<DT> BN10
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   124
<DD> Blanchette J. C., Nipkow T. (2010),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   125
     <STRONG>Nitpick: A Counterexample Generator for Higher-Order Logic Based on a Relational Model Finder</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   126
     ITP 2010, <EM>LNCS</EM> 6172, pp. 131&ndash;146, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   127
<DT> BPTF08
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   128
<DD> Benzm&uuml;ller C., Paulson L. C., Theiss F., Fietzke A. (2008),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   129
  	 <STRONG>LEO-II&mdash;A Cooperative Automatic Theorem Prover for Higher-Order Logic</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   130
  	 IJCAR 2008, <EM>LNAI</EM> 5195, pp. 162&ndash;170, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   131
<DT> BPWW12
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   132
<DD> Blanchette J. C., Popescu A., Wand D., Weidenbach C. (2012),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   133
	 <STRONG>More SPASS with Isabelle</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   134
	 ITP 2012, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   135
<DT> Bro12
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   136
<DD> Brown C. (2012),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   137
	 <STRONG>Satallax: An Automated Higher-Order Prover (System Description)</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   138
	 IJCAR 2012, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   139
<DT> BT07
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   140
<DD> Barrett C., Tinelli C. (2007),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   141
	 <STRONG>CVC3 (System Description)</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   142
  	 CAV 2007, <EM>LNCS</EM> 4590, pp. 298&ndash;302, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   143
<DT> dMB08
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   144
<DD> de Moura L. M., Bj&oslash;rner N. (2008),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   145
     <STRONG>Z3: An Efficient SMT Solver</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   146
	 TACAS 2008, <EM>LNCS</EM> 4963, pp. 337&ndash;340, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   147
<DT> Lov78
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   148
<DD> Loveland D. W. (1978),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   149
     <STRONG>Automated Theorem Proving: A Logical Basis</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   150
     North-Holland Publishing Co.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   151
<DT> Nip89
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   152
<DD> Nipkow T. (1989),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   153
     <STRONG>Equational Reasoning in Isabelle</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   154
     <EM>Sci. Comput. Program.</EM> 12(2),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   155
     pp. 123&ndash;149,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   156
     Elsevier.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   157
<DT> NPW13
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   158
<DD> Nipkow T., Paulson L. C., Wenzel M. (2013),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   159
     <STRONG>Isabelle/HOL: A Proof Assistant for Higher-Order Logic</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   160
     <A HREF="http://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/Isabelle/doc/tutorial.pdf">http://www.cl.cam.ac.uk/research/hvg/Isabelle/dist/Isabelle/doc/tutorial.pdf</a>.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   161
<DT> Pau94
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   162
<DD> Paulson L. C. (1994),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   163
     <STRONG>Isabelle: A Generic Theorem Prover</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   164
     <EM>LNCS</EM> 828,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   165
     Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   166
<DT> Pau99
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   167
<DD> Paulson L. C. (1999),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   168
     <STRONG>A Generic Tableau Prover and Its Integration with Isabelle</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   169
     <EM>J. Univ. Comp. Sci.</EM> 5,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   170
     pp. 73&ndash;87.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   171
<DT> PB10
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   172
<DD> Paulson L. C., Blanchette J. C. (2010),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   173
     <STRONG>Three Years of Experience with Sledgehammer, a Practical Link between Automatic and Interactive Theorem Provers</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   174
     IWIL-2010.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   175
<DT> RV02
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   176
<DD> Riazanov A., Voronkov A. (2002),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   177
  	 <STRONG>The Design and Implementation of Vampire</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   178
  	 <EM>AI Comm.</EM> 15(2-3), 91&ndash;110.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   179
<DT> Sch04
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   180
<DD> Schulz S. (2004),
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   181
  	 <STRONG>System Description: E 0.81</STRONG>,
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   182
  	 IJCAR 2004, <EM>LNAI</EM> 3097, pp. 223&ndash;228, Springer.
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   183
</DL>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   184
<P>
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   185
6c38df1d294a added CASC-related files, to keep a public record of the Isabelle submission at the competition
blanchet
parents:
diff changeset
   186
<HR><!------------------------------------------------------------------------>