lcp@293: % iman.sty : Isabelle Manual Page Layout lcp@110: % lcp@293: \typeout{Document Style iman. Released 17 February 1994} lcp@110: lcp@293: \hyphenation{Isa-belle man-u-script man-u-scripts ap-pen-dix mut-u-al-ly} lcp@293: \hyphenation{data-type data-types co-data-type co-data-types } lcp@293: lcp@293: \let\ts=\thinspace lcp@110: lcp@301: %usage: \iflabelundefined{LABEL}{if not defined}{if defined} lcp@301: \newcommand{\iflabelundefined}[1]{\@ifundefined{r@#1}} lcp@301: lcp@301: lcp@110: %%%INDEXING use sedindex to process the index wenzelm@8827: paulson@10092: \newcommand\seealso[2]{\emph{see also} #1} wenzelm@8827: \usepackage{makeidx} wenzelm@8827: lcp@110: %index, putting page numbers of definitions in boldface wenzelm@6747: \def\bold#1{\textbf{#1}} lcp@293: \newcommand\fnote[1]{#1n} lcp@110: \newcommand\indexbold[1]{\index{#1|bold}} lcp@110: lcp@350: %for indexing constants, symbols, theorems, ... lcp@350: \newcommand\cdx[1]{{\tt#1}\index{#1@{\tt#1} constant}} lcp@350: \newcommand\sdx[1]{{\tt#1}\index{#1@{\tt#1} symbol}} lcp@350: lcp@350: \newcommand\tdx[1]{{\tt#1}\index{#1@{\tt#1} theorem}} lcp@350: \newcommand\tdxbold[1]{{\tt#1}\index{#1@{\tt#1} theorem|bold}} lcp@350: lcp@350: \newcommand\mltydx[1]{{\tt#1}\index{#1@{\tt#1} ML type}} lcp@350: \newcommand\xdx[1]{{\tt#1}\index{#1@{\tt#1} exception}} lcp@350: lcp@350: \newcommand\ndx[1]{{\tt#1}\index{#1@{\tt#1} nonterminal}} lcp@350: \newcommand\ndxbold[1]{{\tt#1}\index{#1@{\tt#1} nonterminal|bold}} lcp@350: lcp@350: \newcommand\cldx[1]{{\tt#1}\index{#1@{\tt#1} class}} paulson@3491: \newcommand\tydx[1]{\textit{#1}\index{#1@{\textit{#1}} type}} lcp@350: \newcommand\thydx[1]{{\tt#1}\index{#1@{\tt#1} theory}} lcp@350: wenzelm@3187: \newcommand\tooldx[1]{{\tt#1}\index{#1@{\tt#1} tool}} wenzelm@3211: \newcommand\settdx[1]{{\tt#1}\index{#1@{\tt#1} setting}} wenzelm@3187: wenzelm@3100: %set argument in \tt font; at the same time, index using * prefix lcp@350: \newcommand\rmindex[1]{{#1}\index{#1}\@} lcp@110: \newcommand\ttindex[1]{{\tt#1}\index{*#1}\@} lcp@110: \newcommand\ttindexbold[1]{{\tt#1}\index{*#1|bold}\@} lcp@110: lcp@110: %set argument in \bf font and index in ROMAN font (for definitions in text!) lcp@110: \newcommand\bfindex[1]{{\bf#1}\index{#1|bold}\@} lcp@110: lcp@110: lcp@110: %%% underscores as ordinary characters, not for subscripting lcp@110: %% use @ or \sb for subscripting; use \at for @ lcp@110: %% only works in \tt font lcp@110: %% must not make _ an active char; would make \ttindex fail! lcp@110: \gdef\underscoreoff{\catcode`\@=8\catcode`\_=\other} lcp@110: \gdef\underscoreon{\catcode`\_=8\makeatother} lcp@110: \chardef\other=12 lcp@110: \chardef\at=`\@ lcp@110: lcp@110: % alternative underscore lcp@110: \def\_{\leavevmode\kern.06em\vbox{\hrule height.2ex width.3em}\hskip0.1em} lcp@110: lcp@110: %%% \dquotes permits usage of "..." for \hbox{...} -- also taken from under.sty lcp@110: {\catcode`\"=\active lcp@110: \gdef\dquotes{\catcode`\"=\active \let"=\@mathText}% lcp@110: \gdef\@mathText#1"{\hbox{\mathTextFont #1\/}}} lcp@110: \def\mathTextFont{\frenchspacing\tt} paulson@6123: \def\dquotesoff{\catcode`\"=\other} lcp@110: lcp@110: %%%% meta-logical connectives lcp@110: lcp@110: \let\Forall=\bigwedge lcp@110: \let\Imp=\Longrightarrow lcp@110: \let\To=\Rightarrow wenzelm@7455: \newcommand{\PROP}{\mathop{\mathrm{PROP}}} wenzelm@7455: \newcommand{\Var}[1]{{?\!#1}} wenzelm@7455: \newcommand{\All}[1]{\Forall#1.} %quantification lcp@110: lcp@110: %%%% ``WARNING'' environment lcp@110: \def\dbend{\vtop to 0pt{\vss\hbox{\Huge\bf!}\vss}} lcp@110: \newenvironment{warn}{\medskip\medbreak\begingroup \clubpenalty=10000 lcp@293: \small %%WAS\baselineskip=0.9\baselineskip wenzelm@39860: \noindent \ifdim\parindent > 0pt\hangindent\parindent\else\hangindent1.5em\fi wenzelm@39860: \hangafter=-2 lcp@293: \hbox to0pt{\hskip-\hangindent\dbend\hfill}\ignorespaces}% lcp@293: {\par\endgroup\medbreak} lcp@110: lcp@110: lcp@110: %%%% Standard logical symbols lcp@110: \let\turn=\vdash lcp@110: \let\conj=\wedge lcp@110: \let\disj=\vee lcp@110: \let\imp=\rightarrow lcp@110: \let\bimp=\leftrightarrow lcp@293: \newcommand\all[1]{\forall#1.} %quantification lcp@110: \newcommand\ex[1]{\exists#1.} lcp@110: \newcommand{\pair}[1]{\langle#1\rangle} lcp@110: wenzelm@5752: \newcommand{\lparr}{\mathopen{(\!|}} wenzelm@5752: \newcommand{\rparr}{\mathclose{|\!)}} wenzelm@5752: \newcommand{\fs}{\mathpunct{,\,}} wenzelm@5752: \newcommand{\ty}{\mathrel{::}} wenzelm@5752: \newcommand{\asn}{\mathrel{:=}} wenzelm@5752: \newcommand{\more}{\ldots} wenzelm@5752: \newcommand{\record}[1]{\lparr #1 \rparr} wenzelm@5765: \newcommand{\dtt}{\mathord.} wenzelm@5752: lcp@110: \newcommand\lbrakk{\mathopen{[\![}} lcp@110: \newcommand\rbrakk{\mathclose{]\!]}} lcp@110: \newcommand\List[1]{\lbrakk#1\rbrakk} %was \obj lcp@110: \newcommand\vpile[1]{\begin{array}{c}#1\end{array}} wenzelm@5752: \newenvironment{matharray}[1]{\[\begin{array}{#1}}{\end{array}\]} wenzelm@9693: \newcommand{\Text}[1]{\mbox{#1}} lcp@110: wenzelm@7976: \DeclareMathSymbol{\dshsym}{\mathalpha}{letters}{"2D} wenzelm@7976: \newcommand{\dsh}{\mathit{\dshsym}} wenzelm@7976: lcp@110: \let\int=\cap lcp@110: \let\un=\cup lcp@110: \let\inter=\bigcap lcp@110: \let\union=\bigcup lcp@110: lcp@110: \def\ML{{\sc ml}} lcp@110: \def\OBJ{{\sc obj}} lcp@350: \def\AST{{\sc ast}} lcp@110: lcp@110: %macros to change the treatment of symbols lcp@110: \def\relsemicolon{\mathcode`\;="303B} %treat ; like a relation lcp@110: \def\binperiod{\mathcode`\.="213A} %treat . like a binary operator lcp@110: \def\binvert{\mathcode`\|="226A} %treat | like a binary operator lcp@110: lcp@110: %redefinition of \sloppy and \fussy to use \emergencystretch lcp@110: \def\sloppy{\tolerance2000 \hfuzz.5pt \vfuzz.5pt \emergencystretch=15pt} lcp@110: \def\fussy{\tolerance200 \hfuzz.1pt \vfuzz.1pt \emergencystretch=0pt} lcp@110: wenzelm@7169: %non-bf version of description wenzelm@7169: \def\descrlabel#1{\hspace\labelsep #1} wenzelm@7169: \def\descr{\list{}{\labelwidth\z@ \itemindent-\leftmargin\let\makelabel\descrlabel}} wenzelm@7169: \let\enddescr\endlist wenzelm@7169: lcp@110: % The mathcodes for the letters A, ..., Z, a, ..., z are changed to nipkow@140: % generate text italic rather than math italic by default. This makes lcp@110: % multi-letter identifiers look better. The mathcode for character c berghofe@3096: % is set to |"7000| (variable family) + |"400| (text italic) + |c|. nipkow@140: % berghofe@3096: \DeclareSymbolFont{italics}{\encodingdefault}{\rmdefault}{m}{it}% lcp@110: \def\@setmcodes#1#2#3{{\count0=#1 \count1=#3 nipkow@140: \loop \global\mathcode\count0=\count1 \ifnum \count0<#2 nipkow@140: \advance\count0 by1 \advance\count1 by1 \repeat}} berghofe@3096: \@setmcodes{`A}{`Z}{"7\hexnumber@\symitalics41} berghofe@3096: \@setmcodes{`a}{`z}{"7\hexnumber@\symitalics61}