src/Doc/Isar_Ref/Document_Preparation.thy
changeset 63138 70f4d67235a0
parent 63120 629a4c5e953e
child 63531 847eefdca90d
equal deleted inserted replaced
63137:9553f11d67c4 63138:70f4d67235a0
   460   to indicate some modification in the way it is printed in the document.
   460   to indicate some modification in the way it is printed in the document.
   461 
   461 
   462   @{rail \<open>
   462   @{rail \<open>
   463     @{syntax_def tags}: ( tag * )
   463     @{syntax_def tags}: ( tag * )
   464     ;
   464     ;
   465     tag: '%' (@{syntax ident} | @{syntax string})
   465     tag: '%' (@{syntax short_ident} | @{syntax string})
   466   \<close>}
   466   \<close>}
   467 
   467 
   468   Some tags are pre-declared for certain classes of commands, serving as
   468   Some tags are pre-declared for certain classes of commands, serving as
   469   default markup if no tags are given in the text:
   469   default markup if no tags are given in the text:
   470 
   470 
   536     '@'? (string | @{syntax antiquotation}) |
   536     '@'? (string | @{syntax antiquotation}) |
   537     '\<newline>'
   537     '\<newline>'
   538   \<close>}
   538   \<close>}
   539   \endgroup
   539   \endgroup
   540 
   540 
   541   The lexical syntax of \<open>identifier\<close> coincides with that of @{syntax ident} in
   541   The lexical syntax of \<open>identifier\<close> coincides with that of @{syntax
   542   regular Isabelle syntax, but \<open>string\<close> uses single quotes instead of double
   542   short_ident} in regular Isabelle syntax, but \<open>string\<close> uses single quotes
   543   quotes of the standard @{syntax string} category.
   543   instead of double quotes of the standard @{syntax string} category.
   544 
   544 
   545   Each \<open>rule\<close> defines a formal language (with optional name), using a notation
   545   Each \<open>rule\<close> defines a formal language (with optional name), using a notation
   546   that is similar to EBNF or regular expressions with recursion. The meaning
   546   that is similar to EBNF or regular expressions with recursion. The meaning
   547   and visual appearance of these rail language elements is illustrated by the
   547   and visual appearance of these rail language elements is illustrated by the
   548   following representative examples.
   548   following representative examples.