src/Doc/System/Environment.thy
changeset 83321 7505b5e592b1
parent 83320 7376008e7318
child 83524 d76a77fe5d7a
--- a/src/Doc/System/Environment.thy	Mon Oct 20 13:29:52 2025 +0200
+++ b/src/Doc/System/Environment.thy	Mon Oct 20 14:38:15 2025 +0200
@@ -325,7 +325,6 @@
 \<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
@@ -342,10 +341,6 @@
   a 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>\<open>use_thy\<close> 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}.