src/Doc/Isar_Ref/Outer_Syntax.thy
changeset 63139 d905741a80e8
parent 63138 70f4d67235a0
child 63140 0644c2e5a989
equal deleted inserted replaced
63138:70f4d67235a0 63139:d905741a80e8
   236   admitted as well. A marginal @{syntax comment} is of the form \<^verbatim>\<open>--\<close>~@{syntax
   236   admitted as well. A marginal @{syntax comment} is of the form \<^verbatim>\<open>--\<close>~@{syntax
   237   text} or \<^verbatim>\<open>\<comment>\<close>~@{syntax text}. Any number of these may occur within
   237   text} or \<^verbatim>\<open>\<comment>\<close>~@{syntax text}. Any number of these may occur within
   238   Isabelle/Isar commands.
   238   Isabelle/Isar commands.
   239 
   239 
   240   @{rail \<open>
   240   @{rail \<open>
   241     @{syntax_def text}: @{syntax verbatim} | @{syntax cartouche} | @{syntax name}
   241     @{syntax_def text}: @{syntax embedded} | @{syntax verbatim}
   242     ;
   242     ;
   243     @{syntax_def comment}: ('--' | @'\<comment>') @{syntax text}
   243     @{syntax_def comment}: ('--' | @'\<comment>') @{syntax text}
   244   \<close>}
   244   \<close>}
   245 \<close>
   245 \<close>
   246 
   246