diff -r c98c6eb3dd4c -r dbb1f02e667d src/Doc/Isar_Ref/Inner_Syntax.thy --- a/src/Doc/Isar_Ref/Inner_Syntax.thy Tue Jan 16 11:30:03 2018 +0100 +++ b/src/Doc/Isar_Ref/Inner_Syntax.thy Tue Jan 16 15:42:21 2018 +0100 @@ -567,7 +567,6 @@ @{syntax_def (inner) str_token} & = & \<^verbatim>\''\ \\\ \<^verbatim>\''\ \\ @{syntax_def (inner) string_token} & = & \<^verbatim>\"\ \\\ \<^verbatim>\"\ \\ @{syntax_def (inner) cartouche} & = & @{verbatim "\"} \\\ @{verbatim "\"} \\ - @{syntax_def (inner) comment_cartouche} & = & @{verbatim "\ \"} \\\ @{verbatim "\"} \\ \end{supertabular} \end{center} @@ -582,10 +581,8 @@ (inner) float_const}, provide robust access to the respective tokens: the syntax tree holds a syntactic constant instead of a free variable. - A @{syntax (inner) comment_cartouche} resembles the outer syntax notation - for marginal @{syntax_ref comment} (\secref{sec:comments}), but is - syntactically more restrictive: only the symbol-form with \<^verbatim>\\\ and text - cartouche is supported. + Formal document comments (\secref{sec:comments}) may be also used within the + inner syntax. \