diff -r 760e21900b01 -r 28e788ca2c5d src/Doc/Isar_Ref/Symbols.thy --- a/src/Doc/Isar_Ref/Symbols.thy Thu Oct 22 21:16:27 2015 +0200 +++ b/src/Doc/Isar_Ref/Symbols.thy Thu Oct 22 21:16:49 2015 +0200 @@ -6,25 +6,24 @@ text \ Isabelle supports an infinite number of non-ASCII symbols, which are - represented in source text as @{verbatim \\\}@{verbatim "<"}\name\@{verbatim ">"} (where \name\ may be any identifier). It + represented in source text as \<^verbatim>\\\\<^verbatim>\<\\name\\<^verbatim>\>\ (where \name\ may be any identifier). It is left to front-end tools how to present these symbols to the user. The collection of predefined standard symbols given below is available by default for Isabelle document output, due to - appropriate definitions of @{verbatim \\isasym\}\name\ for each @{verbatim \\\}@{verbatim "<"}\name\@{verbatim - ">"} in the @{verbatim isabellesym.sty} file. Most of these symbols + appropriate definitions of \<^verbatim>\\isasym\\name\ for each \<^verbatim>\\\\<^verbatim>\<\\name\\<^verbatim>\>\ in + the \<^verbatim>\isabellesym.sty\ file. Most of these symbols are displayed properly in Isabelle/jEdit and {\LaTeX} generated from Isabelle. Moreover, any single symbol (or ASCII character) may be prefixed by - @{verbatim "\<^sup>"} for superscript and @{verbatim "\<^sub>"} for subscript, - such as @{verbatim "A\<^sup>\"} for \A\<^sup>\\ and @{verbatim "A\<^sub>1"} for + \<^verbatim>\\<^sup>\ for superscript and \<^verbatim>\\<^sub>\ for subscript, + such as \<^verbatim>\A\<^sup>\\ for \A\<^sup>\\ and \<^verbatim>\A\<^sub>1\ for \A\<^sub>1\. Sub- and superscripts that span a region of text can - be marked up with @{verbatim "\<^bsub>"}\\\@{verbatim - "\<^esub>"} and @{verbatim "\<^bsup>"}\\\@{verbatim "\<^esup>"} + be marked up with \<^verbatim>\\<^bsub>\\\\\<^verbatim>\\<^esub>\ and \<^verbatim>\\<^bsup>\\\\\<^verbatim>\\<^esup>\ respectively, but note that there are limitations in the typographic rendering quality of this form. Furthermore, all ASCII characters and most other symbols may be printed in bold by prefixing - @{verbatim "\<^bold>"} such as @{verbatim "\<^bold>\"} for \\<^bold>\\. Note that - @{verbatim "\<^sup>"}, @{verbatim "\<^sub>"}, @{verbatim "\<^bold>"} cannot be combined. + \<^verbatim>\\<^bold>\ such as \<^verbatim>\\<^bold>\\ for \\<^bold>\\. Note that + \<^verbatim>\\<^sup>\, \<^verbatim>\\<^sub>\, \<^verbatim>\\<^bold>\ cannot be combined. Further details of Isabelle document preparation are covered in \chref{ch:document-prep}.