diff -r 5b49c650d413 -r 72900f34dbb3 src/Doc/System/Sessions.thy --- a/src/Doc/System/Sessions.thy Mon Jun 07 09:36:21 2021 +0200 +++ b/src/Doc/System/Sessions.thy Mon Jun 07 11:42:05 2021 +0200 @@ -201,8 +201,9 @@ info, see also \secref{sec:info}. \<^item> @{system_option_def "document"} controls document output for a - particular session or theory; \<^verbatim>\document=pdf\ means enabled, - \<^verbatim>\document=false\ means disabled (especially for particular theories). + particular session or theory; \<^verbatim>\document=pdf\ or \<^verbatim>\document=true\ means + enabled, \<^verbatim>\document=""\ or \<^verbatim>\document=false\ means disabled (especially + for particular theories). \<^item> @{system_option_def "document_output"} specifies an alternative directory for generated output of the document preparation system; the @@ -278,7 +279,8 @@ \<^item> @{system_option_def system_log} specifies an optional log file for low-level messages produced by \<^ML>\Output.system_message\ in - Isabelle/ML; ``\<^verbatim>\-\'' refers to console progress of the build job. + Isabelle/ML; the value ``\<^verbatim>\true\'' refers to console progress of the build + job. \<^item> @{system_option_def "system_heaps"} determines the directories for session heap images: \<^path>\$ISABELLE_HEAPS\ is the user directory and @@ -410,11 +412,12 @@ The build process depends on additional options (\secref{sec:system-options}) that are passed to the prover eventually. The settings variable @{setting_ref ISABELLE_BUILD_OPTIONS} allows to provide - additional defaults, e.g.\ \<^verbatim>\ISABELLE_BUILD_OPTIONS="document=pdf threads=4"\. - Moreover, the environment of system build options may be augmented on the - command line via \<^verbatim>\-o\~\name\\<^verbatim>\=\\value\ or \<^verbatim>\-o\~\name\, which abbreviates - \<^verbatim>\-o\~\name\\<^verbatim>\=true\ for Boolean options. Multiple occurrences of \<^verbatim>\-o\ on - the command-line are applied in the given order. + additional defaults, e.g.\ \<^verbatim>\ISABELLE_BUILD_OPTIONS="document=pdf + threads=4"\. Moreover, the environment of system build options may be + augmented on the command line via \<^verbatim>\-o\~\name\\<^verbatim>\=\\value\ or \<^verbatim>\-o\~\name\, + which abbreviates \<^verbatim>\-o\~\name\\<^verbatim>\=true\ for Boolean or string options. + Multiple occurrences of \<^verbatim>\-o\ on the command-line are applied in the given + order. \<^medskip> Option \<^verbatim>\-P\ enables PDF/HTML presentation in the given directory, where @@ -496,7 +499,7 @@ \<^smallskip> Build all sessions with HTML browser info and PDF document preparation: - @{verbatim [display] \isabelle build -a -o browser_info -o document=pdf\} + @{verbatim [display] \isabelle build -a -o browser_info -o document\} \<^smallskip> Build all sessions with a maximum of 8 parallel prover processes and 4