src/Doc/JEdit/JEdit.thy
changeset 62917 eed66ba99bd9
parent 62914 930a30c1a9af
child 62969 9f394a16c557
equal deleted inserted replaced
62916:621afc4607ec 62917:eed66ba99bd9
   239     -f           fresh build
   239     -f           fresh build
   240     -j OPTION    add jEdit runtime option
   240     -j OPTION    add jEdit runtime option
   241     -l NAME      logic image name
   241     -l NAME      logic image name
   242     -m MODE      add print mode for output
   242     -m MODE      add print mode for output
   243     -n           no build of session image on startup
   243     -n           no build of session image on startup
   244     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
       
   245     -s           system build mode for session image
   244     -s           system build mode for session image
   246 
   245 
   247   Start jEdit with Isabelle plugin setup and open FILES
   246   Start jEdit with Isabelle plugin setup and open FILES
   248   (default "$USER_HOME/Scratch.thy" or ":" for empty buffer).\<close>}
   247   (default "$USER_HOME/Scratch.thy" or ":" for empty buffer).\<close>}
   249 
   248 
   259 
   258 
   260   The \<^verbatim>\<open>-m\<close> option specifies additional print modes for the prover process.
   259   The \<^verbatim>\<open>-m\<close> option specifies additional print modes for the prover process.
   261   Note that the system option @{system_option_ref jedit_print_mode} allows to
   260   Note that the system option @{system_option_ref jedit_print_mode} allows to
   262   do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> dialog of
   261   do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> dialog of
   263   Isabelle/jEdit), without requiring command-line invocation.
   262   Isabelle/jEdit), without requiring command-line invocation.
   264 
       
   265   The \<^verbatim>\<open>-o\<close> option specifies Isabelle system options that override the
       
   266   persistent preferences (see also \secref{sec:options}). Options may be
       
   267   changed on the command line via \<^verbatim>\<open>-o\<close>~\<open>name\<close>\<^verbatim>\<open>=\<close>\<open>value\<close> or \<^verbatim>\<open>-o\<close>~\<open>name\<close>,
       
   268   which abbreviates \<^verbatim>\<open>-o\<close>~\<open>name\<close>\<^verbatim>\<open>=true\<close> for Boolean options. Multiple
       
   269   occurrences of \<^verbatim>\<open>-o\<close> on the command-line are applied in the given order.
       
   270 
   263 
   271   The \<^verbatim>\<open>-J\<close> and \<^verbatim>\<open>-j\<close> options allow to pass additional low-level options to
   264   The \<^verbatim>\<open>-J\<close> and \<^verbatim>\<open>-j\<close> options allow to pass additional low-level options to
   272   the JVM or jEdit, respectively. The defaults are provided by the Isabelle
   265   the JVM or jEdit, respectively. The defaults are provided by the Isabelle
   273   settings environment @{cite "isabelle-system"}, but note that these only
   266   settings environment @{cite "isabelle-system"}, but note that these only
   274   work for the command-line tool described here, and not the regular
   267   work for the command-line tool described here, and not the regular