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