src/Doc/System/Environment.thy
changeset 68541 12b4b3bc585d
parent 68523 ccacc84e0251
child 69593 3dda49e08b9d
--- a/src/Doc/System/Environment.thy	Fri Jun 29 15:54:41 2018 +0200
+++ b/src/Doc/System/Environment.thy	Fri Jun 29 16:45:54 2018 +0200
@@ -407,6 +407,7 @@
 
   Options are:
     -d DIR       include session directory
+    -i NAME      include session in name-space of theories
     -l NAME      logic session name (default ISABELLE_LOGIC)
     -m MODE      add print mode for output
     -n           no build of session image on startup
@@ -421,6 +422,9 @@
   Option \<^verbatim>\<open>-l\<close> specifies the logic session name. By default, its heap image is
   checked and built on demand, but the option \<^verbatim>\<open>-n\<close> skips that.
 
+  Option \<^verbatim>\<open>-i\<close> includes additional sessions into the name-space of theories:
+  multiple occurrences are possible.
+
   Option \<^verbatim>\<open>-r\<close> indicates a bootstrap from the raw Poly/ML system, which is
   relevant for Isabelle/Pure development.