src/Doc/System/Sessions.thy
changeset 66970 13857f49d215
parent 66916 aca50a1572c5
child 66971 43b2aac6053c
--- a/src/Doc/System/Sessions.thy	Tue Oct 31 22:17:38 2017 +0100
+++ b/src/Doc/System/Sessions.thy	Wed Nov 01 12:28:20 2017 +0100
@@ -55,7 +55,7 @@
     @{syntax_def session_entry}: @'session' spec '='
       (@{syntax system_name} '+')? body
     ;
-    body: description? options? (theories+) \<newline> (document_files*)
+    body: description? options? (sessions?) (theories*) \<newline> (document_files*)
     ;
     spec: @{syntax system_name} groups? dir?
     ;
@@ -73,7 +73,7 @@
     ;
     sessions: @'sessions' (@{syntax system_name}+)
     ;
-    theories: @'theories' opts? (theory_entry*)
+    theories: @'theories' opts? (theory_entry+)
     ;
     theory_entry: @{syntax system_name} ('(' @'global' ')')?
     ;