src/Doc/JEdit/JEdit.thy
changeset 65541 ae09b9f5980b
parent 65511 ea42dfd95ec8
child 65572 6acb28e5ba41
equal deleted inserted replaced
65540:2b73ed8bf4d9 65541:ae09b9f5980b
   229   jedit} is as follows:
   229   jedit} is as follows:
   230   @{verbatim [display]
   230   @{verbatim [display]
   231 \<open>Usage: isabelle jedit [OPTIONS] [FILES ...]
   231 \<open>Usage: isabelle jedit [OPTIONS] [FILES ...]
   232 
   232 
   233   Options are:
   233   Options are:
   234     -A           explore theory imports of all known sessions
       
   235     -D NAME=X    set JVM system property
   234     -D NAME=X    set JVM system property
   236     -J OPTION    add JVM runtime option
   235     -J OPTION    add JVM runtime option
   237     -R           open ROOT entry of logic session and use its parent
   236     -R           open ROOT entry of logic session and use its parent
   238     -b           build only
   237     -b           build only
   239     -d DIR       include session directory
   238     -d DIR       include session directory
   255 
   254 
   256   By default, the specified image is checked and built on demand. The \<^verbatim>\<open>-s\<close>
   255   By default, the specified image is checked and built on demand. The \<^verbatim>\<open>-s\<close>
   257   option determines where to store the result session image of @{tool build}.
   256   option determines where to store the result session image of @{tool build}.
   258   The \<^verbatim>\<open>-n\<close> option bypasses the implicit build process for the selected
   257   The \<^verbatim>\<open>-n\<close> option bypasses the implicit build process for the selected
   259   session image.
   258   session image.
   260 
       
   261   Option \<^verbatim>\<open>-A\<close> explores theory imports of all known sessions (according to the
       
   262   directories specified via option \<^verbatim>\<open>-d\<close>). This facilitates editing of a
       
   263   complex session hierarchy with session-qualified theory imports, while using
       
   264   a different base session image than usual.
       
   265 
   259 
   266   Option \<^verbatim>\<open>-R\<close> modifies the meaning of option \<^verbatim>\<open>-l\<close> as follows: the \<^verbatim>\<open>ROOT\<close>
   260   Option \<^verbatim>\<open>-R\<close> modifies the meaning of option \<^verbatim>\<open>-l\<close> as follows: the \<^verbatim>\<open>ROOT\<close>
   267   entry of the specified session is opened in the editor, while its parent
   261   entry of the specified session is opened in the editor, while its parent
   268   session is used for formal checking. This facilitates maintenance of a
   262   session is used for formal checking. This facilitates maintenance of a
   269   broken session, by moving the Prover IDE quickly to relevant source files.
   263   broken session, by moving the Prover IDE quickly to relevant source files.