src/Doc/System/Sessions.thy
changeset 50406 c28753665b8e
parent 49131 aa1e2ba3c697
child 50531 f841ac0cb757
equal deleted inserted replaced
50405:366c4a602500 50406:c28753665b8e
   332 \begin{ttbox}
   332 \begin{ttbox}
   333 isabelle build -D '$AFP' -R -v -n
   333 isabelle build -D '$AFP' -R -v -n
   334 \end{ttbox}
   334 \end{ttbox}
   335 *}
   335 *}
   336 
   336 
       
   337 
       
   338 section {* Build dialog *}
       
   339 
       
   340 text {* The @{tool_def build_dialog} provides a simple GUI wrapper to
       
   341   the tool Isabelle @{tool build} tool.  This enables user interfaces
       
   342   like Isabelle/jEdit \secref{sec:tool-jedit} to provide read-made
       
   343   logic image on startup.  Its command-line usage is:
       
   344 \begin{ttbox}
       
   345 Usage: isabelle build_dialog [OPTIONS] LOGIC
       
   346 
       
   347   Options are:
       
   348     -L OPTION    default logic via system option
       
   349     -d DIR       include session directory
       
   350     -s           system build mode: produce output in ISABELLE_HOME
       
   351 
       
   352   Build Isabelle session image LOGIC via GUI dialog.
       
   353 \end{ttbox}
       
   354 
       
   355   \medskip Option @{verbatim "-L"} specifies a system option name as
       
   356   fall-back, if the specified @{text "LOGIC"} name is empty.
       
   357 
       
   358   \medskip Options @{verbatim "-d"} and @{verbatim "-s"} have the same
       
   359   meaning as for the command-line @{tool build} tool itself.
       
   360 *}
       
   361 
   337 end
   362 end