src/Doc/JEdit/JEdit.thy
changeset 73150 c9a836122739
parent 73128 b15fe413b4d2
child 73151 f78a3be79ad1
equal deleted inserted replaced
73149:bdc8cd6f5e6e 73150:c9a836122739
   303   The \<^verbatim>\<open>-c\<close> option merely checks the presence of the server, producing a
   303   The \<^verbatim>\<open>-c\<close> option merely checks the presence of the server, producing a
   304   process return-code.
   304   process return-code.
   305 
   305 
   306   The \<^verbatim>\<open>-n\<close> option reports the server name, and the \<^verbatim>\<open>-s\<close> option provides a
   306   The \<^verbatim>\<open>-n\<close> option reports the server name, and the \<^verbatim>\<open>-s\<close> option provides a
   307   different server name. The default server name is the official distribution
   307   different server name. The default server name is the official distribution
   308   name (e.g.\ \<^verbatim>\<open>Isabelle2020\<close>). Thus @{tool jedit_client} can connect to the
   308   name (e.g.\ \<^verbatim>\<open>Isabelle2021\<close>). Thus @{tool jedit_client} can connect to the
   309   Isabelle desktop application without further options.
   309   Isabelle desktop application without further options.
   310 
   310 
   311   The \<^verbatim>\<open>-p\<close> option allows to override the implicit default of the system
   311   The \<^verbatim>\<open>-p\<close> option allows to override the implicit default of the system
   312   option @{system_option_ref ML_process_policy} for ML processes started by
   312   option @{system_option_ref ML_process_policy} for ML processes started by
   313   the Prover IDE, e.g. to control CPU affinity on multiprocessor systems.
   313   the Prover IDE, e.g. to control CPU affinity on multiprocessor systems.