src/Doc/JEdit/JEdit.thy
changeset 63987 ac96fe9224f6
parent 63871 f745c6e683b7
child 64512 2b90410090ee
--- a/src/Doc/JEdit/JEdit.thy	Sat Oct 01 23:05:25 2016 +0200
+++ b/src/Doc/JEdit/JEdit.thy	Sun Oct 02 12:29:18 2016 +0200
@@ -238,6 +238,7 @@
     -l NAME      logic image name
     -m MODE      add print mode for output
     -n           no build of session image on startup
+    -p CMD       ML process command prefix (process policy)
     -s           system build mode for session image
 
   Start jEdit with Isabelle plugin setup and open FILES
@@ -294,6 +295,10 @@
   name (e.g.\ \<^verbatim>\<open>Isabelle2016\<close>). Thus @{tool jedit_client} can connect to the
   Isabelle desktop application without further options.
 
+  The \<^verbatim>\<open>-p\<close> option allows to override the implicit default of the system
+  option @{system_option_ref ML_process_policy} for ML processes started by
+  the Prover IDE, e.g. to control CPU affinity on multiprocessor systems.
+
   The JVM system property \<^verbatim>\<open>isabelle.jedit_server\<close> provides a different server
   name, e.g.\ use \<^verbatim>\<open>isabelle jedit -Disabelle.jedit_server=\<close>\<open>name\<close> and
   \<^verbatim>\<open>isabelle jedit_client -s\<close>~\<open>name\<close> to connect later on.