src/Doc/Logics-ZF/document/root.tex
author haftmann
Sat, 05 Apr 2014 11:37:00 +0200
changeset 56420 b266e7a86485
parent 48985 src/Doc/ZF/document/root.tex@5386df44a037
permissions -rw-r--r--
closer correspondence of document and session names, while maintaining document names for external reference
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
8248
d7e85fd09291 a smaller point size reduces the number of overfull figures
paulson
parents: 7838
diff changeset
     1
\documentclass[11pt,a4paper]{report}
48956
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
     2
\usepackage{isabelle,isabellesym,railsetup}
48946
a9b8344f5196 more standard document preparation within session context;
wenzelm
parents: 42637
diff changeset
     3
\usepackage{graphicx,logics,ttbox,proof,latexsym}
48956
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
     4
\usepackage{isar}
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
     5
48946
a9b8344f5196 more standard document preparation within session context;
wenzelm
parents: 42637
diff changeset
     6
\usepackage{pdfsetup}   
14154
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
     7
%last package!
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
     8
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
     9
\remarkstrue 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    10
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    11
%%% to index derived rls: ^\([a-zA-Z0-9][a-zA-Z0-9_]*\)        \\tdx{\1}  
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    12
%%% to index rulenames:   ^ *(\([a-zA-Z0-9][a-zA-Z0-9_]*\),     \\tdx{\1}  
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    13
%%% to index constants:   \\tt \([a-zA-Z0-9][a-zA-Z0-9_]*\)     \\cdx{\1}  
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    14
%%% to deverbify:         \\verb|\([^|]*\)|     \\ttindex{\1}  
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    15
6579
d0c6bb2577b1 isabelle_zf image;
wenzelm
parents: 6121
diff changeset
    16
\title{\includegraphics[scale=0.5]{isabelle_zf} \\[4ex] 
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    17
       Isabelle's Logics: FOL and ZF}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    18
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    19
\author{{\em Lawrence C. Paulson}\\
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    20
        Computer Laboratory \\ University of Cambridge \\
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    21
        \texttt{lcp@cl.cam.ac.uk}\\[3ex] 
14154
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    22
        With Contributions by Tobias Nipkow and Markus Wenzel}
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    23
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    24
\newcommand\subcaption[1]{\par {\centering\normalsize\sc#1\par}\bigskip
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    25
  \hrule\bigskip}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    26
\newenvironment{constants}{\begin{center}\small\begin{tabular}{rrrr}}{\end{tabular}\end{center}}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    27
14154
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    28
\let\ts=\thinspace
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    29
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    30
\makeindex
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    31
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    32
\underscoreoff
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    33
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    34
\setcounter{secnumdepth}{2} \setcounter{tocdepth}{2}  %% {secnumdepth}{2}???
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    35
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    36
\pagestyle{headings}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    37
\sloppy
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    38
\binperiod     %%%treat . like a binary operator
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    39
48956
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    40
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    41
\isadroptag{theory}
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    42
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    43
\railtermfont{\isabellestyle{tt}}
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    44
\railnontermfont{\isabellestyle{literal}}
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    45
\railnamefont{\isabellestyle{literal}}
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    46
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    47
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    48
\begin{document}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    49
\maketitle 
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    50
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    51
\begin{abstract}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    52
This manual describes Isabelle's formalizations of many-sorted first-order
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    53
logic (\texttt{FOL}) and Zermelo-Fraenkel set theory (\texttt{ZF}).  See the
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    54
\emph{Reference Manual} for general Isabelle commands, and \emph{Introduction
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    55
  to Isabelle} for an overall tutorial.
14154
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    56
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    57
This manual is part of the earlier Isabelle documentation, 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    58
which is somewhat superseded by the Isabelle/HOL
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    59
\emph{Tutorial}~\cite{isa-tutorial}. However, the present document is the
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    60
only available documentation for Isabelle's versions of first-order logic
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    61
and set theory. Much of it is concerned with 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    62
the primitives for conducting proofs 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    63
using the ML top level.  It has been rewritten to use the Isar proof
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    64
language, but evidence of the old \ML{} orientation remains.
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    65
\end{abstract}
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    66
14154
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    67
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    68
\subsubsection*{Acknowledgements} 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    69
Markus Wenzel made numerous improvements.
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    70
    Philippe de Groote contributed to~ZF.  Philippe No\"el and
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    71
    Martin Coen made many contributions to~ZF.  The research has 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    72
    been funded by the EPSRC (grants GR/G53279, GR/H40570, GR/K57381,
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    73
    GR/K77051, GR/M75440) and by ESPRIT (projects 3245:
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    74
    Logical Frameworks, and 6453: Types) and by the DFG Schwerpunktprogramm
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    75
    \emph{Deduktion}.
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    76
    
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    77
\pagenumbering{roman} \tableofcontents \cleardoublepage
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    78
\pagenumbering{arabic} 
3bc0128e2c74 partial conversion to Isar format
paulson
parents: 9695
diff changeset
    79
\setcounter{page}{1} 
48946
a9b8344f5196 more standard document preparation within session context;
wenzelm
parents: 42637
diff changeset
    80
\input{syntax}
48970
8be091776e93 prefer \input which actually checks file existence;
wenzelm
parents: 48956
diff changeset
    81
\input{FOL}
8be091776e93 prefer \input which actually checks file existence;
wenzelm
parents: 48956
diff changeset
    82
\input{ZF}
48956
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    83
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    84
\isabellestyle{literal}
48970
8be091776e93 prefer \input which actually checks file existence;
wenzelm
parents: 48956
diff changeset
    85
\input{ZF_Isar}
48956
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    86
\isabellestyle{tt}
d54a3d39ba85 prefer doc-src/pdfsetup.sty;
wenzelm
parents: 48946
diff changeset
    87
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    88
\bibliographystyle{plain}
48946
a9b8344f5196 more standard document preparation within session context;
wenzelm
parents: 42637
diff changeset
    89
\bibliography{manual}
8828
5be2d1745c61 improved indexing;
wenzelm
parents: 8248
diff changeset
    90
\printindex
6121
5fe77b9b5185 the separate FOL and ZF logics manual, with new material on datatypes and
paulson
parents:
diff changeset
    91
\end{document}