src/Doc/IsarRef/Document_Preparation.thy
changeset 55120 68a829b7f1a4
parent 55113 497693486858
child 55837 154855d9a564
equal deleted inserted replaced
55119:9ca72949ebac 55120:68a829b7f1a4
   466   @{file "~~/lib/texinputs/pdfsetup.sty"}, which can be used via
   466   @{file "~~/lib/texinputs/pdfsetup.sty"}, which can be used via
   467   @{verbatim "\\usepackage{pdfsetup}"} in @{verbatim "root.tex"}, for
   467   @{verbatim "\\usepackage{pdfsetup}"} in @{verbatim "root.tex"}, for
   468   example.
   468   example.
   469 
   469 
   470   The rail specification language is quoted here as Isabelle @{syntax
   470   The rail specification language is quoted here as Isabelle @{syntax
   471   string}; it has its own grammar given below.
   471   string} or text @{syntax "cartouche"}; it has its own grammar given
   472 
   472   below.
       
   473 
       
   474   \begingroup
       
   475   \def\isasymnewline{\isatext{\tt\isacharbackslash<newline>}}
   473   @{rail \<open>
   476   @{rail \<open>
   474   rule? + ';'
   477   rule? + ';'
   475   ;
   478   ;
   476   rule: ((identifier | @{syntax antiquotation}) ':')? body
   479   rule: ((identifier | @{syntax antiquotation}) ':')? body
   477   ;
   480   ;
   481   ;
   484   ;
   482   atom: '(' body? ')' | identifier |
   485   atom: '(' body? ')' | identifier |
   483     '@'? (string | @{syntax antiquotation}) |
   486     '@'? (string | @{syntax antiquotation}) |
   484     '\<newline>'
   487     '\<newline>'
   485   \<close>}
   488   \<close>}
       
   489   \endgroup
   486 
   490 
   487   The lexical syntax of @{text "identifier"} coincides with that of
   491   The lexical syntax of @{text "identifier"} coincides with that of
   488   @{syntax ident} in regular Isabelle syntax, but @{text string} uses
   492   @{syntax ident} in regular Isabelle syntax, but @{text string} uses
   489   single quotes instead of double quotes of the standard @{syntax
   493   single quotes instead of double quotes of the standard @{syntax
   490   string} category.
   494   string} category.