src/Doc/Datatypes/Datatypes.thy
changeset 55029 61a6bf7d4b02
parent 54958 4933165fd112
child 55073 9b96fb4c8cfd
child 55112 b1a5d603fd12
--- a/src/Doc/Datatypes/Datatypes.thy	Fri Jan 17 18:12:35 2014 +0100
+++ b/src/Doc/Datatypes/Datatypes.thy	Fri Jan 17 20:20:20 2014 +0100
@@ -458,7 +458,7 @@
 \end{matharray}
 
 @{rail "
-  @@{command datatype_new} target? @{syntax dt_options}? \\
+  @@{command datatype_new} target? @{syntax dt_options}? \<newline>
     (@{syntax dt_name} '=' (@{syntax ctor} + '|') + @'and')
   ;
   @{syntax_def dt_options}: '(' (('no_discs_sels' | 'no_code' | 'rep_compat') + ',') ')'
@@ -511,7 +511,7 @@
 mention exactly the same type variables in the same order.
 
 @{rail "
-  @{syntax_def ctor}: (name ':')? name (@{syntax ctor_arg} * ) \\
+  @{syntax_def ctor}: (name ':')? name (@{syntax ctor_arg} * ) \<newline>
     @{syntax dt_sel_defaults}? mixfix?
 "}
 
@@ -1353,7 +1353,7 @@
 \end{matharray}
 
 @{rail "
-  @@{command primrec_new} target? fixes \\ @'where' (@{syntax pr_equation} + '|')
+  @@{command primrec_new} target? fixes \<newline> @'where' (@{syntax pr_equation} + '|')
   ;
   @{syntax_def pr_equation}: thmdecl? prop
 "}
@@ -1575,7 +1575,7 @@
 \end{matharray}
 
 @{rail "
-  @@{command codatatype} target? \\
+  @@{command codatatype} target? \<newline>
     (@{syntax dt_name} '=' (@{syntax ctor} + '|') + @'and')
 "}
 
@@ -2242,7 +2242,8 @@
 \end{matharray}
 
 @{rail "
-  (@@{command primcorec} | @@{command primcorecursive}) target? \\ @{syntax pcr_option}? fixes @'where'
+  (@@{command primcorec} | @@{command primcorecursive}) target? \<newline>
+    @{syntax pcr_option}? fixes @'where'
     (@{syntax pcr_formula} + '|')
   ;
   @{syntax_def pcr_option}: '(' ('sequential' | 'exhaustive') ')'
@@ -2325,8 +2326,8 @@
 \end{matharray}
 
 @{rail "
-  @@{command bnf} target? (name ':')? typ \\
-    'map:' term ('sets:' (term +))? 'bd:' term \\
+  @@{command bnf} target? (name ':')? typ \<newline>
+    'map:' term ('sets:' (term +))? 'bd:' term \<newline>
     ('wits:' (term +))? ('rel:' term)?
 "}
 *}
@@ -2416,7 +2417,7 @@
 \end{matharray}
 
 @{rail "
-  @@{command wrap_free_constructors} target? @{syntax dt_options} \\
+  @@{command wrap_free_constructors} target? @{syntax dt_options} \<newline>
     term_list name @{syntax wfc_discs_sels}?
   ;
   @{syntax_def wfc_discs_sels}: name_list (name_list_list name_term_list_list? )?