diff -r 6437c989a744 -r 7e0178c84994 src/Doc/Isar_Ref/Outer_Syntax.thy --- a/src/Doc/Isar_Ref/Outer_Syntax.thy Wed Apr 09 17:29:37 2014 +0200 +++ b/src/Doc/Isar_Ref/Outer_Syntax.thy Wed Apr 09 17:54:09 2014 +0200 @@ -265,14 +265,14 @@ text {* Large chunks of plain @{syntax text} are usually given @{syntax verbatim}, i.e.\ enclosed in @{verbatim "{"}@{verbatim - "*"}~@{text "\"}~@{verbatim "*"}@{verbatim "}"}. For convenience, - any of the smaller text units conforming to @{syntax nameref} are - admitted as well. A marginal @{syntax comment} is of the form - @{verbatim "--"}~@{syntax text}. Any number of these may occur - within Isabelle/Isar commands. + "*"}~@{text "\"}~@{verbatim "*"}@{verbatim "}"}, or as @{syntax + cartouche} @{text "\\\"}. For convenience, any of the smaller text + units conforming to @{syntax nameref} are admitted as well. A + marginal @{syntax comment} is of the form @{verbatim "--"}~@{syntax + text}. Any number of these may occur within Isabelle/Isar commands. @{rail \ - @{syntax_def text}: @{syntax verbatim} | @{syntax nameref} + @{syntax_def text}: @{syntax verbatim} | @{syntax cartouche} | @{syntax nameref} ; @{syntax_def comment}: '--' @{syntax text} \} @@ -424,9 +424,9 @@ \item selections from named facts @{text "a(i)"} or @{text "a(j - k)"}, - \item literal fact propositions using @{syntax_ref altstring} syntax - @{verbatim "`"}@{text "\"}@{verbatim "`"} (see also method - @{method_ref fact}). + \item literal fact propositions using token syntax @{syntax_ref altstring} + @{verbatim "`"}@{text "\"}@{verbatim "`"} or @{syntax_ref cartouche} + @{text "\\\"} (see also method @{method_ref fact}). \end{enumerate} @@ -451,7 +451,8 @@ @{syntax_def thmdef}: thmbind '=' ; @{syntax_def thmref}: - (@{syntax nameref} selection? | @{syntax altstring}) @{syntax attributes}? | + (@{syntax nameref} selection? | @{syntax altstring} | @{syntax cartouche}) + @{syntax attributes}? | '[' @{syntax attributes} ']' ; @{syntax_def thmrefs}: @{syntax thmref} +