src/HOL/Cardinals/document/root.tex
author wenzelm
Tue, 05 Nov 2019 14:28:00 +0100
changeset 71047 87c132cf5860
parent 58715 cb8d2470623b
child 73404 299f6a8faccc
permissions -rw-r--r--
more options;

\documentclass[11pt,a4paper]{article}
\usepackage{isabelle,isabellesym}

% this should be the last package used
\usepackage{pdfsetup}

% urls in roman style, theory text in math-similar italics
\urlstyle{rm}
\isabellestyle{it}

\bibliographystyle{plain}

\begin{document}

\title{Ordinals and cardinals in HOL}
\author{Andrei Popescu \& Dmitriy Traytel}
\date{}
\maketitle

\tableofcontents

% sane default for proof documents
\parindent 0pt\parskip 0.5ex

\input{intro.tex}

\bibliography{root}

% generated text of all theories
\input{session}

% optional bibliography
%\bibliographystyle{abbrv}
%\bibliography{root}

\end{document}

%%% Local Variables:
%%% mode: latex
%%% TeX-master: t
%%% End: