author | wenzelm |
Fri, 12 Apr 2019 22:57:17 +0200 | |
changeset 70140 | d13865c21e36 |
parent 70122 | a0b21b4b7a4a |
child 71146 | f7a9889068ff |
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 |
|
69597 | 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} |
|
69597 | 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> \\ |
|
68809 | 97 |
@{antiquotation_def locale} & : & \<open>antiquotation\<close> \\ |
61493 | 98 |
@{antiquotation_def "text"} & : & \<open>antiquotation\<close> \\ |
99 |
@{antiquotation_def goals} & : & \<open>antiquotation\<close> \\ |
|
100 |
@{antiquotation_def subgoals} & : & \<open>antiquotation\<close> \\ |
|
101 |
@{antiquotation_def prf} & : & \<open>antiquotation\<close> \\ |
|
102 |
@{antiquotation_def full_prf} & : & \<open>antiquotation\<close> \\ |
|
103 |
@{antiquotation_def ML} & : & \<open>antiquotation\<close> \\ |
|
104 |
@{antiquotation_def ML_op} & : & \<open>antiquotation\<close> \\ |
|
105 |
@{antiquotation_def ML_type} & : & \<open>antiquotation\<close> \\ |
|
106 |
@{antiquotation_def ML_structure} & : & \<open>antiquotation\<close> \\ |
|
107 |
@{antiquotation_def ML_functor} & : & \<open>antiquotation\<close> \\ |
|
108 |
@{antiquotation_def emph} & : & \<open>antiquotation\<close> \\ |
|
109 |
@{antiquotation_def bold} & : & \<open>antiquotation\<close> \\ |
|
110 |
@{antiquotation_def verbatim} & : & \<open>antiquotation\<close> \\ |
|
67219 | 111 |
@{antiquotation_def session} & : & \<open>antiquotation\<close> \\ |
61493 | 112 |
@{antiquotation_def "file"} & : & \<open>antiquotation\<close> \\ |
113 |
@{antiquotation_def "url"} & : & \<open>antiquotation\<close> \\ |
|
114 |
@{antiquotation_def "cite"} & : & \<open>antiquotation\<close> \\ |
|
61494 | 115 |
@{command_def "print_antiquotations"}\<open>\<^sup>*\<close> & : & \<open>context \<rightarrow>\<close> \\ |
27043 | 116 |
\end{matharray} |
117 |
||
61614 | 118 |
The overall content of an Isabelle/Isar theory may alternate between formal |
119 |
and informal text. The main body consists of formal specification and proof |
|
120 |
commands, interspersed with markup commands (\secref{sec:markup}) or |
|
121 |
document comments (\secref{sec:comments}). The argument of markup commands |
|
122 |
quotes informal text to be printed in the resulting document, but may again |
|
123 |
refer to formal entities via \<^emph>\<open>document antiquotations\<close>. |
|
27043 | 124 |
|
61503 | 125 |
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
|
126 |
within a text block makes |
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
127 |
\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
|
128 |
|
61614 | 129 |
Antiquotations usually spare the author tedious typing of logical entities |
130 |
in full detail. Even more importantly, some degree of consistency-checking |
|
131 |
between the main body of formal text and its informal explanation is |
|
132 |
achieved, since terms and types appearing in antiquotations are checked |
|
133 |
within the current theory or proof context. |
|
27043 | 134 |
|
61614 | 135 |
\<^medskip> |
136 |
Antiquotations are in general written as |
|
137 |
\<^verbatim>\<open>@{\<close>\<open>name\<close>~\<^verbatim>\<open>[\<close>\<open>options\<close>\<^verbatim>\<open>]\<close>~\<open>arguments\<close>\<^verbatim>\<open>}\<close>. The short form |
|
138 |
\<^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>) |
|
139 |
works for a single argument that is a cartouche. A cartouche without special |
|
140 |
decoration is equivalent to \<^verbatim>\<open>\<^cartouche>\<close>\<open>\<open>argument_content\<close>\<close>, which is |
|
141 |
equivalent to \<^verbatim>\<open>@{cartouche\<close>~\<open>\<open>argument_content\<close>\<close>\<^verbatim>\<open>}\<close>. The special name |
|
61595 | 142 |
@{antiquotation_def cartouche} is defined in the context: Isabelle/Pure |
143 |
introduces that as an alias to @{antiquotation_ref text} (see below). |
|
144 |
Consequently, \<open>\<open>foo_bar + baz \<le> bazar\<close>\<close> prints literal quasi-formal text |
|
61614 | 145 |
(unchecked). A control symbol \<^verbatim>\<open>\\<close>\<^verbatim>\<open><^\<close>\<open>name\<close>\<^verbatim>\<open>>\<close> within the body text, but |
146 |
without a subsequent cartouche, is equivalent to \<^verbatim>\<open>@{\<close>\<open>name\<close>\<^verbatim>\<open>}\<close>. |
|
61472 | 147 |
|
61474 | 148 |
\begingroup |
149 |
\def\isasymcontrolstart{\isatt{\isacharbackslash\isacharless\isacharcircum}} |
|
69597 | 150 |
\<^rail>\<open> |
61472 | 151 |
@{syntax_def antiquotation}: |
61474 | 152 |
'@{' antiquotation_body '}' | |
61491
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
153 |
'\<controlstart>' @{syntax_ref name} '>' @{syntax_ref cartouche} | |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
154 |
@{syntax_ref cartouche} |
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 |
options: '[' (option * ',') ']' |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
157 |
; |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
158 |
option: @{syntax name} | @{syntax name} '=' @{syntax name} |
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
159 |
; |
69597 | 160 |
\<close> |
61474 | 161 |
\endgroup |
59917
9830c944670f
more uniform "verbose" option to print name space;
wenzelm
parents:
59783
diff
changeset
|
162 |
|
61614 | 163 |
Note that the syntax of antiquotations may \<^emph>\<open>not\<close> include source comments |
164 |
\<^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
|
165 |
|
43618 | 166 |
%% FIXME less monolithic presentation, move to individual sections!? |
69597 | 167 |
\<^rail>\<open> |
61472 | 168 |
@{syntax_def antiquotation_body}: |
61614 | 169 |
(@@{antiquotation text} | @@{antiquotation cartouche} | @@{antiquotation theory_text}) |
170 |
options @{syntax text} | |
|
68481 | 171 |
@@{antiquotation theory} options @{syntax embedded} | |
62969 | 172 |
@@{antiquotation thm} options styles @{syntax thms} | |
42617 | 173 |
@@{antiquotation lemma} options @{syntax prop} @'by' @{syntax method} @{syntax method}? | |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
174 |
@@{antiquotation prop} options styles @{syntax prop} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
175 |
@@{antiquotation term} options styles @{syntax term} | |
43618 | 176 |
@@{antiquotation (HOL) value} options styles @{syntax term} | |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
177 |
@@{antiquotation term_type} options styles @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
178 |
@@{antiquotation typeof} options styles @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
179 |
@@{antiquotation const} options @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
180 |
@@{antiquotation abbrev} options @{syntax term} | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
181 |
@@{antiquotation typ} options @{syntax type} | |
63120
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
62969
diff
changeset
|
182 |
@@{antiquotation type} options @{syntax embedded} | |
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
62969
diff
changeset
|
183 |
@@{antiquotation class} options @{syntax embedded} | |
68809 | 184 |
@@{antiquotation locale} options @{syntax embedded} | |
61623 | 185 |
(@@{antiquotation command} | @@{antiquotation method} | @@{antiquotation attribute}) |
186 |
options @{syntax name} |
|
46261 | 187 |
; |
188 |
@{syntax antiquotation}: |
|
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
189 |
@@{antiquotation goals} options | |
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
190 |
@@{antiquotation subgoals} options | |
62969 | 191 |
@@{antiquotation prf} options @{syntax thms} | |
192 |
@@{antiquotation full_prf} options @{syntax thms} | |
|
58069
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
193 |
@@{antiquotation ML} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
194 |
@@{antiquotation ML_op} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
195 |
@@{antiquotation ML_type} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
196 |
@@{antiquotation ML_structure} options @{syntax text} | |
0255436b3d85
more liberal embedded "text", which includes cartouches;
wenzelm
parents:
56594
diff
changeset
|
197 |
@@{antiquotation ML_functor} options @{syntax text} | |
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
198 |
@@{antiquotation emph} options @{syntax text} | |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
199 |
@@{antiquotation bold} options @{syntax text} | |
58716
23a380cc45f4
official support for "tt" style variants, avoid fragile \verb in LaTeX;
wenzelm
parents:
58618
diff
changeset
|
200 |
@@{antiquotation verbatim} options @{syntax text} | |
67219 | 201 |
@@{antiquotation session} options @{syntax embedded} | |
63672 | 202 |
@@{antiquotation path} options @{syntax embedded} | |
62969 | 203 |
@@{antiquotation "file"} options @{syntax name} | |
63669 | 204 |
@@{antiquotation dir} options @{syntax name} | |
63120
629a4c5e953e
embedded content may be delimited via cartouches;
wenzelm
parents:
62969
diff
changeset
|
205 |
@@{antiquotation url} options @{syntax embedded} | |
58593 | 206 |
@@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and') |
27043 | 207 |
; |
32892 | 208 |
styles: '(' (style + ',') ')' |
32891 | 209 |
; |
42596
6c621a9d612a
modernized rail diagrams using @{rail} antiquotation;
wenzelm
parents:
40879
diff
changeset
|
210 |
style: (@{syntax name} +) |
61473
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
211 |
; |
34d1913f0b20
clarified control antiquotations: decode control symbol to get name;
wenzelm
parents:
61472
diff
changeset
|
212 |
@@{command print_antiquotations} ('!'?) |
69597 | 213 |
\<close> |
27043 | 214 |
|
61614 | 215 |
\<^descr> \<open>@{text s}\<close> prints uninterpreted source text \<open>s\<close>, i.e.\ inner syntax. This |
216 |
is particularly useful to print portions of text according to the Isabelle |
|
217 |
document style, without demanding well-formedness, e.g.\ small pieces of |
|
218 |
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
|
219 |
|
97261e6c1d42
another antiquotation short form: undecorated cartouche as alias for @{text};
wenzelm
parents:
61479
diff
changeset
|
220 |
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
|
221 |
further decoration. |
27043 | 222 |
|
61614 | 223 |
\<^descr> \<open>@{theory_text s}\<close> prints uninterpreted theory source text \<open>s\<close>, i.e.\ |
224 |
outer syntax with command keywords and other tokens. |
|
27043 | 225 |
|
68484 | 226 |
\<^descr> \<open>@{theory A}\<close> prints the session-qualified theory name \<open>A\<close>, which is |
227 |
guaranteed to refer to a valid ancestor theory in the current context. |
|
61614 | 228 |
|
229 |
\<^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 |
|
230 |
allowed here, including attributes (\secref{sec:syn-att}). |
|
27043 | 231 |
|
61493 | 232 |
\<^descr> \<open>@{prop \<phi>}\<close> prints a well-typed proposition \<open>\<phi>\<close>. |
27043 | 233 |
|
61614 | 234 |
\<^descr> \<open>@{lemma \<phi> by m}\<close> proves a well-typed proposition \<open>\<phi>\<close> by method \<open>m\<close> and |
235 |
prints the original \<open>\<phi>\<close>. |
|
27453 | 236 |
|
61493 | 237 |
\<^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
|
238 |
|
61614 | 239 |
\<^descr> \<open>@{value t}\<close> evaluates a term \<open>t\<close> and prints its result, see also |
240 |
@{command_ref (HOL) value}. |
|
27043 | 241 |
|
61614 | 242 |
\<^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
|
243 |
|
61614 | 244 |
\<^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
|
245 |
|
61614 | 246 |
\<^descr> \<open>@{const c}\<close> prints a logical or syntactic constant \<open>c\<close>. |
27043 | 247 |
|
61614 | 248 |
\<^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> |
249 |
as defined in the current context. |
|
39305
d4fa19eb0822
'class' and 'type' are now antiquoations by default
haftmann
parents:
32898
diff
changeset
|
250 |
|
61493 | 251 |
\<^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
|
252 |
|
61614 | 253 |
\<^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
|
254 |
|
61493 | 255 |
\<^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
|
256 |
|
68809 | 257 |
\<^descr> \<open>@{locale c}\<close> prints a locale \<open>c\<close>. |
258 |
||
61623 | 259 |
\<^descr> \<open>@{command name}\<close>, \<open>@{method name}\<close>, \<open>@{attribute name}\<close> print checked |
260 |
entities of the Isar language. |
|
261 |
||
61614 | 262 |
\<^descr> \<open>@{goals}\<close> prints the current \<^emph>\<open>dynamic\<close> goal state. This is mainly for |
263 |
support of tactic-emulation scripts within Isar. Presentation of goal states |
|
264 |
does not conform to the idea of human-readable proof documents! |
|
27043 | 265 |
|
61614 | 266 |
When explaining proofs in detail it is usually better to spell out the |
267 |
reasoning via proper Isar proof commands, instead of peeking at the internal |
|
268 |
machine configuration. |
|
27043 | 269 |
|
61614 | 270 |
\<^descr> \<open>@{subgoals}\<close> is similar to \<open>@{goals}\<close>, but does not print the main goal. |
27043 | 271 |
|
61614 | 272 |
\<^descr> \<open>@{prf a\<^sub>1 \<dots> a\<^sub>n}\<close> prints the (compact) proof terms corresponding to the |
273 |
theorems \<open>a\<^sub>1 \<dots> a\<^sub>n\<close>. Note that this requires proof terms to be switched on |
|
274 |
for the current logic session. |
|
27043 | 275 |
|
61614 | 276 |
\<^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 |
277 |
proof terms, i.e.\ also displays information omitted in the compact proof |
|
278 |
term, which is denoted by ``\<open>_\<close>'' placeholders there. |
|
27043 | 279 |
|
61614 | 280 |
\<^descr> \<open>@{ML s}\<close>, \<open>@{ML_op s}\<close>, \<open>@{ML_type s}\<close>, \<open>@{ML_structure s}\<close>, and |
281 |
\<open>@{ML_functor s}\<close> check text \<open>s\<close> as ML value, infix operator, type, |
|
282 |
structure, and functor respectively. The source is printed verbatim. |
|
27043 | 283 |
|
61614 | 284 |
\<^descr> \<open>@{emph s}\<close> prints document source recursively, with {\LaTeX} markup |
285 |
\<^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
|
286 |
|
61614 | 287 |
\<^descr> \<open>@{bold s}\<close> prints document source recursively, with {\LaTeX} markup |
288 |
\<^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
|
289 |
|
61614 | 290 |
\<^descr> \<open>@{verbatim s}\<close> prints uninterpreted source text literally as ASCII |
291 |
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
|
292 |
|
67219 | 293 |
\<^descr> \<open>@{session name}\<close> prints given session name verbatim. The name is checked |
294 |
wrt.\ the dependencies of the current session. |
|
295 |
||
63669 | 296 |
\<^descr> \<open>@{path name}\<close> prints the file-system path name verbatim. |
40801 | 297 |
|
63669 | 298 |
\<^descr> \<open>@{file name}\<close> is like \<open>@{path name}\<close>, but ensures that \<open>name\<close> refers to a |
299 |
plain file. |
|
300 |
||
301 |
\<^descr> \<open>@{dir name}\<close> is like \<open>@{path name}\<close>, but ensures that \<open>name\<close> refers to a |
|
302 |
directory. |
|
54705 | 303 |
|
61614 | 304 |
\<^descr> \<open>@{url name}\<close> produces markup for the given URL, which results in an |
305 |
active hyperlink within the text. |
|
54702
3daeba5130f0
added document antiquotation @{url}, which produces formal markup for LaTeX and PIDE;
wenzelm
parents:
54346
diff
changeset
|
306 |
|
61614 | 307 |
\<^descr> \<open>@{cite name}\<close> produces a citation \<^verbatim>\<open>\cite{name}\<close> in {\LaTeX}, where the |
67297
86a099f896fc
formal check of @{cite} bibtex entries -- only in batch-mode session builds;
wenzelm
parents:
67263
diff
changeset
|
308 |
name refers to some Bib{\TeX} database entry. This is only checked in |
86a099f896fc
formal check of @{cite} bibtex entries -- only in batch-mode session builds;
wenzelm
parents:
67263
diff
changeset
|
309 |
batch-mode session builds. |
58593 | 310 |
|
61614 | 311 |
The variant \<open>@{cite \<open>opt\<close> name}\<close> produces \<^verbatim>\<open>\cite[opt]{name}\<close> with some |
312 |
free-form optional argument. Multiple names are output with commas, e.g. |
|
313 |
\<open>@{cite foo \<AND> bar}\<close> becomes \<^verbatim>\<open>\cite{foo,bar}\<close>. |
|
58593 | 314 |
|
315 |
The {\LaTeX} macro name is determined by the antiquotation option |
|
316 |
@{antiquotation_option_def cite_macro}, or the configuration option |
|
61614 | 317 |
@{attribute cite_macro} in the context. For example, \<open>@{cite [cite_macro = |
318 |
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
|
319 |
|
61614 | 320 |
\<^descr> @{command "print_antiquotations"} prints all document antiquotations that |
321 |
are defined in the current context; the ``\<open>!\<close>'' option indicates extra |
|
322 |
verbosity. |
|
58618 | 323 |
\<close> |
27043 | 324 |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
325 |
|
58618 | 326 |
subsection \<open>Styled antiquotations\<close> |
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
327 |
|
61624 | 328 |
text \<open> |
329 |
The antiquotations \<open>thm\<close>, \<open>prop\<close> and \<open>term\<close> admit an extra \<^emph>\<open>style\<close> |
|
330 |
specification to modify the printed result. A style is specified by a name |
|
331 |
with a possibly empty number of arguments; multiple styles can be sequenced |
|
332 |
with commas. The following standard styles are available: |
|
27043 | 333 |
|
61624 | 334 |
\<^descr> \<open>lhs\<close> extracts the first argument of any application form with at least |
335 |
two arguments --- typically meta-level or object-level equality, or any |
|
336 |
other binary relation. |
|
27043 | 337 |
|
61624 | 338 |
\<^descr> \<open>rhs\<close> is like \<open>lhs\<close>, but extracts the second argument. |
27043 | 339 |
|
61624 | 340 |
\<^descr> \<open>concl\<close> extracts the conclusion \<open>C\<close> from a rule in Horn-clause normal form |
341 |
\<open>A\<^sub>1 \<Longrightarrow> \<dots> A\<^sub>n \<Longrightarrow> C\<close>. |
|
27043 | 342 |
|
61624 | 343 |
\<^descr> \<open>prem\<close> \<open>n\<close> extract premise number \<open>n\<close> from from a rule in Horn-clause |
344 |
normal form \<open>A\<^sub>1 \<Longrightarrow> \<dots> A\<^sub>n \<Longrightarrow> C\<close>. |
|
58618 | 345 |
\<close> |
27043 | 346 |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
347 |
|
58618 | 348 |
subsection \<open>General options\<close> |
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
349 |
|
61624 | 350 |
text \<open> |
351 |
The following options are available to tune the printed output of |
|
352 |
antiquotations. Note that many of these coincide with system and |
|
54346 | 353 |
configuration options of the same names. |
27043 | 354 |
|
61624 | 355 |
\<^descr> @{antiquotation_option_def show_types}~\<open>= bool\<close> and |
356 |
@{antiquotation_option_def show_sorts}~\<open>= bool\<close> control printing of |
|
357 |
explicit type and sort constraints. |
|
27043 | 358 |
|
61624 | 359 |
\<^descr> @{antiquotation_option_def show_structs}~\<open>= bool\<close> controls printing of |
360 |
implicit structures. |
|
27043 | 361 |
|
61624 | 362 |
\<^descr> @{antiquotation_option_def show_abbrevs}~\<open>= bool\<close> controls folding of |
363 |
abbreviations. |
|
40879
ca132ef44944
configuration option "show_abbrevs" supersedes print mode "no_abbrevs", with inverted meaning;
wenzelm
parents:
40801
diff
changeset
|
364 |
|
61624 | 365 |
\<^descr> @{antiquotation_option_def names_long}~\<open>= bool\<close> forces names of types |
366 |
and constants etc.\ to be printed in their fully qualified internal form. |
|
27043 | 367 |
|
61624 | 368 |
\<^descr> @{antiquotation_option_def names_short}~\<open>= bool\<close> forces names of types |
369 |
and constants etc.\ to be printed unqualified. Note that internalizing the |
|
370 |
output again in the current context may well yield a different result. |
|
27043 | 371 |
|
61624 | 372 |
\<^descr> @{antiquotation_option_def names_unique}~\<open>= bool\<close> determines whether the |
373 |
printed version of qualified names should be made sufficiently long to |
|
374 |
avoid overlap with names declared further back. Set to \<open>false\<close> for more |
|
375 |
concise output. |
|
27043 | 376 |
|
61624 | 377 |
\<^descr> @{antiquotation_option_def eta_contract}~\<open>= bool\<close> prints terms in |
378 |
\<open>\<eta>\<close>-contracted form. |
|
27043 | 379 |
|
61624 | 380 |
\<^descr> @{antiquotation_option_def display}~\<open>= bool\<close> indicates if the text is to |
381 |
be output as multi-line ``display material'', rather than a small piece of |
|
382 |
text without line breaks (which is the default). |
|
27043 | 383 |
|
61624 | 384 |
In this mode the embedded entities are printed in the same style as the |
385 |
main theory text. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
386 |
|
61624 | 387 |
\<^descr> @{antiquotation_option_def break}~\<open>= bool\<close> controls line breaks in |
388 |
non-display material. |
|
27043 | 389 |
|
70121 | 390 |
\<^descr> @{antiquotation_option_def cartouche}~\<open>= bool\<close> indicates if the output |
391 |
should be delimited as cartouche. |
|
392 |
||
61624 | 393 |
\<^descr> @{antiquotation_option_def quotes}~\<open>= bool\<close> indicates if the output |
70121 | 394 |
should be delimited via double quotes (option @{antiquotation_option |
395 |
cartouche} takes precedence). Note that the Isabelle {\LaTeX} styles may |
|
396 |
suppress quotes on their own account. |
|
27043 | 397 |
|
61624 | 398 |
\<^descr> @{antiquotation_option_def mode}~\<open>= name\<close> adds \<open>name\<close> to the print mode |
399 |
to be used for presentation. Note that the standard setup for {\LaTeX} |
|
61997 | 400 |
output is already present by default, with mode ``\<open>latex\<close>''. |
27043 | 401 |
|
61624 | 402 |
\<^descr> @{antiquotation_option_def margin}~\<open>= nat\<close> and |
403 |
@{antiquotation_option_def indent}~\<open>= nat\<close> change the margin or |
|
404 |
indentation for pretty printing of display material. |
|
405 |
||
406 |
\<^descr> @{antiquotation_option_def goals_limit}~\<open>= nat\<close> determines the maximum |
|
407 |
number of subgoals to be printed (for goal-based antiquotation). |
|
27043 | 408 |
|
61624 | 409 |
\<^descr> @{antiquotation_option_def source}~\<open>= bool\<close> prints the original source |
410 |
text of the antiquotation arguments, rather than its internal |
|
411 |
representation. Note that formal checking of @{antiquotation "thm"}, |
|
412 |
@{antiquotation "term"}, etc. is still enabled; use the @{antiquotation |
|
413 |
"text"} antiquotation for unchecked output. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
414 |
|
61624 | 415 |
Regular \<open>term\<close> and \<open>typ\<close> antiquotations with \<open>source = false\<close> involve a |
416 |
full round-trip from the original source to an internalized logical entity |
|
417 |
back to a source form, according to the syntax of the current context. |
|
418 |
Thus the printed output is not under direct control of the author, it may |
|
419 |
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
|
420 |
|
61624 | 421 |
In contrast, @{antiquotation_option source}~\<open>= true\<close> admits direct |
422 |
printing of the given source text, with the desirable well-formedness |
|
423 |
check in the background, but without modification of the printed text. |
|
28749
99f6da3bbbf7
renamed "formal comments" to "document comments";
wenzelm
parents:
28747
diff
changeset
|
424 |
|
70122
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
425 |
Cartouche delimiters of the argument are stripped for antiquotations that |
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
426 |
are internally categorized as ``embedded''. |
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
427 |
|
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
428 |
\<^descr> @{antiquotation_option_def source_cartouche} is like |
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
429 |
@{antiquotation_option source}, but cartouche delimiters are always |
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
430 |
preserved in the output. |
a0b21b4b7a4a
strip cartouches from arguments of "embedded" document antiquotations, corresponding to automated update via "isabelle update -u control_cartouches" -- e.g. relevant for documents with thy_output_source (e.g. doc "isar-ref", "jedit", "system");
wenzelm
parents:
70121
diff
changeset
|
431 |
|
61624 | 432 |
For Boolean flags, ``\<open>name = true\<close>'' may be abbreviated as ``\<open>name\<close>''. All |
433 |
of the above flags are disabled by default, unless changed specifically for |
|
434 |
a logic session in the corresponding \<^verbatim>\<open>ROOT\<close> file. |
|
61458 | 435 |
\<close> |
27043 | 436 |
|
437 |
||
62274 | 438 |
section \<open>Markdown-like text structure\<close> |
439 |
||
440 |
text \<open> |
|
441 |
The markup commands @{command_ref text}, @{command_ref txt}, @{command_ref |
|
442 |
text_raw} (\secref{sec:markup}) consist of plain text. Its internal |
|
443 |
structure consists of paragraphs and (nested) lists, using special Isabelle |
|
444 |
symbols and some rules for indentation and blank lines. This quasi-visual |
|
63680 | 445 |
format resembles \<^emph>\<open>Markdown\<close>\<^footnote>\<open>\<^url>\<open>http://commonmark.org\<close>\<close>, but the full |
446 |
complexity of that notation is avoided. |
|
62274 | 447 |
|
448 |
This is a summary of the main principles of minimal Markdown in Isabelle: |
|
449 |
||
450 |
\<^item> List items start with the following markers |
|
451 |
\<^descr>[itemize:] \<^verbatim>\<open>\<^item>\<close> |
|
452 |
\<^descr>[enumerate:] \<^verbatim>\<open>\<^enum>\<close> |
|
453 |
\<^descr>[description:] \<^verbatim>\<open>\<^descr>\<close> |
|
454 |
||
455 |
\<^item> Adjacent list items with same indentation and same marker are grouped |
|
456 |
into a single list. |
|
457 |
||
458 |
\<^item> Singleton blank lines separate paragraphs. |
|
459 |
||
460 |
\<^item> Multiple blank lines escape from the current list hierarchy. |
|
461 |
||
462 |
Notable differences to official Markdown: |
|
463 |
||
464 |
\<^item> Indentation of list items needs to match exactly. |
|
465 |
||
466 |
\<^item> Indentation is unlimited (official Markdown interprets four spaces as |
|
467 |
block quote). |
|
468 |
||
469 |
\<^item> List items always consist of paragraphs --- there is no notion of |
|
470 |
``tight'' list. |
|
471 |
||
472 |
\<^item> Section headings are expressed via Isar document markup commands |
|
473 |
(\secref{sec:markup}). |
|
474 |
||
475 |
\<^item> URLs, font styles, other special content is expressed via antiquotations |
|
476 |
(\secref{sec:antiq}), usually with proper nesting of sub-languages via |
|
477 |
text cartouches. |
|
478 |
\<close> |
|
479 |
||
480 |
||
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
481 |
section \<open>Document markers and command tags \label{sec:document-markers}\<close> |
27043 | 482 |
|
61624 | 483 |
text \<open> |
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
484 |
\emph{Document markers} are formal comments of the form \<open>\<^marker>\<open>marker_body\<close>\<close> |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
485 |
(using the control symbol \<^verbatim>\<open>\<^marker>\<close>) and may occur anywhere within the |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
486 |
outer syntax of a command: the inner syntax of a marker body resembles that |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
487 |
for attributes (\secref{sec:syn-att}). In contrast, \emph{Command tags} may |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
488 |
only occur after a command keyword and are treated as special markers as |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
489 |
explained below. |
27043 | 490 |
|
69597 | 491 |
\<^rail>\<open> |
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
492 |
@{syntax_def marker}: '\<^marker>' @{syntax cartouche} |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
493 |
; |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
494 |
@{syntax_def marker_body}: (@{syntax name} @{syntax args} * ',') |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
495 |
; |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
496 |
@{syntax_def tags}: tag* |
27043 | 497 |
; |
63138
70f4d67235a0
clarified syntax category names according to Isabelle/ML/Scala;
wenzelm
parents:
63120
diff
changeset
|
498 |
tag: '%' (@{syntax short_ident} | @{syntax string}) |
69597 | 499 |
\<close> |
27043 | 500 |
|
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
501 |
Document markers are stripped from the document output, but surrounding |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
502 |
white-space is preserved: e.g.\ a marker at the end of a line does not |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
503 |
affect the subsequent line break. Markers operate within the semantic |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
504 |
presentation context of a command, and may modify it to change the overall |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
505 |
appearance of a command span (e.g.\ by adding tags). |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
506 |
|
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
507 |
Each document marker has its own syntax defined in the theory context; the |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
508 |
following markers are predefined in Isabelle/Pure: |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
509 |
|
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
510 |
\<^rail>\<open> |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
511 |
(@@{document_marker_def title} | |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
512 |
@@{document_marker_def creator} | |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
513 |
@@{document_marker_def contributor} | |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
514 |
@@{document_marker_def date} | |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
515 |
@@{document_marker_def license} | |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
516 |
@@{document_marker_def description}) @{syntax embedded} |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
517 |
; |
70140 | 518 |
@@{document_marker_def tag} (scope?) @{syntax name} |
519 |
; |
|
520 |
scope: '(' ('proof' | 'command') ')' |
|
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
521 |
\<close> |
27043 | 522 |
|
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
523 |
\<^descr> \<open>\<^marker>\<open>title arg\<close>\<close>, \<open>\<^marker>\<open>creator arg\<close>\<close>, \<open>\<^marker>\<open>contributor arg\<close>\<close>, \<open>\<^marker>\<open>date arg\<close>\<close>, |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
524 |
\<open>\<^marker>\<open>license arg\<close>\<close>, and \<open>\<^marker>\<open>description arg\<close>\<close> produce markup in the PIDE |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
525 |
document, without any immediate effect on typesetting. This vocabulary is |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
526 |
taken from the Dublin Core Metadata |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
527 |
Initiative\<^footnote>\<open>\<^url>\<open>https://www.dublincore.org/specifications/dublin-core/dcmi-terms\<close>\<close>. |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
528 |
The argument is an uninterpreted string, except for @{document_marker |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
529 |
description}, which consists of words that are subject to spell-checking. |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
530 |
|
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
531 |
\<^descr> \<open>\<^marker>\<open>tag name\<close>\<close> updates the list of command tags in the presentation |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
532 |
context: later declarations take precedence, so \<open>\<^marker>\<open>tag a, tag b, tag c\<close>\<close> |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
533 |
produces a reversed list. The default tags are given by the original |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
534 |
\<^theory_text>\<open>keywords\<close> declaration of a command, and the system option |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
535 |
@{system_option_ref document_tags}. |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
536 |
|
70140 | 537 |
The optional \<open>scope\<close> tells how far the tagging is applied to subsequent |
538 |
proof structure: ``\<^theory_text>\<open>("proof")\<close>'' means it applies to the following proof |
|
539 |
text, and ``\<^theory_text>\<open>(command)\<close>'' means it only applies to the current command. |
|
540 |
The default within a proof body is ``\<^theory_text>\<open>("proof")\<close>'', but for toplevel goal |
|
541 |
statements it is ``\<^theory_text>\<open>(command)\<close>''. Thus a \<open>tag\<close> marker for \<^theory_text>\<open>theorem\<close>, |
|
542 |
\<^theory_text>\<open>lemma\<close> etc. does \emph{not} affect its proof by default. |
|
543 |
||
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
544 |
An old-style command tag \<^verbatim>\<open>%\<close>\<open>name\<close> is treated like a document marker |
70140 | 545 |
\<open>\<^marker>\<open>tag (proof) name\<close>\<close>: the list of command tags precedes the list of |
546 |
document markers. The head of the resulting tags in the presentation |
|
547 |
context is turned into {\LaTeX} environments to modify the type-setting. |
|
548 |
The following tags are pre-declared for certain classes of commands, and |
|
549 |
serve as default markup for certain kinds of commands: |
|
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
550 |
|
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
551 |
\<^medskip> |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
552 |
\begin{tabular}{ll} |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
553 |
\<open>document\<close> & document markup commands \\ |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
554 |
\<open>theory\<close> & theory begin/end \\ |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
555 |
\<open>proof\<close> & all proof commands \\ |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
556 |
\<open>ML\<close> & all commands involving ML code \\ |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
557 |
\end{tabular} |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
558 |
\<^medskip> |
27043 | 559 |
|
61624 | 560 |
The Isabelle document preparation system @{cite "isabelle-system"} allows |
561 |
tagged command regions to be presented specifically, e.g.\ to fold proof |
|
562 |
texts, or drop parts of the text completely. |
|
27043 | 563 |
|
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
564 |
For example ``\<^theory_text>\<open>by auto\<close>~\<open>\<^marker>\<open>tag invisible\<close>\<close>'' causes that piece of proof to |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
565 |
be treated as \<open>invisible\<close> instead of \<open>proof\<close> (the default), which may be |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
566 |
shown or hidden depending on the document setup. In contrast, ``\<^theory_text>\<open>by |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
567 |
auto\<close>~\<open>\<^marker>\<open>tag visible\<close>\<close>'' forces this text to be shown invariably. |
27043 | 568 |
|
61624 | 569 |
Explicit tag specifications within a proof apply to all subsequent commands |
69962
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
570 |
of the same level of nesting. For example, ``\<^theory_text>\<open>proof\<close>~\<open>\<^marker>\<open>tag invisible\<close> |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
571 |
\<dots>\<close>~\<^theory_text>\<open>qed\<close>'' forces the whole sub-proof to be typeset as \<open>visible\<close> (unless |
82e945d472d5
documentation of document markers and re-interpreted command tags;
wenzelm
parents:
69597
diff
changeset
|
572 |
some of its parts are tagged differently). |
28750 | 573 |
|
61421 | 574 |
\<^medskip> |
61624 | 575 |
Command tags merely produce certain markup environments for type-setting. |
63680 | 576 |
The meaning of these is determined by {\LaTeX} macros, as defined in |
577 |
\<^file>\<open>~~/lib/texinputs/isabelle.sty\<close> or by the document author. The Isabelle |
|
61624 | 578 |
document preparation tools also provide some high-level options to specify |
579 |
the meaning of arbitrary tags to ``keep'', ``drop'', or ``fold'' the |
|
580 |
corresponding parts of the text. Logic sessions may also specify ``document |
|
581 |
versions'', where given tags are interpreted in some particular way. Again |
|
582 |
see @{cite "isabelle-system"} for further details. |
|
58618 | 583 |
\<close> |
27043 | 584 |
|
585 |
||
58618 | 586 |
section \<open>Railroad diagrams\<close> |
42658 | 587 |
|
58618 | 588 |
text \<open> |
42658 | 589 |
\begin{matharray}{rcl} |
61493 | 590 |
@{antiquotation_def "rail"} & : & \<open>antiquotation\<close> \\ |
42658 | 591 |
\end{matharray} |
592 |
||
69597 | 593 |
\<^rail>\<open> |
59937 | 594 |
'rail' @{syntax text} |
69597 | 595 |
\<close> |
42658 | 596 |
|
61624 | 597 |
The @{antiquotation rail} antiquotation allows to include syntax diagrams |
63680 | 598 |
into Isabelle documents. {\LaTeX} requires the style file |
599 |
\<^file>\<open>~~/lib/texinputs/railsetup.sty\<close>, which can be used via |
|
61503 | 600 |
\<^verbatim>\<open>\usepackage{railsetup}\<close> in \<^verbatim>\<open>root.tex\<close>, for example. |
42658 | 601 |
|
61624 | 602 |
The rail specification language is quoted here as Isabelle @{syntax string} |
603 |
or text @{syntax "cartouche"}; it has its own grammar given below. |
|
42658 | 604 |
|
55120 | 605 |
\begingroup |
61474 | 606 |
\def\isasymnewline{\isatt{\isacharbackslash\isacharless newline\isachargreater}} |
69597 | 607 |
\<^rail>\<open> |
42658 | 608 |
rule? + ';' |
609 |
; |
|
610 |
rule: ((identifier | @{syntax antiquotation}) ':')? body |
|
611 |
; |
|
612 |
body: concatenation + '|' |
|
613 |
; |
|
614 |
concatenation: ((atom '?'?) +) (('*' | '+') atom?)? |
|
615 |
; |
|
616 |
atom: '(' body? ')' | identifier | |
|
617 |
'@'? (string | @{syntax antiquotation}) | |
|
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
55029
diff
changeset
|
618 |
'\<newline>' |
69597 | 619 |
\<close> |
55120 | 620 |
\endgroup |
42658 | 621 |
|
63138
70f4d67235a0
clarified syntax category names according to Isabelle/ML/Scala;
wenzelm
parents:
63120
diff
changeset
|
622 |
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
|
623 |
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
|
624 |
instead of double quotes of the standard @{syntax string} category. |
42658 | 625 |
|
61624 | 626 |
Each \<open>rule\<close> defines a formal language (with optional name), using a notation |
627 |
that is similar to EBNF or regular expressions with recursion. The meaning |
|
628 |
and visual appearance of these rail language elements is illustrated by the |
|
629 |
following representative examples. |
|
42658 | 630 |
|
61503 | 631 |
\<^item> Empty \<^verbatim>\<open>()\<close> |
42658 | 632 |
|
69597 | 633 |
\<^rail>\<open>()\<close> |
42658 | 634 |
|
61503 | 635 |
\<^item> Nonterminal \<^verbatim>\<open>A\<close> |
42658 | 636 |
|
69597 | 637 |
\<^rail>\<open>A\<close> |
42658 | 638 |
|
61503 | 639 |
\<^item> Nonterminal via Isabelle antiquotation \<^verbatim>\<open>@{syntax method}\<close> |
42658 | 640 |
|
69597 | 641 |
\<^rail>\<open>@{syntax method}\<close> |
42658 | 642 |
|
61503 | 643 |
\<^item> Terminal \<^verbatim>\<open>'xyz'\<close> |
42658 | 644 |
|
69597 | 645 |
\<^rail>\<open>'xyz'\<close> |
42658 | 646 |
|
61503 | 647 |
\<^item> Terminal in keyword style \<^verbatim>\<open>@'xyz'\<close> |
42658 | 648 |
|
69597 | 649 |
\<^rail>\<open>@'xyz'\<close> |
42658 | 650 |
|
61503 | 651 |
\<^item> Terminal via Isabelle antiquotation \<^verbatim>\<open>@@{method rule}\<close> |
42658 | 652 |
|
69597 | 653 |
\<^rail>\<open>@@{method rule}\<close> |
42658 | 654 |
|
61503 | 655 |
\<^item> Concatenation \<^verbatim>\<open>A B C\<close> |
42658 | 656 |
|
69597 | 657 |
\<^rail>\<open>A B C\<close> |
42658 | 658 |
|
61503 | 659 |
\<^item> Newline inside concatenation \<^verbatim>\<open>A B C \<newline> D E F\<close> |
42658 | 660 |
|
69597 | 661 |
\<^rail>\<open>A B C \<newline> D E F\<close> |
42658 | 662 |
|
61503 | 663 |
\<^item> Variants \<^verbatim>\<open>A | B | C\<close> |
42658 | 664 |
|
69597 | 665 |
\<^rail>\<open>A | B | C\<close> |
42658 | 666 |
|
61503 | 667 |
\<^item> Option \<^verbatim>\<open>A ?\<close> |
42658 | 668 |
|
69597 | 669 |
\<^rail>\<open>A ?\<close> |
42658 | 670 |
|
61503 | 671 |
\<^item> Repetition \<^verbatim>\<open>A *\<close> |
42658 | 672 |
|
69597 | 673 |
\<^rail>\<open>A *\<close> |
42658 | 674 |
|
61503 | 675 |
\<^item> Repetition with separator \<^verbatim>\<open>A * sep\<close> |
42658 | 676 |
|
69597 | 677 |
\<^rail>\<open>A * sep\<close> |
42658 | 678 |
|
61503 | 679 |
\<^item> Strict repetition \<^verbatim>\<open>A +\<close> |
42658 | 680 |
|
69597 | 681 |
\<^rail>\<open>A +\<close> |
42658 | 682 |
|
61503 | 683 |
\<^item> Strict repetition with separator \<^verbatim>\<open>A + sep\<close> |
42658 | 684 |
|
69597 | 685 |
\<^rail>\<open>A + sep\<close> |
58618 | 686 |
\<close> |
42658 | 687 |
|
27043 | 688 |
end |