| author | paulson | 
| Tue, 24 Feb 1998 11:35:33 +0100 | |
| changeset 4648 | f04da668581c | 
| parent 4244 | f50dace8be9f | 
| child 5752 | c3df312f34a2 | 
| permissions | -rw-r--r-- | 
| 293 | 1  | 
% iman.sty : Isabelle Manual Page Layout  | 
| 110 | 2  | 
%  | 
| 293 | 3  | 
\typeout{Document Style iman. Released 17 February 1994}
 | 
| 110 | 4  | 
|
| 293 | 5  | 
\hyphenation{Isa-belle man-u-script man-u-scripts ap-pen-dix mut-u-al-ly}
 | 
6  | 
\hyphenation{data-type data-types co-data-type co-data-types }
 | 
|
7  | 
||
8  | 
\let\ts=\thinspace  | 
|
| 110 | 9  | 
|
| 301 | 10  | 
%usage: \iflabelundefined{LABEL}{if not defined}{if defined}
 | 
11  | 
\newcommand{\iflabelundefined}[1]{\@ifundefined{r@#1}}
 | 
|
12  | 
||
13  | 
||
| 110 | 14  | 
%%%INDEXING use sedindex to process the index  | 
15  | 
%index, putting page numbers of definitions in boldface  | 
|
16  | 
\newcommand\bold[1]{{\bf#1}}
 | 
|
| 293 | 17  | 
\newcommand\fnote[1]{#1n}
 | 
| 110 | 18  | 
\newcommand\indexbold[1]{\index{#1|bold}}
 | 
19  | 
||
| 350 | 20  | 
%for indexing constants, symbols, theorems, ...  | 
21  | 
\newcommand\cdx[1]{{\tt#1}\index{#1@{\tt#1} constant}}
 | 
|
22  | 
\newcommand\sdx[1]{{\tt#1}\index{#1@{\tt#1} symbol}}
 | 
|
23  | 
||
24  | 
\newcommand\tdx[1]{{\tt#1}\index{#1@{\tt#1} theorem}}
 | 
|
25  | 
\newcommand\tdxbold[1]{{\tt#1}\index{#1@{\tt#1} theorem|bold}}
 | 
|
26  | 
||
27  | 
\newcommand\mltydx[1]{{\tt#1}\index{#1@{\tt#1} ML type}}
 | 
|
28  | 
\newcommand\xdx[1]{{\tt#1}\index{#1@{\tt#1} exception}}
 | 
|
29  | 
||
30  | 
\newcommand\ndx[1]{{\tt#1}\index{#1@{\tt#1} nonterminal}}
 | 
|
31  | 
\newcommand\ndxbold[1]{{\tt#1}\index{#1@{\tt#1} nonterminal|bold}}
 | 
|
32  | 
||
33  | 
\newcommand\cldx[1]{{\tt#1}\index{#1@{\tt#1} class}}
 | 
|
| 
3491
 
59ffc1c83403
Modified the \tydx command to set types in italics instead of \tt
 
paulson 
parents: 
3211 
diff
changeset
 | 
34  | 
\newcommand\tydx[1]{\textit{#1}\index{#1@{\textit{#1}} type}}
 | 
| 350 | 35  | 
\newcommand\thydx[1]{{\tt#1}\index{#1@{\tt#1} theory}}
 | 
36  | 
||
| 3187 | 37  | 
\newcommand\tooldx[1]{{\tt#1}\index{#1@{\tt#1} tool}}
 | 
| 3211 | 38  | 
\newcommand\settdx[1]{{\tt#1}\index{#1@{\tt#1} setting}}
 | 
| 3187 | 39  | 
|
| 110 | 40  | 
%for cross-references: 2nd argument (page number) is ignored  | 
41  | 
\newcommand\see[2]{{\it see \/}{#1}}
 | 
|
42  | 
\newcommand\seealso[2]{{\it see also \/}{#1}}
 | 
|
43  | 
||
| 3100 | 44  | 
%set argument in \tt font; at the same time, index using * prefix  | 
| 350 | 45  | 
\newcommand\rmindex[1]{{#1}\index{#1}\@}
 | 
| 110 | 46  | 
\newcommand\ttindex[1]{{\tt#1}\index{*#1}\@}
 | 
47  | 
\newcommand\ttindexbold[1]{{\tt#1}\index{*#1|bold}\@}
 | 
|
48  | 
||
49  | 
%set argument in \bf font and index in ROMAN font (for definitions in text!)  | 
|
50  | 
\newcommand\bfindex[1]{{\bf#1}\index{#1|bold}\@}
 | 
|
51  | 
||
52  | 
||
53  | 
%%% underscores as ordinary characters, not for subscripting  | 
|
54  | 
%% use @ or \sb for subscripting; use \at for @  | 
|
55  | 
%% only works in \tt font  | 
|
56  | 
%% must not make _ an active char; would make \ttindex fail!  | 
|
57  | 
\gdef\underscoreoff{\catcode`\@=8\catcode`\_=\other}
 | 
|
58  | 
\gdef\underscoreon{\catcode`\_=8\makeatother}
 | 
|
59  | 
\chardef\other=12  | 
|
60  | 
\chardef\at=`\@  | 
|
61  | 
||
62  | 
% alternative underscore  | 
|
63  | 
\def\_{\leavevmode\kern.06em\vbox{\hrule height.2ex width.3em}\hskip0.1em}
 | 
|
64  | 
||
65  | 
%%% \dquotes permits usage of "..." for \hbox{...} -- also taken from under.sty
 | 
|
66  | 
{\catcode`\"=\active
 | 
|
67  | 
\gdef\dquotes{\catcode`\"=\active  \let"=\@mathText}%
 | 
|
68  | 
\gdef\@mathText#1"{\hbox{\mathTextFont #1\/}}}
 | 
|
69  | 
\def\mathTextFont{\frenchspacing\tt}
 | 
|
70  | 
||
71  | 
%%%% meta-logical connectives  | 
|
72  | 
||
73  | 
\let\Forall=\bigwedge  | 
|
74  | 
\let\Imp=\Longrightarrow  | 
|
75  | 
\let\To=\Rightarrow  | 
|
76  | 
\newcommand\Var[1]{{?\!#1}}
 | 
|
77  | 
||
78  | 
%%%% ``WARNING'' environment  | 
|
79  | 
\def\dbend{\vtop to 0pt{\vss\hbox{\Huge\bf!}\vss}}
 | 
|
80  | 
\newenvironment{warn}{\medskip\medbreak\begingroup \clubpenalty=10000 
 | 
|
| 293 | 81  | 
\small %%WAS\baselineskip=0.9\baselineskip  | 
82  | 
\noindent \hangindent\parindent \hangafter=-2  | 
|
83  | 
         \hbox to0pt{\hskip-\hangindent\dbend\hfill}\ignorespaces}%
 | 
|
84  | 
        {\par\endgroup\medbreak}
 | 
|
| 110 | 85  | 
|
86  | 
||
87  | 
%%%% Standard logical symbols  | 
|
88  | 
\let\turn=\vdash  | 
|
89  | 
\let\conj=\wedge  | 
|
90  | 
\let\disj=\vee  | 
|
91  | 
\let\imp=\rightarrow  | 
|
92  | 
\let\bimp=\leftrightarrow  | 
|
| 293 | 93  | 
\newcommand\all[1]{\forall#1.}  %quantification
 | 
| 110 | 94  | 
\newcommand\ex[1]{\exists#1.}
 | 
95  | 
\newcommand{\pair}[1]{\langle#1\rangle}
 | 
|
96  | 
||
97  | 
\newcommand\lbrakk{\mathopen{[\![}}
 | 
|
98  | 
\newcommand\rbrakk{\mathclose{]\!]}}
 | 
|
99  | 
\newcommand\List[1]{\lbrakk#1\rbrakk}  %was \obj
 | 
|
100  | 
\newcommand\vpile[1]{\begin{array}{c}#1\end{array}}
 | 
|
101  | 
||
102  | 
\let\int=\cap  | 
|
103  | 
\let\un=\cup  | 
|
104  | 
\let\inter=\bigcap  | 
|
105  | 
\let\union=\bigcup  | 
|
106  | 
||
107  | 
\def\ML{{\sc ml}}
 | 
|
108  | 
\def\OBJ{{\sc obj}}
 | 
|
| 350 | 109  | 
\def\AST{{\sc ast}}
 | 
| 110 | 110  | 
|
| 3109 | 111  | 
\def\Pure{{\tt Pure}\@}
 | 
112  | 
\def\CPure{{\tt CPure}\@}
 | 
|
| 110 | 113  | 
\def\LCF{{\tt LCF}\@}
 | 
114  | 
\def\FOL{{\tt FOL}\@}
 | 
|
115  | 
\def\HOL{{\tt HOL}\@}
 | 
|
| 1648 | 116  | 
\def\HOLCF{{\tt HOLCF}\@}
 | 
| 110 | 117  | 
\def\LK{{\tt LK}\@}
 | 
118  | 
\def\ZF{{\tt ZF}\@}
 | 
|
119  | 
\def\CTT{{\tt CTT}\@}
 | 
|
| 3109 | 120  | 
\def\Cube{{\tt Cube}\@}
 | 
121  | 
\def\Modal{{\tt Modal}\@}
 | 
|
| 110 | 122  | 
|
123  | 
%macros to change the treatment of symbols  | 
|
124  | 
\def\relsemicolon{\mathcode`\;="303B}   %treat ; like a relation
 | 
|
125  | 
\def\binperiod{\mathcode`\.="213A}   %treat . like a binary operator
 | 
|
126  | 
\def\binvert{\mathcode`\|="226A}     %treat | like a binary operator
 | 
|
127  | 
||
128  | 
%redefinition of \sloppy and \fussy to use \emergencystretch  | 
|
129  | 
\def\sloppy{\tolerance2000 \hfuzz.5pt \vfuzz.5pt \emergencystretch=15pt}
 | 
|
130  | 
\def\fussy{\tolerance200 \hfuzz.1pt \vfuzz.1pt \emergencystretch=0pt}
 | 
|
131  | 
||
| 350 | 132  | 
%%%% \tt things  | 
133  | 
||
134  | 
\def\ttdescriptionlabel#1{\hspace\labelsep \tt #1}
 | 
|
135  | 
\def\ttdescription{\list{}{\labelwidth\z@ \itemindent-\leftmargin
 | 
|
136  | 
\let\makelabel\ttdescriptionlabel}}  | 
|
137  | 
||
138  | 
\let\endttdescription\endlist  | 
|
139  | 
||
| 293 | 140  | 
\chardef\ttilde=`\~ % A tilde for \tt font  | 
141  | 
\chardef\ttback=`\\ % A backslash for \tt font  | 
|
142  | 
\chardef\ttlbrace=`\{   % A left brace for \tt font
 | 
|
143  | 
\chardef\ttrbrace=`\} % A right brace for \tt font  | 
|
| 110 | 144  | 
|
| 4244 | 145  | 
\newcommand\out{\ \ttfamily\slshape}   %% for output from terminal sessions
 | 
| 110 | 146  | 
|
147  | 
% The mathcodes for the letters A, ..., Z, a, ..., z are changed to  | 
|
| 
140
 
3a8c68d1d466
changed itmath trickery to be compatible with NFSS (itmath.sty)
 
nipkow 
parents: 
110 
diff
changeset
 | 
148  | 
% generate text italic rather than math italic by default. This makes  | 
| 110 | 149  | 
% multi-letter identifiers look better. The mathcode for character c  | 
| 3096 | 150  | 
% is set to |"7000| (variable family) + |"400| (text italic) + |c|.  | 
| 
140
 
3a8c68d1d466
changed itmath trickery to be compatible with NFSS (itmath.sty)
 
nipkow 
parents: 
110 
diff
changeset
 | 
151  | 
%  | 
| 3096 | 152  | 
\DeclareSymbolFont{italics}{\encodingdefault}{\rmdefault}{m}{it}%
 | 
| 110 | 153  | 
\def\@setmcodes#1#2#3{{\count0=#1 \count1=#3
 | 
| 
140
 
3a8c68d1d466
changed itmath trickery to be compatible with NFSS (itmath.sty)
 
nipkow 
parents: 
110 
diff
changeset
 | 
154  | 
\loop \global\mathcode\count0=\count1 \ifnum \count0<#2  | 
| 
 
3a8c68d1d466
changed itmath trickery to be compatible with NFSS (itmath.sty)
 
nipkow 
parents: 
110 
diff
changeset
 | 
155  | 
\advance\count0 by1 \advance\count1 by1 \repeat}}  | 
| 3096 | 156  | 
\@setmcodes{`A}{`Z}{"7\hexnumber@\symitalics41}
 | 
157  | 
\@setmcodes{`a}{`z}{"7\hexnumber@\symitalics61}
 |