src/Doc/System/Environment.thy
changeset 62677 0df43889f496
parent 62643 6f7ac44365d7
child 62829 4141c2a8458b
--- a/src/Doc/System/Environment.thy	Fri Mar 18 22:15:51 2016 +0100
+++ b/src/Doc/System/Environment.thy	Fri Mar 18 22:19:46 2016 +0100
@@ -305,6 +305,7 @@
 \<open>Usage: isabelle process [OPTIONS]
 
   Options are:
+    -T THEORY    load theory
     -d DIR       include session directory
     -e ML_EXPR   evaluate ML expression on startup
     -f ML_FILE   evaluate ML file on startup
@@ -321,6 +322,10 @@
   premature exit of the ML process with return code 1.
 
   \<^medskip>
+  Option \<^verbatim>\<open>-T\<close> loads a specified theory file. This is a wrapper for \<^verbatim>\<open>-e\<close> with
+  a suitable @{ML use_thy} invocation.
+
+  \<^medskip>
   Option \<^verbatim>\<open>-l\<close> specifies the logic session name. Option \<^verbatim>\<open>-d\<close> specifies
   additional directories for session roots, see also \secref{sec:tool-build}.