diff -r aa1fe1103ab8 -r b87784e19a77 src/Doc/Implementation/ML.thy --- a/src/Doc/Implementation/ML.thy Thu Sep 22 00:12:17 2016 +0200 +++ b/src/Doc/Implementation/ML.thy Thu Sep 22 11:25:27 2016 +0200 @@ -1217,13 +1217,6 @@ \<^enum> a control symbol ``\<^verbatim>\\<^ident>\'', for example ``\<^verbatim>\\<^bold>\'', - \<^enum> a raw symbol ``\<^verbatim>\\\\<^verbatim>\<^raw:\\text\\<^verbatim>\>\'' where \text\ consists of - printable characters excluding ``\<^verbatim>\.\'' and ``\<^verbatim>\>\'', for example - ``\<^verbatim>\\<^raw:$\sum_{i = 1}^n$>\'', - - \<^enum> a numbered raw control symbol ``\<^verbatim>\\\\<^verbatim>\<^raw\\n\\<^verbatim>\>\, where \n\ consists - of digits, for example ``\<^verbatim>\\<^raw42>\''. - The \ident\ syntax for symbol names is \letter (letter | digit)\<^sup>*\, where \letter = A..Za..z\ and \digit = 0..9\. There are infinitely many regular symbols and control symbols, but a fixed collection of standard symbols is @@ -1275,7 +1268,7 @@ \<^descr> Type @{ML_type "Symbol.sym"} is a concrete datatype that represents the different kinds of symbols explicitly, with constructors @{ML "Symbol.Char"}, @{ML "Symbol.UTF8"}, @{ML "Symbol.Sym"}, @{ML - "Symbol.Control"}, @{ML "Symbol.Raw"}, @{ML "Symbol.Malformed"}. + "Symbol.Control"}, @{ML "Symbol.Malformed"}. \<^descr> @{ML "Symbol.decode"} converts the string representation of a symbol into the datatype version.