src/Doc/Isar_Ref/Outer_Syntax.thy
changeset 63137 9553f11d67c4
parent 63120 629a4c5e953e
child 63138 70f4d67235a0
equal deleted inserted replaced
63136:fd11a538daac 63137:9553f11d67c4
   220   content without delimiters.
   220   content without delimiters.
   221 
   221 
   222   @{rail \<open>
   222   @{rail \<open>
   223     @{syntax_def embedded}: @{syntax cartouche} | @{syntax string} |
   223     @{syntax_def embedded}: @{syntax cartouche} | @{syntax string} |
   224       @{syntax ident} | @{syntax longident} | @{syntax symident} |
   224       @{syntax ident} | @{syntax longident} | @{syntax symident} |
   225       @{syntax nat}
   225       @{syntax var} | @{syntax typefree} | @{syntax typevar} | @{syntax nat}
   226   \<close>}
   226   \<close>}
   227 \<close>
   227 \<close>
   228 
   228 
   229 
   229 
   230 subsection \<open>Comments \label{sec:comments}\<close>
   230 subsection \<open>Comments \label{sec:comments}\<close>
   276   symbolic identifiers (e.g.\ \<^verbatim>\<open>++\<close> or \<open>\<forall>\<close> are available as well, provided
   276   symbolic identifiers (e.g.\ \<^verbatim>\<open>++\<close> or \<open>\<forall>\<close> are available as well, provided
   277   these have not been superseded by commands or other keywords already (such
   277   these have not been superseded by commands or other keywords already (such
   278   as \<^verbatim>\<open>=\<close> or \<^verbatim>\<open>+\<close>).
   278   as \<^verbatim>\<open>=\<close> or \<^verbatim>\<open>+\<close>).
   279 
   279 
   280   @{rail \<open>
   280   @{rail \<open>
   281     @{syntax_def type}: @{syntax embedded} | @{syntax typefree} |
   281     @{syntax_def type}: @{syntax embedded}
   282       @{syntax typevar}
   282     ;
   283     ;
   283     @{syntax_def term}: @{syntax embedded}
   284     @{syntax_def term}: @{syntax embedded} | @{syntax var}
   284     ;
   285     ;
   285     @{syntax_def prop}: @{syntax embedded}
   286     @{syntax_def prop}: @{syntax term}
       
   287   \<close>}
   286   \<close>}
   288 
   287 
   289   Positional instantiations are specified as a sequence of terms, or the
   288   Positional instantiations are specified as a sequence of terms, or the
   290   placeholder ``\<open>_\<close>'' (underscore), which means to skip a position.
   289   placeholder ``\<open>_\<close>'' (underscore), which means to skip a position.
   291 
   290