src/Doc/System/Sessions.thy
changeset 50406 c28753665b8e
parent 49131 aa1e2ba3c697
child 50531 f841ac0cb757
--- a/src/Doc/System/Sessions.thy	Thu Dec 06 21:16:46 2012 +0100
+++ b/src/Doc/System/Sessions.thy	Thu Dec 06 21:46:20 2012 +0100
@@ -334,4 +334,29 @@
 \end{ttbox}
 *}
 
+
+section {* Build dialog *}
+
+text {* The @{tool_def build_dialog} provides a simple GUI wrapper to
+  the tool Isabelle @{tool build} tool.  This enables user interfaces
+  like Isabelle/jEdit \secref{sec:tool-jedit} to provide read-made
+  logic image on startup.  Its command-line usage is:
+\begin{ttbox}
+Usage: isabelle build_dialog [OPTIONS] LOGIC
+
+  Options are:
+    -L OPTION    default logic via system option
+    -d DIR       include session directory
+    -s           system build mode: produce output in ISABELLE_HOME
+
+  Build Isabelle session image LOGIC via GUI dialog.
+\end{ttbox}
+
+  \medskip Option @{verbatim "-L"} specifies a system option name as
+  fall-back, if the specified @{text "LOGIC"} name is empty.
+
+  \medskip Options @{verbatim "-d"} and @{verbatim "-s"} have the same
+  meaning as for the command-line @{tool build} tool itself.
+*}
+
 end