author | wenzelm |
Tue, 15 Aug 2017 12:11:25 +0200 | |
changeset 66432 | 3a78bbfe9cf3 |
parent 63680 | 6e1e8b5abbfa |
child 67139 | 8fe0aba577af |
permissions | -rw-r--r-- |
61656 | 1 |
(*:maxLineLen=78:*) |
2 |
||
27043 | 3 |
theory Document_Preparation |
63531 | 4 |
imports Main Base |
27043 | 5 |
begin |
6 |
||
58618 | 7 |
chapter \<open>Document preparation \label{ch:document-prep}\<close> |
27043 | 8 |
|
61624 | 9 |
text \<open> |
10 |
Isabelle/Isar provides a simple document preparation system based on |
|
11 |
{PDF-\LaTeX}, with support for hyperlinks and bookmarks within that format. |
|
12 |
This allows to produce papers, books, theses etc.\ from Isabelle theory |
|
13 |
sources. |
|
27043 | 14 |
|
61624 | 15 |
{\LaTeX} output is generated while processing a \<^emph>\<open>session\<close> in batch mode, as |
16 |
explained in the \<^emph>\<open>The Isabelle System Manual\<close> @{cite "isabelle-system"}. |
|
17 |
The main Isabelle tools to get started with document preparation are |
|
18 |
@{tool_ref mkroot} and @{tool_ref build}. |
|
27043 | 19 |
|
61624 | 20 |
The classic Isabelle/HOL tutorial @{cite "isabelle-hol-book"} also explains |
21 |
some aspects of theory presentation. |
|
22 |
\<close> |
|
27043 | 23 |
|
24 |
||
58618 | 25 |
section \<open>Markup commands \label{sec:markup}\<close> |
27043 | 26 |
|
58618 | 27 |
text \<open> |
27043 | 28 |
\begin{matharray}{rcl} |
61493 | 29 |
@{command_def "chapter"} & : & \<open>any \<rightarrow> any\<close> \\ |
30 |
@{command_def "section"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
31 |
@{command_def "subsection"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
32 |
@{command_def "subsubsection"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
33 |
@{command_def "paragraph"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
34 |
@{command_def "subparagraph"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
35 |
@{command_def "text"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
36 |
@{command_def "txt"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
37 |
@{command_def "text_raw"} & : & \<open>any \<rightarrow> any\<close> \\ |
|
27043 | 38 |
\end{matharray} |
39 |
||
61624 | 40 |
Markup commands provide a structured way to insert text into the document |
41 |
generated from a theory. Each markup command takes a single @{syntax text} |
|
42 |
argument, which is passed as argument to a corresponding {\LaTeX} macro. The |
|
63680 | 43 |
default macros provided by \<^file>\<open>~~/lib/texinputs/isabelle.sty\<close> can be |
61624 | 44 |
redefined according to the needs of the underlying document and {\LaTeX} |
45 |
styles. |
|
28747 | 46 |
|
61624 | 47 |
Note that formal comments (\secref{sec:comments}) are similar to markup |
48 |
commands, but have a different status within Isabelle/Isar syntax. |
|
27043 | 49 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
50 |
@{rail \<open> |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
51 |
(@@{command chapter} | @@{command section} | @@{command subsection} | |
62912 | 52 |
@@{command subsubsection} | @@{command paragraph} | @@{command subparagraph}) |
53 |
@{syntax text} ';'? | |
|
54 |
(@@{command text} | @@{command txt} | @@{command text_raw}) @{syntax text} |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
55 |
\<close>} |
27043 | 56 |
|
61624 | 57 |
\<^descr> @{command chapter}, @{command section}, @{command subsection} etc.\ mark |
58 |
section headings within the theory source. This works in any context, even |
|
59 |
before the initial @{command theory} command. The corresponding {\LaTeX} |
|
60 |
macros are \<^verbatim>\<open>\isamarkupchapter\<close>, \<^verbatim>\<open>\isamarkupsection\<close>, |
|
61 |
\<^verbatim>\<open>\isamarkupsubsection\<close> etc.\ |
|
27043 | 62 |
|
61624 | 63 |
\<^descr> @{command text} and @{command txt} specify paragraphs of plain text. |
64 |
This corresponds to a {\LaTeX} environment \<^verbatim>\<open>\begin{isamarkuptext}\<close> \<open>\<dots>\<close> |
|
65 |
\<^verbatim>\<open>\end{isamarkuptext}\<close> etc. |
|
27043 | 66 |
|
61624 | 67 |
\<^descr> @{command text_raw} is similar to @{command text}, but without any |
68 |
surrounding markup environment. This allows to inject arbitrary {\LaTeX} |
|
69 |
source into the generated document. |
|
27043 | 70 |
|
61463 | 71 |
All text passed to any of the above markup commands may refer to formal |
61624 | 72 |
entities via \<^emph>\<open>document antiquotations\<close>, see also \secref{sec:antiq}. These |
73 |
are interpreted in the present theory or proof context. |
|
27043 | 74 |
|
61421 | 75 |
\<^medskip> |
61624 | 76 |
The proof markup commands closely resemble those for theory specifications, |
77 |
but have a different formal status and produce different {\LaTeX} macros. |
|
58618 | 78 |
\<close> |
27043 | 79 |
|
80 |
||
60286 | 81 |
section \<open>Document antiquotations \label{sec:antiq}\<close> |
27043 | 82 |
|
58618 | 83 |
text \<open> |
27043 | 84 |
\begin{matharray}{rcl} |
61493 | 85 |
@{antiquotation_def "theory"} & : & \<open>antiquotation\<close> \\ |
86 |
@{antiquotation_def "thm"} & : & \<open>antiquotation\<close> \\ |
|
87 |
@{antiquotation_def "lemma"} & : & \<open>antiquotation\<close> \\ |
|
88 |
@{antiquotation_def "prop"} & : & \<open>antiquotation\<close> \\ |
|
89 |
@{antiquotation_def "term"} & : & \<open>antiquotation\<close> \\ |
|
90 |
@{antiquotation_def term_type} & : & \<open>antiquotation\<close> \\ |
|
91 |
@{antiquotation_def typeof} & : & \<open>antiquotation\<close> \\ |
|
92 |
@{antiquotation_def const} & : & \<open>antiquotation\<close> \\ |
|
93 |
@{antiquotation_def abbrev} & : & \<open>antiquotation\<close> \\ |
|
94 |
@{antiquotation_def typ} & : & \<open>antiquotation\<close> \\ |
|
95 |
@{antiquotation_def type} & : & \<open>antiquotation\<close> \\ |
|
96 |
@{antiquotation_def class} & : & \<open>antiquotation\<close> \\ |
|
97 |
@{antiquotation_def "text"} & : & \<open>antiquotation\<close> \\ |
|
98 |
@{antiquotation_def goals} & : & \<open>antiquotation\<close> \\ |
|
99 |
@{antiquotation_def subgoals} & : & \<open>antiquotation\<close> \\ |
|
100 |
@{antiquotation_def prf} & : & \<open>antiquotation\<close> \\ |
|
101 |
@{antiquotation_def full_prf} & : & \<open>antiquotation\<close> \\ |
|
102 |
@{antiquotation_def ML} & : & \<open>antiquotation\<close> \\ |
|
103 |
@{antiquotation_def ML_op} & : & \<open>antiquotation\<close> \\ |
|
104 |
@{antiquotation_def ML_type} & : & \<open>antiquotation\<close> \\ |
|
105 |
@{antiquotation_def ML_structure} & : & \<open>antiquotation\<close> \\ |
|
106 |
@{antiquotation_def ML_functor} & : & \<open>antiquotation\<close> \\ |
|
107 |
@{antiquotation_def emph} & : & \<open>antiquotation\<close> \\ |
|
108 |
@{antiquotation_def bold} & : & \<open>antiquotation\<close> \\ |
|
109 |
@{antiquotation_def verbatim} & : & \<open>antiquotation\<close> \\ |
|
110 |
@{antiquotation_def "file"} & : & \<open>antiquotation\<close> \\ |
|
111 |
@{antiquotation_def "url"} & : & \<open>antiquotation\<close> \\ |
|
112 |
@{antiquotation_def "cite"} & : & \<open>antiquotation\<close> \\ |
|
61494 | 113 |
@{command_def "print_antiquotations"}\<open>\<^sup>*\<close> & : & \<open>context \<rightarrow>\<close> \\ |
27043 | 114 |
\end{matharray} |
115 |
||
61614 | 116 |
The overall content of an Isabelle/Isar theory may alternate between formal |
117 |
and informal text. The main body consists of formal specification and proof |
|
118 |
commands, interspersed with markup commands (\secref{sec:markup}) or |
|
119 |
document comments (\secref{sec:comments}). The argument of markup commands |
|
120 |
quotes informal text to be printed in the resulting document, but may again |
|
121 |
refer to formal entities via \<^emph>\<open>document antiquotations\<close>. |
|
27043 | 122 |
|
61503 | 123 |
For example, embedding \<^verbatim>\<open>@{term [show_types] "f x = a + x"}\<close> |
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
124 |
within a text block makes |
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
125 |
\isa{{\isacharparenleft}f{\isasymColon}{\isacharprime}a\ {\isasymRightarrow}\ {\isacharprime}a{\isacharparenright}\ {\isacharparenleft}x{\isasymColon}{\isacharprime}a{\isacharparenright}\ {\isacharequal}\ {\isacharparenleft}a{\isasymColon}{\isacharprime}a{\isacharparenright}\ {\isacharplus}\ x} appear in the final {\LaTeX} document. |
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
126 |
|
61614 | 127 |
Antiquotations usually spare the author tedious typing of logical entities |
128 |
in full detail. Even more importantly, some degree of consistency-checking |
|
129 |
between the main body of formal text and its informal explanation is |
|
130 |
achieved, since terms and types appearing in antiquotations are checked |
|
131 |
within the current theory or proof context. |
|
27043 | 132 |
|
61614 | 133 |
\<^medskip> |
134 |
Antiquotations are in general written as |
|
135 |
\<^verbatim>\<open>@{\<close>\<open>name\<close>~\<^verbatim>\<open>[\<close>\<open>options\<close>\<^verbatim>\<open>]\<close>~\<open>arguments\<close>\<^verbatim>\<open>}\<close>. The short form |
|
136 |
\<^verbatim>\<open>\\<close>\<^verbatim>\<open><^\<close>\<open>name\<close>\<^verbatim>\<open>>\<close>\<open>\<open>argument_content\<close>\<close> (without surrounding \<^verbatim>\<open>@{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>) |
|
137 |
works for a single argument that is a cartouche. A cartouche without special |
|
138 |
decoration is equivalent to \<^verbatim>\<open>\<^cartouche>\<close>\<open>\<open>argument_content\<close>\<close>, which is |
|
139 |
equivalent to \<^verbatim>\<open>@{cartouche\<close>~\<open>\<open>argument_content\<close>\<close>\<^verbatim>\<open>}\<close>. The special name |
|
61595 | 140 |
@{antiquotation_def cartouche} is defined in the context: Isabelle/Pure |
141 |
introduces that as an alias to @{antiquotation_ref text} (see below). |
|
142 |
Consequently, \<open>\<open>foo_bar + baz \<le> bazar\<close>\<close> prints literal quasi-formal text |
|
61614 | 143 |
(unchecked). A control symbol \<^verbatim>\<open>\\<close>\<^verbatim>\<open><^\<close>\<open>name\<close>\<^verbatim>\<open>>\<close> within the body text, but |
144 |
without a subsequent cartouche, is equivalent to \<^verbatim>\<open>@{\<close>\<open>name\<close>\<^verbatim>\<open>}\<close>. |
|
61472 | 145 |
|
61474 | 146 |
\begingroup |
147 |
\def\isasymcontrolstart{\isatt{\isacharbackslash\isacharless\isacharcircum}} |
|
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59783
diff
changeset
|
148 |
@{rail \<open> |
61472 | 149 |
@{syntax_def antiquotation}: |
61474 | 150 |
'@{' antiquotation_body '}' | |
61491
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
151 |
'\<controlstart>' @{syntax_ref name} '>' @{syntax_ref cartouche} | |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
152 |
@{syntax_ref cartouche} |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
153 |
; |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
154 |
options: '[' (option * ',') ']' |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
155 |
; |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
156 |
option: @{syntax name} | @{syntax name} '=' @{syntax name} |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
157 |
; |
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59783
diff
changeset
|
158 |
\<close>} |
61474 | 159 |
\endgroup |
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59783
diff
changeset
|
160 |
|
61614 | 161 |
Note that the syntax of antiquotations may \<^emph>\<open>not\<close> include source comments |
162 |
\<^verbatim>\<open>(*\<close>~\<open>\<dots>\<close>~\<^verbatim>\<open>*)\<close> nor verbatim text \<^verbatim>\<open>{*\<close>~\<open>\<dots>\<close>~\<^verbatim>\<open>*}\<close>. |
|
61491
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
163 |
|
43618 | 164 |
%% FIXME less monolithic presentation, move to individual sections!? |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
165 |
@{rail \<open> |
61472 | 166 |
@{syntax_def antiquotation_body}: |
61614 | 167 |
(@@{antiquotation text} | @@{antiquotation cartouche} | @@{antiquotation theory_text}) |
168 |
options @{syntax text} | |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
169 |
@@{antiquotation theory} options @{syntax name} | |
62969 | 170 |
@@{antiquotation thm} options styles @{syntax thms} | |
42617 | 171 |
@@{antiquotation lemma} options @{syntax prop} @'by' @{syntax method} @{syntax method}? | |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
172 |
@@{antiquotation prop} options styles @{syntax prop} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
173 |
@@{antiquotation term} options styles @{syntax term} | |
43618 | 174 |
@@{antiquotation (HOL) value} options styles @{syntax term} | |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
175 |
@@{antiquotation term_type} options styles @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
176 |
@@{antiquotation typeof} options styles @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
177 |
@@{antiquotation const} options @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
178 |
@@{antiquotation abbrev} options @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
179 |
@@{antiquotation typ} options @{syntax type} | |
63120
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
62969
diff
changeset
|
180 |
@@{antiquotation type} options @{syntax embedded} | |
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
62969
diff
changeset
|
181 |
@@{antiquotation class} options @{syntax embedded} | |
61623 | 182 |
(@@{antiquotation command} | @@{antiquotation method} | @@{antiquotation attribute}) |
183 |
options @{syntax name} |
|
46261 | 184 |
; |
185 |
@{syntax antiquotation}: |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
186 |
@@{antiquotation goals} options | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
187 |
@@{antiquotation subgoals} options | |
62969 | 188 |
@@{antiquotation prf} options @{syntax thms} | |
189 |
@@{antiquotation full_prf} options @{syntax thms} | |
|
58069
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
190 |
@@{antiquotation ML} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
191 |
@@{antiquotation ML_op} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
192 |
@@{antiquotation ML_type} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
193 |
@@{antiquotation ML_structure} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
194 |
@@{antiquotation ML_functor} options @{syntax text} | |
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
195 |
@@{antiquotation emph} options @{syntax text} | |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
196 |
@@{antiquotation bold} options @{syntax text} | |
58716
23a380cc45f4
official support for "tt" style variants, avoid fragile \verb in LaTeX;
wenzelm
parents:
58618
diff
changeset
|
197 |
@@{antiquotation verbatim} options @{syntax text} | |
63672 | 198 |
@@{antiquotation path} options @{syntax embedded} | |
62969 | 199 |
@@{antiquotation "file"} options @{syntax name} | |
63669 | 200 |
@@{antiquotation dir} options @{syntax name} | |
63120
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
62969
diff
changeset
|
201 |
@@{antiquotation url} options @{syntax embedded} | |
58593 | 202 |
@@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and') |
27043 | 203 |
; |
32892 | 204 |
styles: '(' (style + ',') ')' |
32891 | 205 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
206 |
style: (@{syntax name} +) |
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
207 |
; |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
208 |
@@{command print_antiquotations} ('!'?) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
209 |
\<close>} |
27043 | 210 |
|
61614 | 211 |
\<^descr> \<open>@{text s}\<close> prints uninterpreted source text \<open>s\<close>, i.e.\ inner syntax. This |
212 |
is particularly useful to print portions of text according to the Isabelle |
|
213 |
document style, without demanding well-formedness, e.g.\ small pieces of |
|
214 |
terms that should not be parsed or type-checked yet. |
|
61491
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
215 |
|
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
216 |
It is also possible to write this in the short form \<open>\<open>s\<close>\<close> without any |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
217 |
further decoration. |
27043 | 218 |
|
61614 | 219 |
\<^descr> \<open>@{theory_text s}\<close> prints uninterpreted theory source text \<open>s\<close>, i.e.\ |
220 |
outer syntax with command keywords and other tokens. |
|
27043 | 221 |
|
61614 | 222 |
\<^descr> \<open>@{theory A}\<close> prints the name \<open>A\<close>, which is guaranteed to refer to a valid |
223 |
ancestor theory in the current context. |
|
224 |
||
225 |
\<^descr> \<open>@{thm a\<^sub>1 \<dots> a\<^sub>n}\<close> prints theorems \<open>a\<^sub>1 \<dots> a\<^sub>n\<close>. Full fact expressions are |
|
226 |
allowed here, including attributes (\secref{sec:syn-att}). |
|
27043 | 227 |
|
61493 | 228 |
\<^descr> \<open>@{prop \<phi>}\<close> prints a well-typed proposition \<open>\<phi>\<close>. |
27043 | 229 |
|
61614 | 230 |
\<^descr> \<open>@{lemma \<phi> by m}\<close> proves a well-typed proposition \<open>\<phi>\<close> by method \<open>m\<close> and |
231 |
prints the original \<open>\<phi>\<close>. |
|
27453 | 232 |
|
61493 | 233 |
\<^descr> \<open>@{term t}\<close> prints a well-typed term \<open>t\<close>. |
43613
7afbaf5a406b
adding a minimalistic documentation of the value antiquotation in the Isar reference manual
bulwahn
parents:
42936
diff
changeset
|
234 |
|
61614 | 235 |
\<^descr> \<open>@{value t}\<close> evaluates a term \<open>t\<close> and prints its result, see also |
236 |
@{command_ref (HOL) value}. |
|
27043 | 237 |
|
61614 | 238 |
\<^descr> \<open>@{term_type t}\<close> prints a well-typed term \<open>t\<close> annotated with its type. |
32898
e871d897969c
term styles also cover antiquotations term_type and typeof
haftmann
parents:
32892
diff
changeset
|
239 |
|
61614 | 240 |
\<^descr> \<open>@{typeof t}\<close> prints the type of a well-typed term \<open>t\<close>. |
32898
e871d897969c
term styles also cover antiquotations term_type and typeof
haftmann
parents:
32892
diff
changeset
|
241 |
|
61614 | 242 |
\<^descr> \<open>@{const c}\<close> prints a logical or syntactic constant \<open>c\<close>. |
27043 | 243 |
|
61614 | 244 |
\<^descr> \<open>@{abbrev c x\<^sub>1 \<dots> x\<^sub>n}\<close> prints a constant abbreviation \<open>c x\<^sub>1 \<dots> x\<^sub>n \<equiv> rhs\<close> |
245 |
as defined in the current context. |
|
39305
d4fa19eb0822
'class' and 'type' are now antiquoations by default
haftmann
parents:
32898
diff
changeset
|
246 |
|
61493 | 247 |
\<^descr> \<open>@{typ \<tau>}\<close> prints a well-formed type \<open>\<tau>\<close>. |
39305
d4fa19eb0822
'class' and 'type' are now antiquoations by default
haftmann
parents:
32898
diff
changeset
|
248 |
|
61614 | 249 |
\<^descr> \<open>@{type \<kappa>}\<close> prints a (logical or syntactic) type constructor \<open>\<kappa>\<close>. |
39305
d4fa19eb0822
'class' and 'type' are now antiquoations by default
haftmann
parents:
32898
diff
changeset
|
250 |
|
61493 | 251 |
\<^descr> \<open>@{class c}\<close> prints a class \<open>c\<close>. |
39305
d4fa19eb0822
'class' and 'type' are now antiquoations by default
haftmann
parents:
32898
diff
changeset
|
252 |
|
61623 | 253 |
\<^descr> \<open>@{command name}\<close>, \<open>@{method name}\<close>, \<open>@{attribute name}\<close> print checked |
254 |
entities of the Isar language. |
|
255 |
||
61614 | 256 |
\<^descr> \<open>@{goals}\<close> prints the current \<^emph>\<open>dynamic\<close> goal state. This is mainly for |
257 |
support of tactic-emulation scripts within Isar. Presentation of goal states |
|
258 |
does not conform to the idea of human-readable proof documents! |
|
27043 | 259 |
|
61614 | 260 |
When explaining proofs in detail it is usually better to spell out the |
261 |
reasoning via proper Isar proof commands, instead of peeking at the internal |
|
262 |
machine configuration. |
|
27043 | 263 |
|
61614 | 264 |
\<^descr> \<open>@{subgoals}\<close> is similar to \<open>@{goals}\<close>, but does not print the main goal. |
27043 | 265 |
|
61614 | 266 |
\<^descr> \<open>@{prf a\<^sub>1 \<dots> a\<^sub>n}\<close> prints the (compact) proof terms corresponding to the |
267 |
theorems \<open>a\<^sub>1 \<dots> a\<^sub>n\<close>. Note that this requires proof terms to be switched on |
|
268 |
for the current logic session. |
|
27043 | 269 |
|
61614 | 270 |
\<^descr> \<open>@{full_prf a\<^sub>1 \<dots> a\<^sub>n}\<close> is like \<open>@{prf a\<^sub>1 \<dots> a\<^sub>n}\<close>, but prints the full |
271 |
proof terms, i.e.\ also displays information omitted in the compact proof |
|
272 |
term, which is denoted by ``\<open>_\<close>'' placeholders there. |
|
27043 | 273 |
|
61614 | 274 |
\<^descr> \<open>@{ML s}\<close>, \<open>@{ML_op s}\<close>, \<open>@{ML_type s}\<close>, \<open>@{ML_structure s}\<close>, and |
275 |
\<open>@{ML_functor s}\<close> check text \<open>s\<close> as ML value, infix operator, type, |
|
276 |
structure, and functor respectively. The source is printed verbatim. |
|
27043 | 277 |
|
61614 | 278 |
\<^descr> \<open>@{emph s}\<close> prints document source recursively, with {\LaTeX} markup |
279 |
\<^verbatim>\<open>\emph{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>. |
|
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
280 |
|
61614 | 281 |
\<^descr> \<open>@{bold s}\<close> prints document source recursively, with {\LaTeX} markup |
282 |
\<^verbatim>\<open>\textbf{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>. |
|
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
283 |
|
61614 | 284 |
\<^descr> \<open>@{verbatim s}\<close> prints uninterpreted source text literally as ASCII |
285 |
characters, using some type-writer font style. |
|
58716
23a380cc45f4
official support for "tt" style variants, avoid fragile \verb in LaTeX;
wenzelm
parents:
58618
diff
changeset
|
286 |
|
63669 | 287 |
\<^descr> \<open>@{path name}\<close> prints the file-system path name verbatim. |
40801 | 288 |
|
63669 | 289 |
\<^descr> \<open>@{file name}\<close> is like \<open>@{path name}\<close>, but ensures that \<open>name\<close> refers to a |
290 |
plain file. |
|
291 |
||
292 |
\<^descr> \<open>@{dir name}\<close> is like \<open>@{path name}\<close>, but ensures that \<open>name\<close> refers to a |
|
293 |
directory. |
|
54705 | 294 |
|
61614 | 295 |
\<^descr> \<open>@{url name}\<close> produces markup for the given URL, which results in an |
296 |
active hyperlink within the text. |
|
54702
3daeba5130f0
added document antiquotation @{url}, which produces formal markup for LaTeX and PIDE;
wenzelm
parents:
54346
diff
changeset
|
297 |
|
61614 | 298 |
\<^descr> \<open>@{cite name}\<close> produces a citation \<^verbatim>\<open>\cite{name}\<close> in {\LaTeX}, where the |
299 |
name refers to some Bib{\TeX} database entry. |
|
58593 | 300 |
|
61614 | 301 |
The variant \<open>@{cite \<open>opt\<close> name}\<close> produces \<^verbatim>\<open>\cite[opt]{name}\<close> with some |
302 |
free-form optional argument. Multiple names are output with commas, e.g. |
|
303 |
\<open>@{cite foo \<AND> bar}\<close> becomes \<^verbatim>\<open>\cite{foo,bar}\<close>. |
|
58593 | 304 |
|
305 |
The {\LaTeX} macro name is determined by the antiquotation option |
|
306 |
@{antiquotation_option_def cite_macro}, or the configuration option |
|
61614 | 307 |
@{attribute cite_macro} in the context. For example, \<open>@{cite [cite_macro = |
308 |
nocite] foobar}\<close> produces \<^verbatim>\<open>\nocite{foobar}\<close>. |
|
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
309 |
|
61614 | 310 |
\<^descr> @{command "print_antiquotations"} prints all document antiquotations that |
311 |
are defined in the current context; the ``\<open>!\<close>'' option indicates extra |
|
312 |
verbosity. |
|
58618 | 313 |
\<close> |
27043 | 314 |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
315 |
|
58618 | 316 |
subsection \<open>Styled antiquotations\<close> |
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
317 |
|
61624 | 318 |
text \<open> |
319 |
The antiquotations \<open>thm\<close>, \<open>prop\<close> and \<open>term\<close> admit an extra \<^emph>\<open>style\<close> |
|
320 |
specification to modify the printed result. A style is specified by a name |
|
321 |
with a possibly empty number of arguments; multiple styles can be sequenced |
|
322 |
with commas. The following standard styles are available: |
|
27043 | 323 |
|
61624 | 324 |
\<^descr> \<open>lhs\<close> extracts the first argument of any application form with at least |
325 |
two arguments --- typically meta-level or object-level equality, or any |
|
326 |
other binary relation. |
|
27043 | 327 |
|
61624 | 328 |
\<^descr> \<open>rhs\<close> is like \<open>lhs\<close>, but extracts the second argument. |
27043 | 329 |
|
61624 | 330 |
\<^descr> \<open>concl\<close> extracts the conclusion \<open>C\<close> from a rule in Horn-clause normal form |
331 |
\<open>A\<^sub>1 \<Longrightarrow> \<dots> A\<^sub>n \<Longrightarrow> C\<close>. |
|
27043 | 332 |
|
61624 | 333 |
\<^descr> \<open>prem\<close> \<open>n\<close> extract premise number \<open>n\<close> from from a rule in Horn-clause |
334 |
normal form \<open>A\<^sub>1 \<Longrightarrow> \<dots> A\<^sub>n \<Longrightarrow> C\<close>. |
|
58618 | 335 |
\<close> |
27043 | 336 |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
337 |
|
58618 | 338 |
subsection \<open>General options\<close> |
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
339 |
|
61624 | 340 |
text \<open> |
341 |
The following options are available to tune the printed output of |
|
342 |
antiquotations. Note that many of these coincide with system and |
|
54346 | 343 |
configuration options of the same names. |
27043 | 344 |
|
61624 | 345 |
\<^descr> @{antiquotation_option_def show_types}~\<open>= bool\<close> and |
346 |
@{antiquotation_option_def show_sorts}~\<open>= bool\<close> control printing of |
|
347 |
explicit type and sort constraints. |
|
27043 | 348 |
|
61624 | 349 |
\<^descr> @{antiquotation_option_def show_structs}~\<open>= bool\<close> controls printing of |
350 |
implicit structures. |
|
27043 | 351 |
|
61624 | 352 |
\<^descr> @{antiquotation_option_def show_abbrevs}~\<open>= bool\<close> controls folding of |
353 |
abbreviations. |
|
40879
ca132ef44944
configuration option "show_abbrevs" supersedes print mode "no_abbrevs", with inverted meaning;
wenzelm
parents:
40801
diff
changeset
|
354 |
|
61624 | 355 |
\<^descr> @{antiquotation_option_def names_long}~\<open>= bool\<close> forces names of types |
356 |
and constants etc.\ to be printed in their fully qualified internal form. |
|
27043 | 357 |
|
61624 | 358 |
\<^descr> @{antiquotation_option_def names_short}~\<open>= bool\<close> forces names of types |
359 |
and constants etc.\ to be printed unqualified. Note that internalizing the |
|
360 |
output again in the current context may well yield a different result. |
|
27043 | 361 |
|
61624 | 362 |
\<^descr> @{antiquotation_option_def names_unique}~\<open>= bool\<close> determines whether the |
363 |
printed version of qualified names should be made sufficiently long to |
|
364 |
avoid overlap with names declared further back. Set to \<open>false\<close> for more |
|
365 |
concise output. |
|
27043 | 366 |
|
61624 | 367 |
\<^descr> @{antiquotation_option_def eta_contract}~\<open>= bool\<close> prints terms in |
368 |
\<open>\<eta>\<close>-contracted form. |
|
27043 | 369 |
|
61624 | 370 |
\<^descr> @{antiquotation_option_def display}~\<open>= bool\<close> indicates if the text is to |
371 |
be output as multi-line ``display material'', rather than a small piece of |
|
372 |
text without line breaks (which is the default). |
|
27043 | 373 |
|
61624 | 374 |
In this mode the embedded entities are printed in the same style as the |
375 |
main theory text. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
376 |
|
61624 | 377 |
\<^descr> @{antiquotation_option_def break}~\<open>= bool\<close> controls line breaks in |
378 |
non-display material. |
|
27043 | 379 |
|
61624 | 380 |
\<^descr> @{antiquotation_option_def quotes}~\<open>= bool\<close> indicates if the output |
381 |
should be enclosed in double quotes. |
|
27043 | 382 |
|
61624 | 383 |
\<^descr> @{antiquotation_option_def mode}~\<open>= name\<close> adds \<open>name\<close> to the print mode |
384 |
to be used for presentation. Note that the standard setup for {\LaTeX} |
|
61997 | 385 |
output is already present by default, with mode ``\<open>latex\<close>''. |
27043 | 386 |
|
61624 | 387 |
\<^descr> @{antiquotation_option_def margin}~\<open>= nat\<close> and |
388 |
@{antiquotation_option_def indent}~\<open>= nat\<close> change the margin or |
|
389 |
indentation for pretty printing of display material. |
|
390 |
||
391 |
\<^descr> @{antiquotation_option_def goals_limit}~\<open>= nat\<close> determines the maximum |
|
392 |
number of subgoals to be printed (for goal-based antiquotation). |
|
27043 | 393 |
|
61624 | 394 |
\<^descr> @{antiquotation_option_def source}~\<open>= bool\<close> prints the original source |
395 |
text of the antiquotation arguments, rather than its internal |
|
396 |
representation. Note that formal checking of @{antiquotation "thm"}, |
|
397 |
@{antiquotation "term"}, etc. is still enabled; use the @{antiquotation |
|
398 |
"text"} antiquotation for unchecked output. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
399 |
|
61624 | 400 |
Regular \<open>term\<close> and \<open>typ\<close> antiquotations with \<open>source = false\<close> involve a |
401 |
full round-trip from the original source to an internalized logical entity |
|
402 |
back to a source form, according to the syntax of the current context. |
|
403 |
Thus the printed output is not under direct control of the author, it may |
|
404 |
even fluctuate a bit as the underlying theory is changed later on. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
405 |
|
61624 | 406 |
In contrast, @{antiquotation_option source}~\<open>= true\<close> admits direct |
407 |
printing of the given source text, with the desirable well-formedness |
|
408 |
check in the background, but without modification of the printed text. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
409 |
|
61624 | 410 |
For Boolean flags, ``\<open>name = true\<close>'' may be abbreviated as ``\<open>name\<close>''. All |
411 |
of the above flags are disabled by default, unless changed specifically for |
|
412 |
a logic session in the corresponding \<^verbatim>\<open>ROOT\<close> file. |
|
61458 | 413 |
\<close> |
27043 | 414 |
|
415 |
||
62274 | 416 |
section \<open>Markdown-like text structure\<close> |
417 |
||
418 |
text \<open> |
|
419 |
The markup commands @{command_ref text}, @{command_ref txt}, @{command_ref |
|
420 |
text_raw} (\secref{sec:markup}) consist of plain text. Its internal |
|
421 |
structure consists of paragraphs and (nested) lists, using special Isabelle |
|
422 |
symbols and some rules for indentation and blank lines. This quasi-visual |
|
63680 | 423 |
format resembles \<^emph>\<open>Markdown\<close>\<^footnote>\<open>\<^url>\<open>http://commonmark.org\<close>\<close>, but the full |
424 |
complexity of that notation is avoided. |
|
62274 | 425 |
|
426 |
This is a summary of the main principles of minimal Markdown in Isabelle: |
|
427 |
||
428 |
\<^item> List items start with the following markers |
|
429 |
\<^descr>[itemize:] \<^verbatim>\<open>\<^item>\<close> |
|
430 |
\<^descr>[enumerate:] \<^verbatim>\<open>\<^enum>\<close> |
|
431 |
\<^descr>[description:] \<^verbatim>\<open>\<^descr>\<close> |
|
432 |
||
433 |
\<^item> Adjacent list items with same indentation and same marker are grouped |
|
434 |
into a single list. |
|
435 |
||
436 |
\<^item> Singleton blank lines separate paragraphs. |
|
437 |
||
438 |
\<^item> Multiple blank lines escape from the current list hierarchy. |
|
439 |
||
440 |
Notable differences to official Markdown: |
|
441 |
||
442 |
\<^item> Indentation of list items needs to match exactly. |
|
443 |
||
444 |
\<^item> Indentation is unlimited (official Markdown interprets four spaces as |
|
445 |
block quote). |
|
446 |
||
447 |
\<^item> List items always consist of paragraphs --- there is no notion of |
|
448 |
``tight'' list. |
|
449 |
||
450 |
\<^item> Section headings are expressed via Isar document markup commands |
|
451 |
(\secref{sec:markup}). |
|
452 |
||
453 |
\<^item> URLs, font styles, other special content is expressed via antiquotations |
|
454 |
(\secref{sec:antiq}), usually with proper nesting of sub-languages via |
|
455 |
text cartouches. |
|
456 |
\<close> |
|
457 |
||
458 |
||
58618 | 459 |
section \<open>Markup via command tags \label{sec:tags}\<close> |
27043 | 460 |
|
61624 | 461 |
text \<open> |
462 |
Each Isabelle/Isar command may be decorated by additional presentation tags, |
|
463 |
to indicate some modification in the way it is printed in the document. |
|
27043 | 464 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
465 |
@{rail \<open> |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
466 |
@{syntax_def tags}: ( tag * ) |
27043 | 467 |
; |
63138
70f4d67235a0
clarified syntax category names according to Isabelle/ML/Scala;
wenzelm
parents:
63120
diff
changeset
|
468 |
tag: '%' (@{syntax short_ident} | @{syntax string}) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
469 |
\<close>} |
27043 | 470 |
|
61624 | 471 |
Some tags are pre-declared for certain classes of commands, serving as |
472 |
default markup if no tags are given in the text: |
|
27043 | 473 |
|
61421 | 474 |
\<^medskip> |
27043 | 475 |
\begin{tabular}{ll} |
61493 | 476 |
\<open>theory\<close> & theory begin/end \\ |
477 |
\<open>proof\<close> & all proof commands \\ |
|
478 |
\<open>ML\<close> & all commands involving ML code \\ |
|
27043 | 479 |
\end{tabular} |
61421 | 480 |
\<^medskip> |
27043 | 481 |
|
61624 | 482 |
The Isabelle document preparation system @{cite "isabelle-system"} allows |
483 |
tagged command regions to be presented specifically, e.g.\ to fold proof |
|
484 |
texts, or drop parts of the text completely. |
|
27043 | 485 |
|
61624 | 486 |
For example ``@{command "by"}~\<open>%invisible auto\<close>'' causes that piece of proof |
487 |
to be treated as \<open>invisible\<close> instead of \<open>proof\<close> (the default), which may be |
|
488 |
shown or hidden depending on the document setup. In contrast, ``@{command |
|
489 |
"by"}~\<open>%visible auto\<close>'' forces this text to be shown invariably. |
|
27043 | 490 |
|
61624 | 491 |
Explicit tag specifications within a proof apply to all subsequent commands |
492 |
of the same level of nesting. For example, ``@{command "proof"}~\<open>%visible |
|
493 |
\<dots>\<close>~@{command "qed"}'' forces the whole sub-proof to be typeset as \<open>visible\<close> |
|
494 |
(unless some of its parts are tagged differently). |
|
28750 | 495 |
|
61421 | 496 |
\<^medskip> |
61624 | 497 |
Command tags merely produce certain markup environments for type-setting. |
63680 | 498 |
The meaning of these is determined by {\LaTeX} macros, as defined in |
499 |
\<^file>\<open>~~/lib/texinputs/isabelle.sty\<close> or by the document author. The Isabelle |
|
61624 | 500 |
document preparation tools also provide some high-level options to specify |
501 |
the meaning of arbitrary tags to ``keep'', ``drop'', or ``fold'' the |
|
502 |
corresponding parts of the text. Logic sessions may also specify ``document |
|
503 |
versions'', where given tags are interpreted in some particular way. Again |
|
504 |
see @{cite "isabelle-system"} for further details. |
|
58618 | 505 |
\<close> |
27043 | 506 |
|
507 |
||
58618 | 508 |
section \<open>Railroad diagrams\<close> |
42658 | 509 |
|
58618 | 510 |
text \<open> |
42658 | 511 |
\begin{matharray}{rcl} |
61493 | 512 |
@{antiquotation_def "rail"} & : & \<open>antiquotation\<close> \\ |
42658 | 513 |
\end{matharray} |
514 |
||
55113 | 515 |
@{rail \<open> |
59937 | 516 |
'rail' @{syntax text} |
55113 | 517 |
\<close>} |
42658 | 518 |
|
61624 | 519 |
The @{antiquotation rail} antiquotation allows to include syntax diagrams |
63680 | 520 |
into Isabelle documents. {\LaTeX} requires the style file |
521 |
\<^file>\<open>~~/lib/texinputs/railsetup.sty\<close>, which can be used via |
|
61503 | 522 |
\<^verbatim>\<open>\usepackage{railsetup}\<close> in \<^verbatim>\<open>root.tex\<close>, for example. |
42658 | 523 |
|
61624 | 524 |
The rail specification language is quoted here as Isabelle @{syntax string} |
525 |
or text @{syntax "cartouche"}; it has its own grammar given below. |
|
42658 | 526 |
|
55120 | 527 |
\begingroup |
61474 | 528 |
\def\isasymnewline{\isatt{\isacharbackslash\isacharless newline\isachargreater}} |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
529 |
@{rail \<open> |
42658 | 530 |
rule? + ';' |
531 |
; |
|
532 |
rule: ((identifier | @{syntax antiquotation}) ':')? body |
|
533 |
; |
|
534 |
body: concatenation + '|' |
|
535 |
; |
|
536 |
concatenation: ((atom '?'?) +) (('*' | '+') atom?)? |
|
537 |
; |
|
538 |
atom: '(' body? ')' | identifier | |
|
539 |
'@'? (string | @{syntax antiquotation}) | |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
540 |
'\<newline>' |
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
541 |
\<close>} |
55120 | 542 |
\endgroup |
42658 | 543 |
|
63138
70f4d67235a0
clarified syntax category names according to Isabelle/ML/Scala;
wenzelm
parents:
63120
diff
changeset
|
544 |
The lexical syntax of \<open>identifier\<close> coincides with that of @{syntax |
70f4d67235a0
clarified syntax category names according to Isabelle/ML/Scala;
wenzelm
parents:
63120
diff
changeset
|
545 |
short_ident} in regular Isabelle syntax, but \<open>string\<close> uses single quotes |
70f4d67235a0
clarified syntax category names according to Isabelle/ML/Scala;
wenzelm
parents:
63120
diff
changeset
|
546 |
instead of double quotes of the standard @{syntax string} category. |
42658 | 547 |
|
61624 | 548 |
Each \<open>rule\<close> defines a formal language (with optional name), using a notation |
549 |
that is similar to EBNF or regular expressions with recursion. The meaning |
|
550 |
and visual appearance of these rail language elements is illustrated by the |
|
551 |
following representative examples. |
|
42658 | 552 |
|
61503 | 553 |
\<^item> Empty \<^verbatim>\<open>()\<close> |
42658 | 554 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
555 |
@{rail \<open>()\<close>} |
42658 | 556 |
|
61503 | 557 |
\<^item> Nonterminal \<^verbatim>\<open>A\<close> |
42658 | 558 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
559 |
@{rail \<open>A\<close>} |
42658 | 560 |
|
61503 | 561 |
\<^item> Nonterminal via Isabelle antiquotation \<^verbatim>\<open>@{syntax method}\<close> |
42658 | 562 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
563 |
@{rail \<open>@{syntax method}\<close>} |
42658 | 564 |
|
61503 | 565 |
\<^item> Terminal \<^verbatim>\<open>'xyz'\<close> |
42658 | 566 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
567 |
@{rail \<open>'xyz'\<close>} |
42658 | 568 |
|
61503 | 569 |
\<^item> Terminal in keyword style \<^verbatim>\<open>@'xyz'\<close> |
42658 | 570 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
571 |
@{rail \<open>@'xyz'\<close>} |
42658 | 572 |
|
61503 | 573 |
\<^item> Terminal via Isabelle antiquotation \<^verbatim>\<open>@@{method rule}\<close> |
42658 | 574 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
575 |
@{rail \<open>@@{method rule}\<close>} |
42658 | 576 |
|
61503 | 577 |
\<^item> Concatenation \<^verbatim>\<open>A B C\<close> |
42658 | 578 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
579 |
@{rail \<open>A B C\<close>} |
42658 | 580 |
|
61503 | 581 |
\<^item> Newline inside concatenation \<^verbatim>\<open>A B C \<newline> D E F\<close> |
42658 | 582 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
583 |
@{rail \<open>A B C \<newline> D E F\<close>} |
42658 | 584 |
|
61503 | 585 |
\<^item> Variants \<^verbatim>\<open>A | B | C\<close> |
42658 | 586 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
587 |
@{rail \<open>A | B | C\<close>} |
42658 | 588 |
|
61503 | 589 |
\<^item> Option \<^verbatim>\<open>A ?\<close> |
42658 | 590 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
591 |
@{rail \<open>A ?\<close>} |
42658 | 592 |
|
61503 | 593 |
\<^item> Repetition \<^verbatim>\<open>A *\<close> |
42658 | 594 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
595 |
@{rail \<open>A *\<close>} |
42658 | 596 |
|
61503 | 597 |
\<^item> Repetition with separator \<^verbatim>\<open>A * sep\<close> |
42658 | 598 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
599 |
@{rail \<open>A * sep\<close>} |
42658 | 600 |
|
61503 | 601 |
\<^item> Strict repetition \<^verbatim>\<open>A +\<close> |
42658 | 602 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
603 |
@{rail \<open>A +\<close>} |
42658 | 604 |
|
61503 | 605 |
\<^item> Strict repetition with separator \<^verbatim>\<open>A + sep\<close> |
42658 | 606 |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
607 |
@{rail \<open>A + sep\<close>} |
58618 | 608 |
\<close> |
42658 | 609 |
|
610 |
||
58618 | 611 |
section \<open>Draft presentation\<close> |
27043 | 612 |
|
58618 | 613 |
text \<open> |
27043 | 614 |
\begin{matharray}{rcl} |
61493 | 615 |
@{command_def "display_drafts"}\<open>\<^sup>*\<close> & : & \<open>any \<rightarrow>\<close> \\ |
27043 | 616 |
\end{matharray} |
617 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
618 |
@{rail \<open> |
62969 | 619 |
@@{command display_drafts} (@{syntax name} +) |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
620 |
\<close>} |
27043 | 621 |
|
61624 | 622 |
\<^descr> @{command "display_drafts"}~\<open>paths\<close> performs simple output of a given list |
623 |
of raw source files. Only those symbols that do not require additional |
|
624 |
{\LaTeX} packages are displayed properly, everything else is left verbatim. |
|
58618 | 625 |
\<close> |
27043 | 626 |
|
627 |
end |