diff -r 038458a4d11b -r a2659fbb3b13 src/Doc/Tutorial/Documents/Documents.thy --- a/src/Doc/Tutorial/Documents/Documents.thy Thu Aug 08 17:04:02 2013 +0200 +++ b/src/Doc/Tutorial/Documents/Documents.thy Thu Aug 08 17:24:31 2013 +0200 @@ -121,17 +121,16 @@ @{text "\"} (\verb+\+\verb++), @{text "\"} (\verb+\+\verb++), etc. (excluding @{text "\"}), special letters like @{text "\"} (\verb+\+\verb++) and @{text - "\"} (\verb+\+\verb++), and the control symbols - \verb+\+\verb+<^isub>+ and \verb+\+\verb+<^isup>+ for single letter - sub and super scripts. This means that the input + "\"} (\verb+\+\verb++). Moreover the control symbol + \verb+\+\verb+<^sub>+ may be used to subscript a single letter or digit + in the trailing part of an identifier. This means that the input \medskip - {\small\noindent \verb,\,\verb,\,\verb,\<^isub>1.,~\verb,\,\verb,\<^isub>1 = \,\verb,\<^isup>\,} + {\small\noindent \verb,\,\verb,\,\verb,\<^isub>1.,~\verb,\,\verb,\<^isub>1 = \,\verb,\<^isub>\,} \medskip - \noindent is recognized as the term @{term "\\\<^isub>1. \\<^isub>1 = \\<^isup>\"} - by Isabelle. Note that @{text "\\<^isup>\"} is a single - syntactic entity, not an exponentiation. + \noindent is recognized as the term @{term "\\\<^isub>1. \\<^isub>1 = \\<^isub>\"} + by Isabelle. Replacing our previous definition of @{text xor} by the following specifies an Isabelle symbol for the new operator: