doc-src/System/Thy/Sessions.thy
changeset 48916 f45ccc0d1ace
parent 48903 1621b3f26095
--- a/doc-src/System/Thy/Sessions.thy	Thu Aug 23 21:23:14 2012 +0200
+++ b/doc-src/System/Thy/Sessions.thy	Fri Aug 24 11:03:52 2012 +0200
@@ -48,7 +48,7 @@
   @{rail "
     @{syntax_def session_entry}: @'session' spec '=' (@{syntax name} '+')? body
     ;
-    body: description? options? ( theories * ) files?
+    body: description? options? ( theories + ) files?
     ;
     spec: @{syntax name} groups? dir?
     ;