| author | Fabian Huch <huch@in.tum.de> | 
| Thu, 14 Dec 2023 13:10:01 +0100 | |
| changeset 79289 | 7c1faa16554b | 
| parent 73511 | 2cdbb6a2f2a7 | 
| permissions | -rw-r--r-- | 
| 47269 | 1 | \usepackage{makeidx}         % allows index generation
 | 
| 2 | \usepackage{graphicx}        % standard LaTeX graphics tool
 | |
| 3 | % when including figure files | |
| 4 | \usepackage{multicol}        % used for the two-column index
 | |
| 5 | \usepackage[bottom]{footmisc}% places footnotes at page bottom
 | |
| 6 | \usepackage{alltt}
 | |
| 7 | ||
| 8 | \usepackage[T1]{fontenc}
 | |
| 73511 
2cdbb6a2f2a7
updated to latest latex due to new mechanism for dealing with bold ccfonts
 nipkow parents: 
58885diff
changeset | 9 | \usepackage[boldsans]{ccfonts}
 | 
| 
2cdbb6a2f2a7
updated to latest latex due to new mechanism for dealing with bold ccfonts
 nipkow parents: 
58885diff
changeset | 10 | \DeclareFontSeriesDefault[rm]{bf}{bx}%bf default for rm: bold extended
 | 
| 
2cdbb6a2f2a7
updated to latest latex due to new mechanism for dealing with bold ccfonts
 nipkow parents: 
58885diff
changeset | 11 | \DeclareFontSeriesDefault[sf]{bf}{sbc}%bf default for sf: semibold
 | 
| 47269 | 12 | \usepackage[euler-digits]{eulervm}
 | 
| 13 | ||
| 14 | \usepackage{isabelle,isabellesym}
 | |
| 15 | \usepackage{mathpartir}
 | |
| 16 | \usepackage{amssymb}
 | |
| 17 | ||
| 18 | \renewcommand*\descriptionlabel[1]{\hspace\labelsep \textbf{#1}\hfil}
 | |
| 19 | ||
| 20 | % this should be the last package used | |
| 51463 | 21 | \usepackage{xcolor}
 | 
| 47269 | 22 | \definecolor{linkcolor}{rgb}{0,0,0.4}
 | 
| 23 | \usepackage[colorlinks=true,linkcolor=linkcolor,citecolor=linkcolor, | |
| 24 | filecolor=linkcolor,pagecolor=linkcolor, | |
| 25 |             urlcolor=linkcolor]{hyperref}
 | |
| 26 | ||
| 27 | % urls in roman style, theory text in math-similar italics | |
| 28 | \urlstyle{tt}
 | |
| 29 | \isabellestyle{it}
 | |
| 30 | ||
| 31 | \renewcommand{\isadigit}[1]{\ensuremath{#1}}
 | |
| 32 | ||
| 33 | % font size | |
| 34 | \renewcommand{\isastyle}{\isastyleminor}
 | |
| 35 | ||
| 36 | % indexing | |
| 37 | \usepackage{ifthen}
 | |
| 38 | \newcommand{\indexdef}[3]%
 | |
| 39 | {\ifthenelse{\equal{}{#1}}{\index{#3 (#2)|bold}}{\index{#3 (#1\ #2)|bold}}}
 | |
| 40 | ||
| 41 | % section commands | |
| 42 | \renewcommand{\chapterautorefname}{Chapter}
 | |
| 43 | \renewcommand{\sectionautorefname}{Section}
 | |
| 51448 | 44 | \renewcommand{\subsectionautorefname}{Section}
 | 
| 47269 | 45 | |
| 46 | \renewcommand{\isamarkupsection}[1]{{\rmfamily\subsection{#1}}}
 | |
| 47 | \renewcommand{\isamarkupsubsection}[1]{{\rmfamily\subsubsection{#1}}}
 | |
| 48 | % isabelle in-text command font | |
| 49 | \newcommand{\isacom}[1]{\isa{\isacommand{#1}}}
 | |
| 49627 | 50 | |
| 51 | \protected\def\isacharunderscore{\raisebox{2pt}{\_\kern-1.7pt}}
 | |
| 52 | \protected\def\isacharunderscorekeyword{\raisebox{2pt}{\_}}
 | |
| 47269 | 53 | % isabelle keyword, adapted from isabelle.sty | 
| 54 | \renewcommand{\isakeyword}[1]
 | |
| 73511 
2cdbb6a2f2a7
updated to latest latex due to new mechanism for dealing with bold ccfonts
 nipkow parents: 
58885diff
changeset | 55 | {\emph{\sffamily\bfseries%
 | 
| 
2cdbb6a2f2a7
updated to latest latex due to new mechanism for dealing with bold ccfonts
 nipkow parents: 
58885diff
changeset | 56 | \def\isachardot{.}\def\isacharunderscore{\isacharunderscorekeyword}%
 | 
| 
2cdbb6a2f2a7
updated to latest latex due to new mechanism for dealing with bold ccfonts
 nipkow parents: 
58885diff
changeset | 57 | \def\isacharbraceleft{\{}\def\isacharbraceright{\}}#1}}
 | 
| 47269 | 58 | |
| 59 | % add \noindent to text blocks automatically | |
| 60 | \renewenvironment{isamarkuptext}{\par\isastyletext\begin{isapar}\noindent}{\end{isapar}}
 | |
| 61 | \renewenvironment{isamarkuptxt}{\par\isastyletext\begin{isapar}\noindent}{\end{isapar}}
 | |
| 62 | ||
| 49615 | 63 | \newcommand{\noquotes}[1]{{\renewcommand{\isachardoublequote}{}\renewcommand{\isachardoublequoteopen}{}\renewcommand{\isachardoublequoteclose}{}#1}}
 | 
| 47269 | 64 | \newcommand{\xsymbol}[1]{\texttt{\char`\\\char`<#1>}}
 | 
| 65 | ||
| 55317 | 66 | %index | 
| 67 | \newcommand{\conceptnoidx}[1]{\textbf{#1}}
 | |
| 68 | \newcommand{\concept}[1]{\conceptnoidx{#1}\index{#1}}
 | |
| 69 | \newcommand{\conceptidx}[2]{\conceptnoidx{#1}\index{#2}}
 | |
| 55319 | 70 | \newcommand{\indexed}[2]{#1\index{#2@\protect#1}}
 | 
| 55317 | 71 | |
| 47269 | 72 | \newcommand{\isabox}{\fbox}
 | 
| 73 | \newcommand{\bigisabox}[1]
 | |
| 74 | {\isabox{\renewcommand{\isanewline}{\\}%
 | |
| 75 |  \begin{tabular}{l}#1\end{tabular}}}
 | |
| 76 | ||
| 77 | %%%% ``WARNING'' environment: 2 ! characters separated by negative thin space | |
| 78 | %\def\warnbang{\vtop to 0pt{\vss\hbox{\let\bfdefault=\bfdefaultold\Huge\textbf{!$\!$!}}\vss}}
 | |
| 79 | ||
| 80 | \def\warnbang{\vtop to 0pt{\vss\hbox{\includegraphics[width=3ex, height=5.5ex]{bang}}\vss}}
 | |
| 81 | ||
| 82 | \newenvironment{warn}{\begin{trivlist}\small\item[]\noindent%
 | |
| 83 | \begingroup\hangindent=\parindent\hangafter=-2%\clubpenalty=10000% | |
| 84 |     \def\par{\endgraf\endgroup}%
 | |
| 85 |     \hbox to0pt{\hskip-\hangindent\warnbang\hfill}\ignorespaces}
 | |
| 86 |   {\par\end{trivlist}}
 | |
| 87 | ||
| 47302 | 88 | \chardef\isachardoublequote=`\"% | 
| 89 | \chardef\isachardoublequoteopen=`\"% | |
| 90 | \chardef\isachardoublequoteclose=`\"% | |
| 47269 | 91 | |
| 92 | \renewcommand{\isacharbackquoteopen}{\isacharbackquote}
 | |
| 93 | \renewcommand{\isacharbackquoteclose}{\isacharbackquote}
 | |
| 94 | ||
| 95 | \hyphenation{Isa-belle}
 |