src/Doc/System/Sessions.thy
changeset 61414 0d2d399c90a4
parent 61407 7ba7b8103565
child 61439 2bf52eec4e8a
equal deleted inserted replaced
61413:6d892287d0e9 61414:0d2d399c90a4
   268   Isabelle sessions.  It manages dependencies between sessions,
   268   Isabelle sessions.  It manages dependencies between sessions,
   269   related sources of theories and auxiliary files, and target heap
   269   related sources of theories and auxiliary files, and target heap
   270   images.  Accordingly, it runs instances of the prover process with
   270   images.  Accordingly, it runs instances of the prover process with
   271   optional document preparation.  Its command-line usage
   271   optional document preparation.  Its command-line usage
   272   is:\footnote{Isabelle/Scala provides the same functionality via
   272   is:\footnote{Isabelle/Scala provides the same functionality via
   273   \texttt{isabelle.Build.build}.}
   273   @{verbatim "isabelle.Build.build"}.}
   274   @{verbatim [display]
   274   @{verbatim [display]
   275 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   275 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   276 
   276 
   277   Options are:
   277   Options are:
   278     -D DIR       include session directory and select its sessions
   278     -D DIR       include session directory and select its sessions
   305   described in (\secref{sec:session-root}).  The totality of sessions
   305   described in (\secref{sec:session-root}).  The totality of sessions
   306   is determined by collecting such specifications from all Isabelle
   306   is determined by collecting such specifications from all Isabelle
   307   component directories (\secref{sec:components}), augmented by more
   307   component directories (\secref{sec:components}), augmented by more
   308   directories given via options @{verbatim "-d"}~@{text "DIR"} on the
   308   directories given via options @{verbatim "-d"}~@{text "DIR"} on the
   309   command line.  Each such directory may contain a session
   309   command line.  Each such directory may contain a session
   310   \texttt{ROOT} file with several session specifications.
   310   @{verbatim ROOT} file with several session specifications.
   311 
   311 
   312   Any session root directory may refer recursively to further
   312   Any session root directory may refer recursively to further
   313   directories of the same kind, by listing them in a catalog file
   313   directories of the same kind, by listing them in a catalog file
   314   @{verbatim "ROOTS"} line-by-line.  This helps to organize large
   314   @{verbatim "ROOTS"} line-by-line.  This helps to organize large
   315   collections of session specifications, or to make @{verbatim "-d"}
   315   collections of session specifications, or to make @{verbatim "-d"}
   345   \<^medskip>
   345   \<^medskip>
   346   The build process depends on additional options
   346   The build process depends on additional options
   347   (\secref{sec:system-options}) that are passed to the prover
   347   (\secref{sec:system-options}) that are passed to the prover
   348   eventually.  The settings variable @{setting_ref
   348   eventually.  The settings variable @{setting_ref
   349   ISABELLE_BUILD_OPTIONS} allows to provide additional defaults, e.g.\
   349   ISABELLE_BUILD_OPTIONS} allows to provide additional defaults, e.g.\
   350   \texttt{ISABELLE_BUILD_OPTIONS="document=pdf threads=4"}. Moreover,
   350   @{verbatim \<open>ISABELLE_BUILD_OPTIONS="document=pdf threads=4"\<close>}. Moreover,
   351   the environment of system build options may be augmented on the
   351   the environment of system build options may be augmented on the
   352   command line via @{verbatim "-o"}~@{text "name"}@{verbatim
   352   command line via @{verbatim "-o"}~@{text "name"}@{verbatim
   353   "="}@{text "value"} or @{verbatim "-o"}~@{text "name"}, which
   353   "="}@{text "value"} or @{verbatim "-o"}~@{text "name"}, which
   354   abbreviates @{verbatim "-o"}~@{text "name"}@{verbatim"=true"} for
   354   abbreviates @{verbatim "-o"}~@{text "name"}@{verbatim"=true"} for
   355   Boolean options.  Multiple occurrences of @{verbatim "-o"} on the
   355   Boolean options.  Multiple occurrences of @{verbatim "-o"} on the