src/HOL/Library/Library/document/root.tex
author wenzelm
Mon, 13 Oct 2008 14:04:28 +0200
changeset 28571 47d88239658d
parent 26590 9114b5fe533a
child 31975 366ad09d39ef
permissions -rw-r--r--
** Update from Fabian ** preferences/provers: separated by white space, avoid low-level char type; sledgehammer command accepts prover list as well; avoid I/O in critical section of AtpManager.info; more systematic synchronization using higher-order combinators; more descriptive errors when atp fails; keep explicitly requested problem files; added remote prover functions; simplified treatment of prover name in diagnostic output; misc tuning and cleanup;


% $Id$

\documentclass[11pt,a4paper]{article}
\usepackage{ifthen}
\usepackage[latin1]{inputenc}
\usepackage[english]{babel}
\usepackage{isabelle,isabellesym,amssymb}
\usepackage{pdfsetup}

\urlstyle{rm}
\isabellestyle{it}
\pagestyle{myheadings}

\begin{document}

\title{The Supplemental Isabelle/HOL Library}
\author{}
\maketitle

\tableofcontents
\newpage

\renewcommand{\isamarkupheader}[1]%
{\ifthenelse{\equal{#1}{}}{\section{\isabellecontext}}{\section{\isabellecontext: #1}}%
\markright{THEORY~``\isabellecontext''}}
\renewcommand{\isasymguillemotright}{$\gg$}

\input{session}

\pagestyle{headings}
\bibliographystyle{abbrv}
\bibliography{root}

\end{document}