doc-src/IsarRef/Thy/Inner_Syntax.thy
changeset 42705 528a2ba8fa74
parent 42669 04dfffda5671
child 42926 a8b655d089ac
equal deleted inserted replaced
42704:3f19e324ff59 42705:528a2ba8fa74
   246       @{syntax string} @{syntax nat} ')'
   246       @{syntax string} @{syntax nat} ')'
   247     ;
   247     ;
   248     @{syntax_def mixfix}: @{syntax \"infix\"} | '(' @{syntax string} prios? @{syntax nat}? ')' |
   248     @{syntax_def mixfix}: @{syntax \"infix\"} | '(' @{syntax string} prios? @{syntax nat}? ')' |
   249     '(' @'binder' @{syntax string} prios? @{syntax nat} ')'
   249     '(' @'binder' @{syntax string} prios? @{syntax nat} ')'
   250     ;
   250     ;
   251     @{syntax_def structmixfix}: @{syntax mixfix} | '(' @'structure' ')'
   251     @{syntax_def struct_mixfix}: @{syntax mixfix} | '(' @'structure' ')'
   252     ;
   252     ;
   253 
   253 
   254     prios: '[' (@{syntax nat} + ',') ']'
   254     prios: '[' (@{syntax nat} + ',') ']'
   255   "}
   255   "}
   256 
   256 
   364   @{rail "
   364   @{rail "
   365     (@@{command type_notation} | @@{command no_type_notation}) @{syntax target}?
   365     (@@{command type_notation} | @@{command no_type_notation}) @{syntax target}?
   366       @{syntax mode}? \\ (@{syntax nameref} @{syntax mixfix} + @'and')
   366       @{syntax mode}? \\ (@{syntax nameref} @{syntax mixfix} + @'and')
   367     ;
   367     ;
   368     (@@{command notation} | @@{command no_notation}) @{syntax target}? @{syntax mode}? \\
   368     (@@{command notation} | @@{command no_notation}) @{syntax target}? @{syntax mode}? \\
   369       (@{syntax nameref} @{syntax structmixfix} + @'and')
   369       (@{syntax nameref} @{syntax struct_mixfix} + @'and')
   370     ;
   370     ;
   371     @@{command write} @{syntax mode}? (@{syntax nameref} @{syntax structmixfix} + @'and')
   371     @@{command write} @{syntax mode}? (@{syntax nameref} @{syntax struct_mixfix} + @'and')
   372   "}
   372   "}
   373 
   373 
   374   \begin{description}
   374   \begin{description}
   375 
   375 
   376   \item @{command "type_notation"}~@{text "c (mx)"} associates mixfix
   376   \item @{command "type_notation"}~@{text "c (mx)"} associates mixfix