doc-src/AxClass/generated/isabelle.sty
author wenzelm
Mon, 21 Aug 2000 13:47:24 +0200
changeset 9665 2a6d7f1409f9
parent 8890 9a44d8d98731
child 9672 2c208c98f541
permissions -rw-r--r--
updated;

%%
%% $Id$
%%
%% macros for Isabelle generated LaTeX output
%%

%%% Simple document preparation (based on theory token language)

% isabelle environments

\newcommand{\isastyle}{\small\tt\slshape}
\newcommand{\isastyletext}{\normalsize\rm}
\newcommand{\isastyletxt}{\rm}
\newcommand{\isastylecmt}{\rm}

\newdimen\isa@parindent\newdimen\isa@parskip

\newenvironment{isabelle}{%
\isa@parindent\parindent\parindent0pt%
\isa@parskip\parskip\parskip0pt%
\isastyle}{}

\newcommand{\isa}[1]{\emph{\isastyle #1}}

\newcommand{\isanewline}{\mbox{}\\\mbox{}}

\chardef\isacharhash=`\#
\chardef\isachardollar=`\$
\chardef\isacharpercent=`\%
\chardef\isacharampersand=`\&
\chardef\isacharprime=`\'
\chardef\isacharparenleft=`\(
\chardef\isacharparenright=`\)
\chardef\isacharasterisk=`\*
\chardef\isacharminus=`\-
\chardef\isacharless=`\<
\chardef\isachargreater=`\>
\chardef\isacharbrackleft=`\[
\chardef\isachardoublequote=`\"
\chardef\isacharbackslash=`\\
\chardef\isacharbrackright=`\]
\chardef\isacharcircum=`\^
\chardef\isacharunderscore=`\_
\chardef\isacharbraceleft=`\{
\chardef\isacharbar=`\|
\chardef\isacharbraceright=`\}
\chardef\isachartilde=`\~


% keyword and section markup

\newcommand{\isacommand}[1]{\emph{\bf #1}}
\newcommand{\isakeyword}[1]{\emph{\bf #1}}
\newcommand{\isabeginblock}{\isakeyword{\{}}
\newcommand{\isaendblock}{\isakeyword{\}}}

\newcommand{\isamarkupheader}[1]{\section{#1}}
\newcommand{\isamarkupchapter}[1]{\chapter{#1}}
\newcommand{\isamarkupsection}[1]{\section{#1}}
\newcommand{\isamarkupsubsection}[1]{\subsection{#1}}
\newcommand{\isamarkupsubsubsection}[1]{\subsubsection{#1}}
\newcommand{\isamarkupsect}[1]{\section{#1}}
\newcommand{\isamarkupsubsect}[1]{\subsection{#1}}
\newcommand{\isamarkupsubsubsect}[1]{\subsubsection{#1}}

\newenvironment{isapar}{\parindent\isa@parindent\parskip\isa@parskip\par\medskip}{\par\smallskip}
\newenvironment{isamarkuptext}{\isastyletext\begin{isapar}}{\end{isapar}}
\newenvironment{isamarkuptxt}{\isastyletxt\begin{isapar}}{\end{isapar}}
\newcommand{\isamarkupcmt}[1]{{\isastylecmt--- #1}}


% alternative styles -- default is "tt"

\newcommand{\isabellestyle}{}
\def\isabellestyle#1{\csname isasetup#1\endcsname}

\newcommand{\isasetupit}{%
\renewcommand{\isastyle}{\small\itshape}%
\renewcommand{\isastyletext}{\normalsize\rm}%
\renewcommand{\isastyletxt}{\rm}%
\renewcommand{\isastylecmt}{\rm}%
\renewcommand{\isachardollar}{\textsl{\$}}%
\renewcommand{\isacharampersand}{\textsl{\&}}%
\renewcommand{\isacharprime}{$'$}%
\renewcommand{\isacharparenleft}{\emph{$($}}%
\renewcommand{\isacharparenright}{\emph{$)$}}%
\renewcommand{\isacharasterisk}{\emph{$*$}}%
\renewcommand{\isacharminus}{\emph{$-$}}%
\renewcommand{\isacharless}{\emph{$<$}}%
\renewcommand{\isachargreater}{\emph{$>$}}%
\renewcommand{\isachardoublequote}{}%
\renewcommand{\isacharbrackleft}{\emph{$[$}}%
\renewcommand{\isacharbrackright}{\emph{$]$}}%
\renewcommand{\isacharunderscore}{-}%
\renewcommand{\isacharbraceleft}{\emph{$\{$}}%
\renewcommand{\isacharbar}{\emph{$\mid$}}%
\renewcommand{\isacharbraceright}{\emph{$\}$}}%
}

\newcommand{\isasetupsl}{\isasetupit\renewcommand{\isastyle}{\small\slshape}}