src/Doc/JEdit/JEdit.thy
changeset 68541 12b4b3bc585d
parent 68472 581a1bfec8ad
child 68736 29dbf3408021
equal deleted inserted replaced
68540:000a0e062529 68541:12b4b3bc585d
   235     -R NAME      build image with requirements from other sessions
   235     -R NAME      build image with requirements from other sessions
   236     -S NAME      like option -R, with focus on selected session
   236     -S NAME      like option -R, with focus on selected session
   237     -b           build only
   237     -b           build only
   238     -d DIR       include session directory
   238     -d DIR       include session directory
   239     -f           fresh build
   239     -f           fresh build
       
   240     -i NAME      include session in name-space of theories
   240     -j OPTION    add jEdit runtime option
   241     -j OPTION    add jEdit runtime option
   241                  (default $JEDIT_OPTIONS)
   242                  (default $JEDIT_OPTIONS)
   242     -l NAME      logic image name
   243     -l NAME      logic image name
   243     -m MODE      add print mode for output
   244     -m MODE      add print mode for output
   244     -n           no build of session image on startup
   245     -n           no build of session image on startup
   263   session and its descendants: the namespace of accessible theories is
   264   session and its descendants: the namespace of accessible theories is
   264   restricted accordingly. This reduces startup time for big projects, notably
   265   restricted accordingly. This reduces startup time for big projects, notably
   265   the ``Archive of Formal Proofs''. The \<^verbatim>\<open>-A\<close> option specifies and alternative
   266   the ``Archive of Formal Proofs''. The \<^verbatim>\<open>-A\<close> option specifies and alternative
   266   ancestor session for options \<^verbatim>\<open>-R\<close> and \<^verbatim>\<open>-S\<close>: this allows to restructure the
   267   ancestor session for options \<^verbatim>\<open>-R\<close> and \<^verbatim>\<open>-S\<close>: this allows to restructure the
   267   hierarchy of session images on the spot.
   268   hierarchy of session images on the spot.
       
   269 
       
   270   The \<^verbatim>\<open>-i\<close> option includes additional sessions into the name-space of
       
   271   theories: multiple occurrences are possible.
   268 
   272 
   269   The \<^verbatim>\<open>-m\<close> option specifies additional print modes for the prover process.
   273   The \<^verbatim>\<open>-m\<close> option specifies additional print modes for the prover process.
   270   Note that the system option @{system_option_ref jedit_print_mode} allows to
   274   Note that the system option @{system_option_ref jedit_print_mode} allows to
   271   do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> dialog of
   275   do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> dialog of
   272   Isabelle/jEdit), without requiring command-line invocation.
   276   Isabelle/jEdit), without requiring command-line invocation.