src/Doc/JEdit/JEdit.thy
changeset 63987 ac96fe9224f6
parent 63871 f745c6e683b7
child 64512 2b90410090ee
equal deleted inserted replaced
63986:c7a4b03727ae 63987:ac96fe9224f6
   236     -f           fresh build
   236     -f           fresh build
   237     -j OPTION    add jEdit runtime option
   237     -j OPTION    add jEdit runtime option
   238     -l NAME      logic image name
   238     -l NAME      logic image name
   239     -m MODE      add print mode for output
   239     -m MODE      add print mode for output
   240     -n           no build of session image on startup
   240     -n           no build of session image on startup
       
   241     -p CMD       ML process command prefix (process policy)
   241     -s           system build mode for session image
   242     -s           system build mode for session image
   242 
   243 
   243   Start jEdit with Isabelle plugin setup and open FILES
   244   Start jEdit with Isabelle plugin setup and open FILES
   244   (default "$USER_HOME/Scratch.thy" or ":" for empty buffer).\<close>}
   245   (default "$USER_HOME/Scratch.thy" or ":" for empty buffer).\<close>}
   245 
   246 
   291 
   292 
   292   The \<^verbatim>\<open>-n\<close> option reports the server name, and the \<^verbatim>\<open>-s\<close> option provides a
   293   The \<^verbatim>\<open>-n\<close> option reports the server name, and the \<^verbatim>\<open>-s\<close> option provides a
   293   different server name. The default server name is the official distribution
   294   different server name. The default server name is the official distribution
   294   name (e.g.\ \<^verbatim>\<open>Isabelle2016\<close>). Thus @{tool jedit_client} can connect to the
   295   name (e.g.\ \<^verbatim>\<open>Isabelle2016\<close>). Thus @{tool jedit_client} can connect to the
   295   Isabelle desktop application without further options.
   296   Isabelle desktop application without further options.
       
   297 
       
   298   The \<^verbatim>\<open>-p\<close> option allows to override the implicit default of the system
       
   299   option @{system_option_ref ML_process_policy} for ML processes started by
       
   300   the Prover IDE, e.g. to control CPU affinity on multiprocessor systems.
   296 
   301 
   297   The JVM system property \<^verbatim>\<open>isabelle.jedit_server\<close> provides a different server
   302   The JVM system property \<^verbatim>\<open>isabelle.jedit_server\<close> provides a different server
   298   name, e.g.\ use \<^verbatim>\<open>isabelle jedit -Disabelle.jedit_server=\<close>\<open>name\<close> and
   303   name, e.g.\ use \<^verbatim>\<open>isabelle jedit -Disabelle.jedit_server=\<close>\<open>name\<close> and
   299   \<^verbatim>\<open>isabelle jedit_client -s\<close>~\<open>name\<close> to connect later on.
   304   \<^verbatim>\<open>isabelle jedit_client -s\<close>~\<open>name\<close> to connect later on.
   300 \<close>
   305 \<close>