src/Doc/Classes/document/style.sty
author wenzelm
Fri, 25 Apr 2014 14:18:13 +0200
changeset 56720 e1317a26f8c0
parent 48985 5386df44a037
child 69660 2bc2a8599369
permissions -rw-r--r--
updated properties for scala.concurrent.ExecutionContext.Implicits.global (future task farm), similar to Isabelle/ML; removed obsolete properties for old actors;


%% toc
\newcommand{\tocentry}[1]{\cleardoublepage\phantomsection\addcontentsline{toc}{chapter}{#1}
\@mkboth{\MakeUppercase{#1}}{\MakeUppercase{#1}}}

%% paragraphs
\setlength{\parindent}{1em}

%% references
\newcommand{\secref}[1]{\S\ref{#1}}
\newcommand{\figref}[1]{figure~\ref{#1}}

%% logical markup
\newcommand{\strong}[1]{{\bfseries {#1}}}
\newcommand{\qn}[1]{\emph{#1}}

%% typographic conventions
\newcommand{\qt}[1]{``{#1}''}
\newcommand{\ditem}[1]{\item[\isastyletext #1]}

%% quote environment
\isakeeptag{quote}
\renewenvironment{quote}
  {\list{}{\leftmargin2em\rightmargin0pt}\parindent0pt\parskip0pt\item\relax}
  {\endlist}
\renewcommand{\isatagquote}{\begin{quote}}
\renewcommand{\endisatagquote}{\end{quote}}
\newcommand{\quotebreak}{\\[1.2ex]}

%% typewriter text
\newenvironment{typewriter}{\renewcommand{\isastyletext}{}%
\renewcommand{\isadigit}[1]{{##1}}%
\parindent0pt%
\makeatletter\isa@parindent0pt\makeatother%
\isabellestyle{tt}\isastyle%
\fontsize{9pt}{9pt}\selectfont}{}

\isakeeptag{quotetypewriter}
\renewcommand{\isatagquotetypewriter}{\begin{quote}\begin{typewriter}}
\renewcommand{\endisatagquotetypewriter}{\end{typewriter}\end{quote}}

%% presentation
\setcounter{secnumdepth}{2} \setcounter{tocdepth}{2}

%% character detail
\renewcommand{\isadigit}[1]{\isamath{#1}}
\binperiod
\underscoreoff

%% format
\pagestyle{headings}
\isabellestyle{it}


%%% Local Variables: 
%%% mode: latex
%%% TeX-master: "implementation"
%%% End: