src/Doc/Datatypes/document/root.tex
author blanchet
Fri, 13 Sep 2013 16:50:35 +0200
changeset 53619 27d2c98d9d9f
parent 53617 da5e1887d7a7
child 53621 9c3a80af72ff
permissions -rw-r--r--
more (co)data docs

\documentclass[12pt,a4paper]{article} % fleqn
\usepackage{cite}
\usepackage{enumitem}
\usepackage{latexsym}
\usepackage{graphicx}
\usepackage{iman}
\usepackage{extra}
\usepackage{isar}
\usepackage{isabelle}
\usepackage{isabellesym}
\usepackage{style}
\usepackage{pdfsetup}
\usepackage{railsetup}
\usepackage{framed}

\setcounter{secnumdepth}{3}
\setcounter{tocdepth}{3}

\newbox\boxA
\setbox\boxA=\hbox{\ }
\parindent=4\wd\boxA

\newcommand\blankline{\vskip-.5\baselineskip}

\newenvironment{indentblock}{\list{}{}\item[]}{\endlist}

\newcommand{\keyw}[1]{\textbf{#1}}
\newcommand{\synt}[1]{\textit{#1}}
\newcommand{\hthm}[1]{\textbf{\textit{#1}}}

%\renewcommand{\isactrlsub}[1]{\/$\sb{\mathrm{#1}}$}
\renewcommand{\isactrlsub}[1]{\/$\sb{#1}$}
\renewcommand{\isadigit}[1]{\/\ensuremath{\mathrm{#1}}}
\renewcommand{\isacharprime}{\isamath{{'}\mskip-2mu}}
\renewcommand{\isacharunderscore}{\mbox{\_}}
\renewcommand{\isacharunderscorekeyword}{\mbox{\_}}
\renewcommand{\isachardoublequote}{\mbox{\upshape{``}}}
\renewcommand{\isachardoublequoteopen}{\mbox{\upshape{``}\kern.1ex}}
\renewcommand{\isachardoublequoteclose}{\/\kern.15ex\mbox{\upshape{''}}}

\hyphenation{isa-belle}

\isadroptag{theory}

\title{%\includegraphics[scale=0.5]{isabelle_hol} \\[4ex]
Defining (Co)datatypes in Isabelle/HOL}
\author{\hbox{} \\
Jasmin Christian Blanchette,
Lorenz Panny, \\
Andrei Popescu, and
Dmitriy Traytel \\
{\normalsize Institut f\"ur Informatik, Technische Universit\"at M\"unchen} \\
\hbox{}}
\begin{document}

\maketitle

\begin{abstract}
\noindent
This tutorial describes how to use the new package for defining datatypes and
codatatypes in Isabelle/HOL. The package provides four main commands:
\keyw{datatype\_new}, \keyw{codatatype}, \keyw{primrec\_new}, and
\keyw{primcorec}. The commands suffixed by \keyw{\_new} are intended to subsume,
and eventually replace, the corresponding commands from the old datatype
package.
\end{abstract}

\tableofcontents

\input{Datatypes.tex}

\let\em=\sl
\bibliography{manual}{}
\bibliographystyle{abbrv}

\end{document}