src/Doc/Datatypes/Datatypes.thy
changeset 53828 408c9a3617e3
parent 53826 92a8ae172242
child 53829 92e71eb22ebe
--- a/src/Doc/Datatypes/Datatypes.thy	Tue Sep 24 16:59:14 2013 +0200
+++ b/src/Doc/Datatypes/Datatypes.thy	Tue Sep 24 17:06:06 2013 +0200
@@ -2023,10 +2023,10 @@
 Primitive corecursive definitions have the following general syntax:
 
 @{rail "
-  (@@{command_def primcorec} | @@{command_def primcorecursive}) target? @{syntax pcr_option}? fixes \\ @'where'
+  (@@{command_def primcorec} | @@{command_def primcorecursive}) target? \\ @{syntax pcr_option}? fixes @'where'
     (@{syntax pcr_formula} + '|')
   ;
-  @{syntax_def pcr_option}: '(' 'sequential' | 'exhaustive' ')'
+  @{syntax_def pcr_option}: '(' ('sequential' | 'exhaustive') ')'
   ;
   @{syntax_def pcr_formula}: thmdecl? prop (@'of' (term * ))?
 "}