src/Doc/JEdit/JEdit.thy
changeset 69854 cc0b3e177b49
parent 69597 ff784d5a5bfb
child 70062 e7a01bbe789b
equal deleted inserted replaced
69853:f7c9a1be333f 69854:cc0b3e177b49
   241                  (default $JEDIT_OPTIONS)
   241                  (default $JEDIT_OPTIONS)
   242     -l NAME      logic image name
   242     -l NAME      logic image name
   243     -m MODE      add print mode for output
   243     -m MODE      add print mode for output
   244     -n           no build of session image on startup
   244     -n           no build of session image on startup
   245     -p CMD       ML process command prefix (process policy)
   245     -p CMD       ML process command prefix (process policy)
   246     -s           system build mode for session image
   246     -s           system build mode for session image (system_heaps=true)
       
   247     -u           user build mode for session image (system_heaps=false)
   247 
   248 
   248   Start jEdit with Isabelle plugin setup and open FILES
   249   Start jEdit with Isabelle plugin setup and open FILES
   249   (default "$USER_HOME/Scratch.thy" or ":" for empty buffer).\<close>}
   250   (default "$USER_HOME/Scratch.thy" or ":" for empty buffer).\<close>}
   250 
   251 
   251   The \<^verbatim>\<open>-l\<close> option specifies the session name of the logic image to be used
   252   The \<^verbatim>\<open>-l\<close> option specifies the session name of the logic image to be used
   252   for proof processing. Additional session root directories may be included
   253   for proof processing. Additional session root directories may be included
   253   via option \<^verbatim>\<open>-d\<close> to augment the session name space (see also @{cite
   254   via option \<^verbatim>\<open>-d\<close> to augment the session name space (see also @{cite
   254   "isabelle-system"}). By default, the specified image is checked and built on
   255   "isabelle-system"}). By default, the specified image is checked and built on
   255   demand. The \<^verbatim>\<open>-s\<close> option determines where to store the result session image
   256   demand, but option \<^verbatim>\<open>-n\<close> bypasses the implicit build process for the
   256   of @{tool build}. The \<^verbatim>\<open>-n\<close> option bypasses the implicit build process for
   257   selected session image. Options \<^verbatim>\<open>-s\<close> and \<^verbatim>\<open>-u\<close> override the default system
   257   the selected session image.
   258   option @{system_option system_heaps}: this determines where to store the
       
   259   session image of @{tool build}.
   258 
   260 
   259   The \<^verbatim>\<open>-R\<close> option builds an auxiliary logic image with all theories from
   261   The \<^verbatim>\<open>-R\<close> option builds an auxiliary logic image with all theories from
   260   other sessions that are not already present in its parent; it also opens the
   262   other sessions that are not already present in its parent; it also opens the
   261   session \<^verbatim>\<open>ROOT\<close> entry in the editor to facilitate editing of the main
   263   session \<^verbatim>\<open>ROOT\<close> entry in the editor to facilitate editing of the main
   262   session. The \<^verbatim>\<open>-S\<close> option is like \<^verbatim>\<open>-R\<close>, with a focus on the selected
   264   session. The \<^verbatim>\<open>-S\<close> option is like \<^verbatim>\<open>-R\<close>, with a focus on the selected