| 
12668
 | 
     1  | 
\chapter{The Basics}
 | 
| 
8743
 | 
     2  | 
  | 
| 
 | 
     3  | 
\section{Introduction}
 | 
| 
 | 
     4  | 
  | 
| 
11405
 | 
     5  | 
This book is a tutorial on how to use the theorem prover Isabelle/HOL as a
  | 
| 
 | 
     6  | 
specification and verification system. Isabelle is a generic system for
  | 
| 
 | 
     7  | 
implementing logical formalisms, and Isabelle/HOL is the specialization
  | 
| 
 | 
     8  | 
of Isabelle for HOL, which abbreviates Higher-Order Logic. We introduce
  | 
| 
 | 
     9  | 
HOL step by step following the equation
  | 
| 
8743
 | 
    10  | 
\[ \mbox{HOL} = \mbox{Functional Programming} + \mbox{Logic}. \]
 | 
| 
11456
 | 
    11  | 
We do not assume that you are familiar with mathematical logic. 
  | 
| 
 | 
    12  | 
However, we do assume that
  | 
| 
 | 
    13  | 
you are used to logical and set theoretic notation, as covered
  | 
| 
 | 
    14  | 
in a good discrete mathematics course~\cite{Rosen-DMA}, and
 | 
| 
11450
 | 
    15  | 
that you are familiar with the basic concepts of functional
  | 
| 
11209
 | 
    16  | 
programming~\cite{Bird-Haskell,Hudak-Haskell,paulson-ml2,Thompson-Haskell}.
 | 
| 
 | 
    17  | 
Although this tutorial initially concentrates on functional programming, do
  | 
| 
 | 
    18  | 
not be misled: HOL can express most mathematical concepts, and functional
  | 
| 
 | 
    19  | 
programming is just one particularly simple and ubiquitous instance.
  | 
| 
8743
 | 
    20  | 
  | 
| 
11205
 | 
    21  | 
Isabelle~\cite{paulson-isa-book} is implemented in ML~\cite{SML}.  This has
 | 
| 
 | 
    22  | 
influenced some of Isabelle/HOL's concrete syntax but is otherwise irrelevant
  | 
| 
11450
 | 
    23  | 
for us: this tutorial is based on
  | 
| 
11213
 | 
    24  | 
Isabelle/Isar~\cite{isabelle-isar-ref}, an extension of Isabelle which hides
 | 
| 
 | 
    25  | 
the implementation language almost completely.  Thus the full name of the
  | 
| 
 | 
    26  | 
system should be Isabelle/Isar/HOL, but that is a bit of a mouthful.
  | 
| 
 | 
    27  | 
  | 
| 
 | 
    28  | 
There are other implementations of HOL, in particular the one by Mike Gordon
  | 
| 
11450
 | 
    29  | 
\index{Gordon, Mike}%
 | 
| 
11213
 | 
    30  | 
\emph{et al.}, which is usually referred to as ``the HOL system''
 | 
| 
 | 
    31  | 
\cite{mgordon-hol}. For us, HOL refers to the logical system, and sometimes
 | 
| 
11450
 | 
    32  | 
its incarnation Isabelle/HOL\@.
  | 
| 
8743
 | 
    33  | 
  | 
| 
 | 
    34  | 
A tutorial is by definition incomplete.  Currently the tutorial only
  | 
| 
 | 
    35  | 
introduces the rudiments of Isar's proof language. To fully exploit the power
  | 
| 
11213
 | 
    36  | 
of Isar, in particular the ability to write readable and structured proofs,
  | 
| 
15429
 | 
    37  | 
you should start with Nipkow's overview~\cite{Nipkow-TYPES02} and consult
 | 
| 
 | 
    38  | 
the Isabelle/Isar Reference Manual~\cite{isabelle-isar-ref} and Wenzel's
 | 
| 
 | 
    39  | 
PhD thesis~\cite{Wenzel-PhD} (which discusses many proof patterns)
 | 
| 
 | 
    40  | 
for further details. If you want to use Isabelle's ML level
  | 
| 
8743
 | 
    41  | 
directly (for example for writing your own proof procedures) see the Isabelle
  | 
| 
 | 
    42  | 
Reference Manual~\cite{isabelle-ref}; for details relating to HOL see the
 | 
| 
 | 
    43  | 
Isabelle/HOL manual~\cite{isabelle-HOL}. All manuals have a comprehensive
 | 
| 
 | 
    44  | 
index.
  | 
| 
 | 
    45  | 
  | 
| 
 | 
    46  | 
\section{Theories}
 | 
| 
 | 
    47  | 
\label{sec:Basic:Theories}
 | 
| 
 | 
    48  | 
  | 
| 
11428
 | 
    49  | 
\index{theories|(}%
 | 
| 
8743
 | 
    50  | 
Working with Isabelle means creating theories. Roughly speaking, a
  | 
| 
11428
 | 
    51  | 
\textbf{theory} is a named collection of types, functions, and theorems,
 | 
| 
8743
 | 
    52  | 
much like a module in a programming language or a specification in a
  | 
| 
 | 
    53  | 
specification language. In fact, theories in HOL can be either. The general
  | 
| 
 | 
    54  | 
format of a theory \texttt{T} is
 | 
| 
 | 
    55  | 
\begin{ttbox}
 | 
| 
15136
 | 
    56  | 
theory T
  | 
| 
15141
 | 
    57  | 
imports B\(@1\) \(\ldots\) B\(@n\)
  | 
| 
15136
 | 
    58  | 
begin
  | 
| 
11450
 | 
    59  | 
{\rmfamily\textit{declarations, definitions, and proofs}}
 | 
| 
8743
 | 
    60  | 
end
  | 
| 
15358
 | 
    61  | 
\end{ttbox}\cmmdx{theory}\cmmdx{imports}
 | 
| 
15136
 | 
    62  | 
where \texttt{B}$@1$ \dots\ \texttt{B}$@n$ are the names of existing
 | 
| 
11450
 | 
    63  | 
theories that \texttt{T} is based on and \textit{declarations,
 | 
| 
 | 
    64  | 
    definitions, and proofs} represents the newly introduced concepts
  | 
| 
8771
 | 
    65  | 
(types, functions etc.) and proofs about them. The \texttt{B}$@i$ are the
 | 
| 
11450
 | 
    66  | 
direct \textbf{parent theories}\indexbold{parent theories} of~\texttt{T}\@.
 | 
| 
 | 
    67  | 
Everything defined in the parent theories (and their parents, recursively) is
  | 
| 
8743
 | 
    68  | 
automatically visible. To avoid name clashes, identifiers can be
  | 
| 
11450
 | 
    69  | 
\textbf{qualified}\indexbold{identifiers!qualified}
 | 
| 
 | 
    70  | 
by theory names as in \texttt{T.f} and~\texttt{B.f}. 
 | 
| 
 | 
    71  | 
Each theory \texttt{T} must
 | 
| 
11428
 | 
    72  | 
reside in a \textbf{theory file}\index{theory files} named \texttt{T.thy}.
 | 
| 
8743
 | 
    73  | 
  | 
| 
 | 
    74  | 
This tutorial is concerned with introducing you to the different linguistic
  | 
| 
11450
 | 
    75  | 
constructs that can fill the \textit{declarations, definitions, and
 | 
| 
 | 
    76  | 
    proofs} above.  A complete grammar of the basic
  | 
| 
12327
 | 
    77  | 
constructs is found in the Isabelle/Isar Reference
  | 
| 
 | 
    78  | 
Manual~\cite{isabelle-isar-ref}.
 | 
| 
8743
 | 
    79  | 
  | 
| 
10885
 | 
    80  | 
HOL's theory collection is available online at
  | 
| 
8743
 | 
    81  | 
\begin{center}\small
 | 
| 
10978
 | 
    82  | 
    \url{http://isabelle.in.tum.de/library/HOL/}
 | 
| 
8743
 | 
    83  | 
\end{center}
 | 
| 
10885
 | 
    84  | 
and is recommended browsing. Note that most of the theories 
  | 
| 
9541
 | 
    85  | 
are based on classical Isabelle without the Isar extension. This means that
  | 
| 
 | 
    86  | 
they look slightly different than the theories in this tutorial, and that all
  | 
| 
 | 
    87  | 
proofs are in separate ML files.
  | 
| 
 | 
    88  | 
  | 
| 
8743
 | 
    89  | 
\begin{warn}
 | 
| 
11428
 | 
    90  | 
  HOL contains a theory \thydx{Main}, the union of all the basic
 | 
| 
10885
 | 
    91  | 
  predefined theories like arithmetic, lists, sets, etc.  
  | 
| 
 | 
    92  | 
  Unless you know what you are doing, always include \isa{Main}
 | 
| 
10971
 | 
    93  | 
  as a direct or indirect parent of all your theories.
  | 
| 
12332
 | 
    94  | 
\end{warn}
 | 
| 
12473
 | 
    95  | 
There is also a growing Library~\cite{HOL-Library}\index{Library}
 | 
| 
13814
 | 
    96  | 
of useful theories that are not part of \isa{Main} but can be included
 | 
| 
12473
 | 
    97  | 
among the parents of a theory and will then be loaded automatically.%
  | 
| 
11428
 | 
    98  | 
\index{theories|)}
 | 
| 
8743
 | 
    99  | 
  | 
| 
 | 
   100  | 
  | 
| 
10885
 | 
   101  | 
\section{Types, Terms and Formulae}
 | 
| 
8743
 | 
   102  | 
\label{sec:TypesTermsForms}
 | 
| 
 | 
   103  | 
  | 
| 
10795
 | 
   104  | 
Embedded in a theory are the types, terms and formulae of HOL\@. HOL is a typed
  | 
| 
8771
 | 
   105  | 
logic whose type system resembles that of functional programming languages
  | 
| 
11450
 | 
   106  | 
like ML or Haskell. Thus there are
  | 
| 
 | 
   107  | 
\index{types|(}
 | 
| 
8743
 | 
   108  | 
\begin{description}
 | 
| 
11450
 | 
   109  | 
\item[base types,] 
  | 
| 
 | 
   110  | 
in particular \tydx{bool}, the type of truth values,
 | 
| 
11428
 | 
   111  | 
and \tydx{nat}, the type of natural numbers.
 | 
| 
11450
 | 
   112  | 
\item[type constructors,]\index{type constructors}
 | 
| 
 | 
   113  | 
 in particular \tydx{list}, the type of
 | 
| 
11428
 | 
   114  | 
lists, and \tydx{set}, the type of sets. Type constructors are written
 | 
| 
8771
 | 
   115  | 
postfix, e.g.\ \isa{(nat)list} is the type of lists whose elements are
 | 
| 
8743
 | 
   116  | 
natural numbers. Parentheses around single arguments can be dropped (as in
  | 
| 
8771
 | 
   117  | 
\isa{nat list}), multiple arguments are separated by commas (as in
 | 
| 
 | 
   118  | 
\isa{(bool,nat)ty}).
 | 
| 
11450
 | 
   119  | 
\item[function types,]\index{function types}
 | 
| 
 | 
   120  | 
denoted by \isasymFun\indexbold{$IsaFun@\isasymFun}.
 | 
| 
8771
 | 
   121  | 
  In HOL \isasymFun\ represents \emph{total} functions only. As is customary,
 | 
| 
 | 
   122  | 
  \isa{$\tau@1$ \isasymFun~$\tau@2$ \isasymFun~$\tau@3$} means
 | 
| 
 | 
   123  | 
  \isa{$\tau@1$ \isasymFun~($\tau@2$ \isasymFun~$\tau@3$)}. Isabelle also
 | 
| 
 | 
   124  | 
  supports the notation \isa{[$\tau@1,\dots,\tau@n$] \isasymFun~$\tau$}
 | 
| 
 | 
   125  | 
  which abbreviates \isa{$\tau@1$ \isasymFun~$\cdots$ \isasymFun~$\tau@n$
 | 
| 
8743
 | 
   126  | 
    \isasymFun~$\tau$}.
  | 
| 
11450
 | 
   127  | 
\item[type variables,]\index{type variables}\index{variables!type}
 | 
| 
10795
 | 
   128  | 
  denoted by \ttindexboldpos{'a}{$Isatype}, \isa{'b} etc., just like in ML\@. They give rise
 | 
| 
8771
 | 
   129  | 
  to polymorphic types like \isa{'a \isasymFun~'a}, the type of the identity
 | 
| 
 | 
   130  | 
  function.
  | 
| 
8743
 | 
   131  | 
\end{description}
 | 
| 
 | 
   132  | 
\begin{warn}
 | 
| 
 | 
   133  | 
  Types are extremely important because they prevent us from writing
  | 
| 
 | 
   134  | 
  nonsense.  Isabelle insists that all terms and formulae must be well-typed
  | 
| 
 | 
   135  | 
  and will print an error message if a type mismatch is encountered. To
  | 
| 
 | 
   136  | 
  reduce the amount of explicit type information that needs to be provided by
  | 
| 
 | 
   137  | 
  the user, Isabelle infers the type of all variables automatically (this is
  | 
| 
 | 
   138  | 
  called \bfindex{type inference}) and keeps quiet about it. Occasionally
 | 
| 
 | 
   139  | 
  this may lead to misunderstandings between you and the system. If anything
  | 
| 
11428
 | 
   140  | 
  strange happens, we recommend that you set the flag\index{flags}
 | 
| 
 | 
   141  | 
  \isa{show_types}\index{*show_types (flag)}.  
 | 
| 
 | 
   142  | 
  Isabelle will then display type information
  | 
| 
11450
 | 
   143  | 
  that is usually suppressed.  Simply type
  | 
| 
8743
 | 
   144  | 
\begin{ttbox}
 | 
| 
 | 
   145  | 
ML "set show_types"
  | 
| 
 | 
   146  | 
\end{ttbox}
 | 
| 
 | 
   147  | 
  | 
| 
 | 
   148  | 
\noindent
  | 
| 
10971
 | 
   149  | 
This can be reversed by \texttt{ML "reset show_types"}. Various other flags,
 | 
| 
11428
 | 
   150  | 
which we introduce as we go along, can be set and reset in the same manner.%
  | 
| 
 | 
   151  | 
\index{flags!setting and resetting}
 | 
| 
11450
 | 
   152  | 
\end{warn}%
 | 
| 
 | 
   153  | 
\index{types|)}
 | 
| 
8743
 | 
   154  | 
  | 
| 
 | 
   155  | 
  | 
| 
11450
 | 
   156  | 
\index{terms|(}
 | 
| 
 | 
   157  | 
\textbf{Terms} are formed as in functional programming by
 | 
| 
8771
 | 
   158  | 
applying functions to arguments. If \isa{f} is a function of type
 | 
| 
 | 
   159  | 
\isa{$\tau@1$ \isasymFun~$\tau@2$} and \isa{t} is a term of type
 | 
| 
 | 
   160  | 
$\tau@1$ then \isa{f~t} is a term of type $\tau@2$. HOL also supports
 | 
| 
 | 
   161  | 
infix functions like \isa{+} and some basic constructs from functional
 | 
| 
11428
 | 
   162  | 
programming, such as conditional expressions:
  | 
| 
8743
 | 
   163  | 
\begin{description}
 | 
| 
11450
 | 
   164  | 
\item[\isa{if $b$ then $t@1$ else $t@2$}]\index{*if expressions}
 | 
| 
11428
 | 
   165  | 
Here $b$ is of type \isa{bool} and $t@1$ and $t@2$ are of the same type.
 | 
| 
11450
 | 
   166  | 
\item[\isa{let $x$ = $t$ in $u$}]\index{*let expressions}
 | 
| 
13814
 | 
   167  | 
is equivalent to $u$ where all free occurrences of $x$ have been replaced by
  | 
| 
8743
 | 
   168  | 
$t$. For example,
  | 
| 
8771
 | 
   169  | 
\isa{let x = 0 in x+x} is equivalent to \isa{0+0}. Multiple bindings are separated
 | 
| 
13814
 | 
   170  | 
by semicolons: \isa{let $x@1$ = $t@1$;\dots; $x@n$ = $t@n$ in $u$}.
 | 
| 
8771
 | 
   171  | 
\item[\isa{case $e$ of $c@1$ \isasymFun~$e@1$ |~\dots~| $c@n$ \isasymFun~$e@n$}]
 | 
| 
11450
 | 
   172  | 
\index{*case expressions}
 | 
| 
8771
 | 
   173  | 
evaluates to $e@i$ if $e$ is of the form $c@i$.
  | 
| 
8743
 | 
   174  | 
\end{description}
 | 
| 
 | 
   175  | 
  | 
| 
 | 
   176  | 
Terms may also contain
  | 
| 
11450
 | 
   177  | 
\isasymlambda-abstractions.\index{lambda@$\lambda$ expressions}
 | 
| 
 | 
   178  | 
For example,
  | 
| 
8771
 | 
   179  | 
\isa{\isasymlambda{}x.~x+1} is the function that takes an argument \isa{x} and
 | 
| 
 | 
   180  | 
returns \isa{x+1}. Instead of
 | 
| 
 | 
   181  | 
\isa{\isasymlambda{}x.\isasymlambda{}y.\isasymlambda{}z.~$t$} we can write
 | 
| 
11450
 | 
   182  | 
\isa{\isasymlambda{}x~y~z.~$t$}.%
 | 
| 
 | 
   183  | 
\index{terms|)}
 | 
| 
8743
 | 
   184  | 
  | 
| 
11450
 | 
   185  | 
\index{formulae|(}%
 | 
| 
 | 
   186  | 
\textbf{Formulae} are terms of type \tydx{bool}.
 | 
| 
11428
 | 
   187  | 
There are the basic constants \cdx{True} and \cdx{False} and
 | 
| 
8771
 | 
   188  | 
the usual logical connectives (in decreasing order of priority):
  | 
| 
11420
 | 
   189  | 
\indexboldpos{\protect\isasymnot}{$HOL0not}, \indexboldpos{\protect\isasymand}{$HOL0and},
 | 
| 
 | 
   190  | 
\indexboldpos{\protect\isasymor}{$HOL0or}, and \indexboldpos{\protect\isasymimp}{$HOL0imp},
 | 
| 
8743
 | 
   191  | 
all of which (except the unary \isasymnot) associate to the right. In
  | 
| 
8771
 | 
   192  | 
particular \isa{A \isasymimp~B \isasymimp~C} means \isa{A \isasymimp~(B
 | 
| 
 | 
   193  | 
  \isasymimp~C)} and is thus logically equivalent to \isa{A \isasymand~B
 | 
| 
 | 
   194  | 
  \isasymimp~C} (which is \isa{(A \isasymand~B) \isasymimp~C}).
 | 
| 
8743
 | 
   195  | 
  | 
| 
11450
 | 
   196  | 
Equality\index{equality} is available in the form of the infix function
 | 
| 
 | 
   197  | 
\isa{=} of type \isa{'a \isasymFun~'a
 | 
| 
8771
 | 
   198  | 
  \isasymFun~bool}. Thus \isa{$t@1$ = $t@2$} is a formula provided $t@1$
 | 
| 
11450
 | 
   199  | 
and $t@2$ are terms of the same type. If $t@1$ and $t@2$ are of type
  | 
| 
 | 
   200  | 
\isa{bool} then \isa{=} acts as \rmindex{if-and-only-if}.
 | 
| 
 | 
   201  | 
The formula
  | 
| 
8771
 | 
   202  | 
\isa{$t@1$~\isasymnoteq~$t@2$} is merely an abbreviation for
 | 
| 
 | 
   203  | 
\isa{\isasymnot($t@1$ = $t@2$)}.
 | 
| 
8743
 | 
   204  | 
  | 
| 
11450
 | 
   205  | 
Quantifiers\index{quantifiers} are written as
 | 
| 
 | 
   206  | 
\isa{\isasymforall{}x.~$P$} and \isa{\isasymexists{}x.~$P$}. 
 | 
| 
11420
 | 
   207  | 
There is even
  | 
| 
11450
 | 
   208  | 
\isa{\isasymuniqex{}x.~$P$}, which
 | 
| 
11420
 | 
   209  | 
means that there exists exactly one \isa{x} that satisfies \isa{$P$}. 
 | 
| 
 | 
   210  | 
Nested quantifications can be abbreviated:
  | 
| 
 | 
   211  | 
\isa{\isasymforall{}x~y~z.~$P$} means
 | 
| 
11450
 | 
   212  | 
\isa{\isasymforall{}x.\isasymforall{}y.\isasymforall{}z.~$P$}.%
 | 
| 
 | 
   213  | 
\index{formulae|)}
 | 
| 
8743
 | 
   214  | 
  | 
| 
 | 
   215  | 
Despite type inference, it is sometimes necessary to attach explicit
  | 
| 
11428
 | 
   216  | 
\bfindex{type constraints} to a term.  The syntax is
 | 
| 
8771
 | 
   217  | 
\isa{$t$::$\tau$} as in \isa{x < (y::nat)}. Note that
 | 
| 
10538
 | 
   218  | 
\ttindexboldpos{::}{$Isatype} binds weakly and should therefore be enclosed
 | 
| 
11450
 | 
   219  | 
in parentheses.  For instance,
  | 
| 
 | 
   220  | 
\isa{x < y::nat} is ill-typed because it is interpreted as
 | 
| 
 | 
   221  | 
\isa{(x < y)::nat}.  Type constraints may be needed to disambiguate
 | 
| 
 | 
   222  | 
expressions
  | 
| 
 | 
   223  | 
involving overloaded functions such as~\isa{+}, 
 | 
| 
 | 
   224  | 
\isa{*} and~\isa{<}.  Section~\ref{sec:overloading} 
 | 
| 
 | 
   225  | 
discusses overloading, while Table~\ref{tab:overloading} presents the most
 | 
| 
10695
 | 
   226  | 
important overloaded function symbols.
  | 
| 
8743
 | 
   227  | 
  | 
| 
11450
 | 
   228  | 
In general, HOL's concrete \rmindex{syntax} tries to follow the conventions of
 | 
| 
 | 
   229  | 
functional programming and mathematics.  Here are the main rules that you
  | 
| 
 | 
   230  | 
should be familiar with to avoid certain syntactic traps:
  | 
| 
8743
 | 
   231  | 
\begin{itemize}
 | 
| 
 | 
   232  | 
\item
  | 
| 
8771
 | 
   233  | 
Remember that \isa{f t u} means \isa{(f t) u} and not \isa{f(t u)}!
 | 
| 
8743
 | 
   234  | 
\item
  | 
| 
8771
 | 
   235  | 
Isabelle allows infix functions like \isa{+}. The prefix form of function
 | 
| 
 | 
   236  | 
application binds more strongly than anything else and hence \isa{f~x + y}
 | 
| 
 | 
   237  | 
means \isa{(f~x)~+~y} and not \isa{f(x+y)}.
 | 
| 
8743
 | 
   238  | 
\item Remember that in HOL if-and-only-if is expressed using equality.  But
  | 
| 
 | 
   239  | 
  equality has a high priority, as befitting a relation, while if-and-only-if
  | 
| 
8771
 | 
   240  | 
  typically has the lowest priority.  Thus, \isa{\isasymnot~\isasymnot~P =
 | 
| 
 | 
   241  | 
    P} means \isa{\isasymnot\isasymnot(P = P)} and not
 | 
| 
 | 
   242  | 
  \isa{(\isasymnot\isasymnot P) = P}. When using \isa{=} to mean
 | 
| 
 | 
   243  | 
  logical equivalence, enclose both operands in parentheses, as in \isa{(A
 | 
| 
8743
 | 
   244  | 
    \isasymand~B) = (B \isasymand~A)}.
  | 
| 
 | 
   245  | 
\item
  | 
| 
 | 
   246  | 
Constructs with an opening but without a closing delimiter bind very weakly
  | 
| 
 | 
   247  | 
and should therefore be enclosed in parentheses if they appear in subterms, as
  | 
| 
11450
 | 
   248  | 
in \isa{(\isasymlambda{}x.~x) = f}.  This includes 
 | 
| 
 | 
   249  | 
\isa{if},\index{*if expressions}
 | 
| 
 | 
   250  | 
\isa{let},\index{*let expressions}
 | 
| 
 | 
   251  | 
\isa{case},\index{*case expressions}
 | 
| 
 | 
   252  | 
\isa{\isasymlambda}, and quantifiers.
 | 
| 
8743
 | 
   253  | 
\item
  | 
| 
8771
 | 
   254  | 
Never write \isa{\isasymlambda{}x.x} or \isa{\isasymforall{}x.x=x}
 | 
| 
12327
 | 
   255  | 
because \isa{x.x} is always taken as a single qualified identifier. Write
 | 
| 
8771
 | 
   256  | 
\isa{\isasymlambda{}x.~x} and \isa{\isasymforall{}x.~x=x} instead.
 | 
| 
11450
 | 
   257  | 
\item Identifiers\indexbold{identifiers} may contain the characters \isa{_} 
 | 
| 
12327
 | 
   258  | 
and~\isa{'}, except at the beginning.
 | 
| 
8743
 | 
   259  | 
\end{itemize}
 | 
| 
 | 
   260  | 
  | 
| 
11450
 | 
   261  | 
For the sake of readability, we use the usual mathematical symbols throughout
  | 
| 
10983
 | 
   262  | 
the tutorial. Their \textsc{ascii}-equivalents are shown in table~\ref{tab:ascii} in
 | 
| 
8771
 | 
   263  | 
the appendix.
  | 
| 
 | 
   264  | 
  | 
| 
11450
 | 
   265  | 
\begin{warn}
 | 
| 
 | 
   266  | 
A particular
  | 
| 
 | 
   267  | 
problem for novices can be the priority of operators. If you are unsure, use
  | 
| 
 | 
   268  | 
additional parentheses. In those cases where Isabelle echoes your
  | 
| 
 | 
   269  | 
input, you can see which parentheses are dropped --- they were superfluous. If
  | 
| 
 | 
   270  | 
you are unsure how to interpret Isabelle's output because you don't know
  | 
| 
 | 
   271  | 
where the (dropped) parentheses go, set the flag\index{flags}
 | 
| 
 | 
   272  | 
\isa{show_brackets}\index{*show_brackets (flag)}:
 | 
| 
 | 
   273  | 
\begin{ttbox}
 | 
| 
 | 
   274  | 
ML "set show_brackets"; \(\dots\); ML "reset show_brackets";
  | 
| 
 | 
   275  | 
\end{ttbox}
 | 
| 
 | 
   276  | 
\end{warn}
 | 
| 
 | 
   277  | 
  | 
| 
8743
 | 
   278  | 
  | 
| 
 | 
   279  | 
\section{Variables}
 | 
| 
 | 
   280  | 
\label{sec:variables}
 | 
| 
11450
 | 
   281  | 
\index{variables|(}
 | 
| 
8743
 | 
   282  | 
  | 
| 
11450
 | 
   283  | 
Isabelle distinguishes free and bound variables, as is customary. Bound
  | 
| 
8743
 | 
   284  | 
variables are automatically renamed to avoid clashes with free variables. In
  | 
| 
11428
 | 
   285  | 
addition, Isabelle has a third kind of variable, called a \textbf{schematic
 | 
| 
 | 
   286  | 
  variable}\index{variables!schematic} or \textbf{unknown}\index{unknowns}, 
 | 
| 
13439
 | 
   287  | 
which must have a~\isa{?} as its first character.  
 | 
| 
11428
 | 
   288  | 
Logically, an unknown is a free variable. But it may be
  | 
| 
8743
 | 
   289  | 
instantiated by another term during the proof process. For example, the
  | 
| 
8771
 | 
   290  | 
mathematical theorem $x = x$ is represented in Isabelle as \isa{?x = ?x},
 | 
| 
8743
 | 
   291  | 
which means that Isabelle can instantiate it arbitrarily. This is in contrast
  | 
| 
 | 
   292  | 
to ordinary variables, which remain fixed. The programming language Prolog
  | 
| 
 | 
   293  | 
calls unknowns {\em logical\/} variables.
 | 
| 
 | 
   294  | 
  | 
| 
 | 
   295  | 
Most of the time you can and should ignore unknowns and work with ordinary
  | 
| 
 | 
   296  | 
variables. Just don't be surprised that after you have finished the proof of
  | 
| 
11450
 | 
   297  | 
a theorem, Isabelle will turn your free variables into unknowns.  It
  | 
| 
8743
 | 
   298  | 
indicates that Isabelle will automatically instantiate those unknowns
  | 
| 
 | 
   299  | 
suitably when the theorem is used in some other proof.
  | 
| 
9689
 | 
   300  | 
Note that for readability we often drop the \isa{?}s when displaying a theorem.
 | 
| 
8743
 | 
   301  | 
\begin{warn}
 | 
| 
11450
 | 
   302  | 
  For historical reasons, Isabelle accepts \isa{?} as an ASCII representation
 | 
| 
 | 
   303  | 
  of the \(\exists\) symbol.  However, the \isa{?} character must then be followed
 | 
| 
 | 
   304  | 
  by a space, as in \isa{?~x. f(x) = 0}.  Otherwise, \isa{?x} is
 | 
| 
 | 
   305  | 
  interpreted as a schematic variable.  The preferred ASCII representation of
  | 
| 
 | 
   306  | 
  the \(\exists\) symbol is \isa{EX}\@. 
 | 
| 
 | 
   307  | 
\end{warn}%
 | 
| 
 | 
   308  | 
\index{variables|)}
 | 
| 
8743
 | 
   309  | 
  | 
| 
10885
 | 
   310  | 
\section{Interaction and Interfaces}
 | 
| 
8771
 | 
   311  | 
  | 
| 
 | 
   312  | 
Interaction with Isabelle can either occur at the shell level or through more
  | 
| 
11301
 | 
   313  | 
advanced interfaces. To keep the tutorial independent of the interface, we
  | 
| 
 | 
   314  | 
have phrased the description of the interaction in a neutral language. For
  | 
| 
8771
 | 
   315  | 
example, the phrase ``to abandon a proof'' means to type \isacommand{oops} at the
 | 
| 
 | 
   316  | 
shell level, which is explained the first time the phrase is used. Other
  | 
| 
 | 
   317  | 
interfaces perform the same act by cursor movements and/or mouse clicks.
  | 
| 
 | 
   318  | 
Although shell-based interaction is quite feasible for the kind of proof
  | 
| 
 | 
   319  | 
scripts currently presented in this tutorial, the recommended interface for
  | 
| 
 | 
   320  | 
Isabelle/Isar is the Emacs-based \bfindex{Proof
 | 
| 
11450
 | 
   321  | 
  General}~\cite{proofgeneral,Aspinall:TACAS:2000}.
 | 
| 
8771
 | 
   322  | 
  | 
| 
 | 
   323  | 
Some interfaces (including the shell level) offer special fonts with
  | 
| 
10983
 | 
   324  | 
mathematical symbols. For those that do not, remember that \textsc{ascii}-equivalents
 | 
| 
10978
 | 
   325  | 
are shown in table~\ref{tab:ascii} in the appendix.
 | 
| 
8771
 | 
   326  | 
  | 
| 
9541
 | 
   327  | 
Finally, a word about semicolons.\indexbold{$Isar@\texttt{;}} 
 | 
| 
 | 
   328  | 
Commands may but need not be terminated by semicolons.
  | 
| 
 | 
   329  | 
At the shell level it is advisable to use semicolons to enforce that a command
  | 
| 
8771
 | 
   330  | 
is executed immediately; otherwise Isabelle may wait for the next keyword
  | 
| 
9541
 | 
   331  | 
before it knows that the command is complete.
  | 
| 
8771
 | 
   332  | 
  | 
| 
 | 
   333  | 
  | 
| 
10885
 | 
   334  | 
\section{Getting Started}
 | 
| 
8743
 | 
   335  | 
  | 
| 
 | 
   336  | 
Assuming you have installed Isabelle, you start it by typing \texttt{isabelle
 | 
| 
 | 
   337  | 
  -I HOL} in a shell window.\footnote{Simply executing \texttt{isabelle -I}
 | 
| 
 | 
   338  | 
  starts the default logic, which usually is already \texttt{HOL}.  This is
 | 
| 
 | 
   339  | 
  controlled by the \texttt{ISABELLE_LOGIC} setting, see \emph{The Isabelle
 | 
| 
 | 
   340  | 
    System Manual} for more details.} This presents you with Isabelle's most
  | 
| 
10983
 | 
   341  | 
basic \textsc{ascii} interface.  In addition you need to open an editor window to
 | 
| 
11450
 | 
   342  | 
create theory files.  While you are developing a theory, we recommend that you
  | 
| 
8743
 | 
   343  | 
type each command into the file first and then enter it into Isabelle by
  | 
| 
 | 
   344  | 
copy-and-paste, thus ensuring that you have a complete record of your theory.
  | 
| 
8771
 | 
   345  | 
As mentioned above, Proof General offers a much superior interface.
  | 
| 
10795
 | 
   346  | 
If you have installed Proof General, you can start it by typing \texttt{Isabelle}.
 |