src/Doc/How_to_Prove_it/document/root.tex
author wenzelm
Fri, 23 Nov 2018 16:43:11 +0100
changeset 69334 6b49700da068
parent 56820 7fbed439b8d3
child 73723 1bbbaae6b5e3
permissions -rw-r--r--
clarified font_domain: strict excludes e.g. space character;

\documentclass[11pt,a4paper]{report}

\input{prelude}

\begin{document}

\title{How to Prove it in Isabelle/HOL}
%\subtitle{\includegraphics[scale=.7]{isabelle_hol}}
\author{Tobias Nipkow}
\maketitle


\begin{abstract}
  How does one perform induction on the length of a list? How are numerals
  converted into \isa{Suc} terms? How does one prove equalities in rings
  and other algebraic structures?

  This document is a collection of practical hints and techniques for dealing
  with specific frequently occurring situations in proofs in Isabelle/HOL.
  Not arbitrary proofs but proofs that refer to material that is part of
  \isa{Main} or \isa{Complex\_Main}.

  This is \emph{not} an introduction to
\begin{itemize}
\item proofs in general; for that see mathematics or logic books.
\item Isabelle/HOL and its proof language; for that see the tutorial
  \cite{ProgProve} or the reference manual~\cite{IsarRef}.
\item the contents of theory \isa{Main}; for that see the overview
  \cite{Main}.
\end{itemize}
\end{abstract}

\setcounter{tocdepth}{1}
\tableofcontents

\input{How_to_Prove_it.tex}

\bibliographystyle{plain}
\bibliography{root}

%\printindex

\end{document}