doc-src/IsarRef/Thy/Document_Preparation.thy
changeset 32892 9742f6130f10
parent 32891 d403b99287ff
child 32898 e871d897969c
--- a/doc-src/IsarRef/Thy/Document_Preparation.thy	Thu Oct 08 15:16:13 2009 +0200
+++ b/doc-src/IsarRef/Thy/Document_Preparation.thy	Thu Oct 08 15:59:15 2009 +0200
@@ -201,9 +201,9 @@
     ;
     option: name | name '=' name
     ;
-    styles: '(' (style * ',') ')'
+    styles: '(' (style + ',') ')'
     ;
-    style: (name *)
+    style: (name +)
     ;
   \end{rail}