src/Doc/System/Sessions.thy
changeset 61572 ddb3ac3fef45
parent 61568 26c76e143b77
child 61575 f18f6e51e901
equal deleted inserted replaced
61571:9c50eb3bff50 61572:ddb3ac3fef45
   257 text \<open>The @{tool_def build} tool invokes the build process for
   257 text \<open>The @{tool_def build} tool invokes the build process for
   258   Isabelle sessions.  It manages dependencies between sessions,
   258   Isabelle sessions.  It manages dependencies between sessions,
   259   related sources of theories and auxiliary files, and target heap
   259   related sources of theories and auxiliary files, and target heap
   260   images.  Accordingly, it runs instances of the prover process with
   260   images.  Accordingly, it runs instances of the prover process with
   261   optional document preparation.  Its command-line usage
   261   optional document preparation.  Its command-line usage
   262   is:\footnote{Isabelle/Scala provides the same functionality via
   262   is:\<^footnote>\<open>Isabelle/Scala provides the same functionality via
   263   \<^verbatim>\<open>isabelle.Build.build\<close>.}
   263   \<^verbatim>\<open>isabelle.Build.build\<close>.\<close>
   264   @{verbatim [display]
   264   @{verbatim [display]
   265 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   265 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   266 
   266 
   267   Options are:
   267   Options are:
   268     -D DIR       include session directory and select its sessions
   268     -D DIR       include session directory and select its sessions