src/Doc/System/Sessions.thy
changeset 65374 a5b38d8d3c1e
parent 64308 b00508facb4f
child 65504 b80477da30eb
--- a/src/Doc/System/Sessions.thy	Tue Apr 04 19:51:56 2017 +0200
+++ b/src/Doc/System/Sessions.thy	Tue Apr 04 21:05:07 2017 +0200
@@ -70,7 +70,9 @@
     ;
     value: @{syntax name} | @{syntax real}
     ;
-    theories: @'theories' opts? ( @{syntax name} * )
+    theory_entry: @{syntax name} ('(' @'global' ')')?
+    ;
+    theories: @'theories' opts? (theory_entry*)
     ;
     files: @'files' (@{syntax name}+)
     ;
@@ -116,6 +118,11 @@
   of \isakeyword{theories} may be given. Options are only active for each
   \isakeyword{theories} block separately.
 
+  A theory name that is followed by \<open>(\<close>\isakeyword{global}\<open>)\<close> is treated
+  literally in other session specifications or theory imports. In contrast,
+  the default is to qualify theory names by the session name, in order to
+  ensure globally unique names in big session trees.
+
   \<^descr> \isakeyword{files}~\<open>files\<close> lists additional source files that are involved
   in the processing of this session. This should cover anything outside the
   formal content of the theory sources. In contrast, files that are loaded