src/Doc/JEdit/JEdit.thy
changeset 68370 bcdc47c9d4af
parent 68224 1f7308050349
child 68394 bc2fd0e2047e
equal deleted inserted replaced
68369:6989752bba4b 68370:bcdc47c9d4af
   226   jedit} is as follows:
   226   jedit} is as follows:
   227   @{verbatim [display]
   227   @{verbatim [display]
   228 \<open>Usage: isabelle jedit [OPTIONS] [FILES ...]
   228 \<open>Usage: isabelle jedit [OPTIONS] [FILES ...]
   229 
   229 
   230   Options are:
   230   Options are:
   231     -A           specify ancestor for base session image (default: parent)
   231     -A NAME      ancestor session for options -R and -S (default: parent)
   232     -B           use base session image, with theories from other sessions
       
   233     -F           focus on selected logic session: ignore unrelated theories
       
   234     -D NAME=X    set JVM system property
   232     -D NAME=X    set JVM system property
   235     -J OPTION    add JVM runtime option
   233     -J OPTION    add JVM runtime option
   236                  (default $JEDIT_JAVA_SYSTEM_OPTIONS $JEDIT_JAVA_OPTIONS)
   234                  (default $JEDIT_JAVA_SYSTEM_OPTIONS $JEDIT_JAVA_OPTIONS)
   237     -P           use parent session image
   235     -R NAME      build image with requirements from other sessions
   238     -R           open ROOT entry of logic session
   236     -S NAME      like option -R, with focus on selected session
   239     -S NAME      edit specified logic session, abbreviates -B -F -R -l NAME
       
   240     -b           build only
   237     -b           build only
   241     -d DIR       include session directory
   238     -d DIR       include session directory
   242     -f           fresh build
   239     -f           fresh build
   243     -j OPTION    add jEdit runtime option
   240     -j OPTION    add jEdit runtime option
   244                  (default $JEDIT_OPTIONS)
   241                  (default $JEDIT_OPTIONS)
   259   By default, the specified image is checked and built on demand. The \<^verbatim>\<open>-s\<close>
   256   By default, the specified image is checked and built on demand. The \<^verbatim>\<open>-s\<close>
   260   option determines where to store the result session image of @{tool build}.
   257   option determines where to store the result session image of @{tool build}.
   261   The \<^verbatim>\<open>-n\<close> option bypasses the implicit build process for the selected
   258   The \<^verbatim>\<open>-n\<close> option bypasses the implicit build process for the selected
   262   session image.
   259   session image.
   263 
   260 
   264   Option \<^verbatim>\<open>-P\<close> and \<^verbatim>\<open>-B\<close> and are mutually exclusive and modify the meaning of
   261   Option \<^verbatim>\<open>-R\<close> builds an auxiliary logic image with all required theories from
   265   option \<^verbatim>\<open>-l\<close> as follows. Option \<^verbatim>\<open>-P\<close> opens the parent session image. Option
   262   \<^emph>\<open>other\<close> sessions, relative to an ancestor session given by option \<^verbatim>\<open>-A\<close>
   266   \<^verbatim>\<open>-B\<close> prepares a logic image on the spot, based on the required theory
   263   (default: parent session). Option \<^verbatim>\<open>-R\<close> also opens the session \<^verbatim>\<open>ROOT\<close> entry
   267   imports from other sessions, relative to an ancestor session given by option
   264   in the editor, to facilitate editing of the main session.
   268   \<^verbatim>\<open>-A\<close> (default: parent session).
   265 
   269 
   266   Option \<^verbatim>\<open>-S\<close> is like \<^verbatim>\<open>-R\<close>, with a focus on the selected session and its
   270   Option \<^verbatim>\<open>-F\<close> focuses on the effective logic session: the accessible
   267   descendants: the namespace of accessible theories is restricted accordingly.
   271   namespace of theories is restricted to sessions that are connected to it.
   268   This reduces startup time for big projects, notably the ``Archive of Formal
   272 
   269   Proofs''.
   273   Option \<^verbatim>\<open>-R\<close> opens the ROOT entry of the specified logic session in the
       
   274   editor. Option \<^verbatim>\<open>-S\<close> sets up the development environment to edit the
       
   275   specified session: it abbreviates \<^verbatim>\<open>-B\<close> \<^verbatim>\<open>-F\<close> \<^verbatim>\<open>-R\<close> \<^verbatim>\<open>-l\<close>.
       
   276 
   270 
   277   The \<^verbatim>\<open>-m\<close> option specifies additional print modes for the prover process.
   271   The \<^verbatim>\<open>-m\<close> option specifies additional print modes for the prover process.
   278   Note that the system option @{system_option_ref jedit_print_mode} allows to
   272   Note that the system option @{system_option_ref jedit_print_mode} allows to
   279   do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> dialog of
   273   do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> dialog of
   280   Isabelle/jEdit), without requiring command-line invocation.
   274   Isabelle/jEdit), without requiring command-line invocation.