src/HOL/Isar_examples/document/root.tex
author wenzelm
Wed, 18 Oct 2000 23:35:56 +0200
changeset 10257 21055ac27708
parent 10146 e89309dde9d3
child 12105 1e4451999200
permissions -rw-r--r--
MultisetOrder mmoved to HOL/Library;


% $Id$

\input{style}

\hyphenation{Isabelle}

\begin{document}

\title{Miscellaneous Isabelle/Isar examples for Higher-Order Logic}
\author{Markus Wenzel \\ \url{http://www.in.tum.de/~wenzelm/} \\[2ex]
  With contributions by Gertrud Bauer and Tobias Nipkow}
\maketitle

\begin{abstract}
  Isar offers a high-level proof (and theory) language for Isabelle.
  We give various examples of Isabelle/Isar proof developments,
  ranging from simple demonstrations of certain language features to
  more advanced applications.
\end{abstract}

\tableofcontents

\parindent 0pt \parskip 0.5ex

\input{BasicLogic.tex}
\input{Cantor.tex}
\input{Peirce.tex}
\input{ExprCompiler.tex}
\input{Group.tex}
\input{Summation.tex}
\input{KnasterTarski.tex}
\input{MutilatedCheckerboard.tex}
%\input{Maybe.tex}
%\input{Type.tex}
\input{W_correct.tex}
%\input{Primes.tex}
\input{Fibonacci.tex}
\input{Puzzle.tex}
\input{NestedDatatype.tex}
\input{Hoare.tex}
\input{HoareEx.tex}

\nocite{isabelle-isar-ref,Wenzel:1999:TPHOL}
\bibliographystyle{plain}
\bibliography{root}

\end{document}