equal
deleted
inserted
replaced
193 @@{antiquotation ML_structure} options @{syntax text} | |
193 @@{antiquotation ML_structure} options @{syntax text} | |
194 @@{antiquotation ML_functor} options @{syntax text} | |
194 @@{antiquotation ML_functor} options @{syntax text} | |
195 @@{antiquotation emph} options @{syntax text} | |
195 @@{antiquotation emph} options @{syntax text} | |
196 @@{antiquotation bold} options @{syntax text} | |
196 @@{antiquotation bold} options @{syntax text} | |
197 @@{antiquotation verbatim} options @{syntax text} | |
197 @@{antiquotation verbatim} options @{syntax text} | |
|
198 @@{antiquotation path} options @{syntax name} | |
198 @@{antiquotation "file"} options @{syntax name} | |
199 @@{antiquotation "file"} options @{syntax name} | |
199 @@{antiquotation file_unchecked} options @{syntax name} | |
200 @@{antiquotation dir} options @{syntax name} | |
200 @@{antiquotation url} options @{syntax embedded} | |
201 @@{antiquotation url} options @{syntax embedded} | |
201 @@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and') |
202 @@{antiquotation cite} options @{syntax cartouche}? (@{syntax name} + @'and') |
202 ; |
203 ; |
203 styles: '(' (style + ',') ')' |
204 styles: '(' (style + ',') ')' |
204 ; |
205 ; |
281 \<^verbatim>\<open>\textbf{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>. |
282 \<^verbatim>\<open>\textbf{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>. |
282 |
283 |
283 \<^descr> \<open>@{verbatim s}\<close> prints uninterpreted source text literally as ASCII |
284 \<^descr> \<open>@{verbatim s}\<close> prints uninterpreted source text literally as ASCII |
284 characters, using some type-writer font style. |
285 characters, using some type-writer font style. |
285 |
286 |
286 \<^descr> \<open>@{file path}\<close> checks that \<open>path\<close> refers to a file (or directory) and |
287 \<^descr> \<open>@{path name}\<close> prints the file-system path name verbatim. |
287 prints it verbatim. |
288 |
288 |
289 \<^descr> \<open>@{file name}\<close> is like \<open>@{path name}\<close>, but ensures that \<open>name\<close> refers to a |
289 \<^descr> \<open>@{file_unchecked path}\<close> is like \<open>@{file path}\<close>, but does not check the |
290 plain file. |
290 existence of the \<open>path\<close> within the file-system. |
291 |
|
292 \<^descr> \<open>@{dir name}\<close> is like \<open>@{path name}\<close>, but ensures that \<open>name\<close> refers to a |
|
293 directory. |
291 |
294 |
292 \<^descr> \<open>@{url name}\<close> produces markup for the given URL, which results in an |
295 \<^descr> \<open>@{url name}\<close> produces markup for the given URL, which results in an |
293 active hyperlink within the text. |
296 active hyperlink within the text. |
294 |
297 |
295 \<^descr> \<open>@{cite name}\<close> produces a citation \<^verbatim>\<open>\cite{name}\<close> in {\LaTeX}, where the |
298 \<^descr> \<open>@{cite name}\<close> produces a citation \<^verbatim>\<open>\cite{name}\<close> in {\LaTeX}, where the |