diff -r df14a62129e9 -r cf69c9112d09 src/Doc/System/Sessions.thy --- a/src/Doc/System/Sessions.thy Mon Jun 13 11:31:59 2022 +0200 +++ b/src/Doc/System/Sessions.thy Mon Jun 13 11:35:00 2022 +0200 @@ -488,53 +488,53 @@ text \ Build a specific logic image: - @{verbatim [display] \isabelle build -b HOLCF\} + @{verbatim [display] \ isabelle build -b HOLCF\} \<^smallskip> Build the main group of logic images: - @{verbatim [display] \isabelle build -b -g main\} + @{verbatim [display] \ isabelle build -b -g main\} \<^smallskip> Build all descendants (and requirements) of \<^verbatim>\FOL\ and \<^verbatim>\ZF\: - @{verbatim [display] \isabelle build -B FOL -B ZF\} + @{verbatim [display] \ isabelle build -B FOL -B ZF\} \<^smallskip> Build all sessions where sources have changed (ignoring heaps): - @{verbatim [display] \isabelle build -a -S\} + @{verbatim [display] \ isabelle build -a -S\} \<^smallskip> Provide a general overview of the status of all Isabelle sessions, without building anything: - @{verbatim [display] \isabelle build -a -n -v\} + @{verbatim [display] \ isabelle build -a -n -v\} \<^smallskip> Build all sessions with HTML browser info and PDF document preparation: - @{verbatim [display] \isabelle build -a -o browser_info -o document\} + @{verbatim [display] \ isabelle build -a -o browser_info -o document\} \<^smallskip> Build all sessions with a maximum of 8 parallel prover processes and 4 worker threads each (on a machine with many cores): - @{verbatim [display] \isabelle build -a -j8 -o threads=4\} + @{verbatim [display] \ isabelle build -a -j8 -o threads=4\} \<^smallskip> Build some session images with cleanup of their descendants, while retaining their ancestry: - @{verbatim [display] \isabelle build -b -c HOL-Library HOL-Algebra\} + @{verbatim [display] \ isabelle build -b -c HOL-Library HOL-Algebra\} \<^smallskip> Clean all sessions without building anything: - @{verbatim [display] \isabelle build -a -n -c\} + @{verbatim [display] \ isabelle build -a -n -c\} \<^smallskip> Build all sessions from some other directory hierarchy, according to the settings variable \<^verbatim>\AFP\ that happens to be defined inside the Isabelle environment: - @{verbatim [display] \isabelle build -D '$AFP'\} + @{verbatim [display] \ isabelle build -D '$AFP'\} \<^smallskip> Inform about the status of all sessions required for AFP, without building anything yet: - @{verbatim [display] \isabelle build -D '$AFP' -R -v -n\} + @{verbatim [display] \ isabelle build -D '$AFP' -R -v -n\} \ @@ -586,7 +586,7 @@ text \ Print messages from theory \<^verbatim>\HOL.Nat\ of session \<^verbatim>\HOL\, using Unicode rendering of Isabelle symbols and a margin of 100 characters: - @{verbatim [display] \isabelle log -T HOL.Nat -U -m 100 HOL\} + @{verbatim [display] \ isabelle log -T HOL.Nat -U -m 100 HOL\} \ @@ -695,17 +695,17 @@ text \ Dump all Isabelle/ZF sessions (which are rather small): - @{verbatim [display] \isabelle dump -v -B ZF\} + @{verbatim [display] \ isabelle dump -v -B ZF\} \<^smallskip> Dump the quite substantial \<^verbatim>\HOL-Analysis\ session, with full bootstrap from Isabelle/Pure: - @{verbatim [display] \isabelle dump -v HOL-Analysis\} + @{verbatim [display] \ isabelle dump -v HOL-Analysis\} \<^smallskip> Dump all sessions connected to HOL-Analysis, using main Isabelle/HOL as basis: - @{verbatim [display] \isabelle dump -v -b HOL -B HOL-Analysis\} + @{verbatim [display] \ isabelle dump -v -b HOL -B HOL-Analysis\} This results in uniform PIDE markup for everything, except for the Isabelle/Pure bootstrap process itself. Producing that on the spot requires @@ -713,8 +713,8 @@ process (in 64bit mode). Here are some relevant settings (\secref{sec:boot}) for such ambitious applications: @{verbatim [display] -\ISABELLE_TOOL_JAVA_OPTIONS="-Xms4g -Xmx32g -Xss16m" -ML_OPTIONS="--minheap 4G --maxheap 32G" +\ ISABELLE_TOOL_JAVA_OPTIONS="-Xms4g -Xmx32g -Xss16m" + ML_OPTIONS="--minheap 4G --maxheap 32G" \} \ @@ -797,17 +797,17 @@ Update some cartouche notation in all theory sources required for session \<^verbatim>\HOL-Analysis\ (and ancestors): - @{verbatim [display] \isabelle update -u mixfix_cartouches HOL-Analysis\} + @{verbatim [display] \ isabelle update -u mixfix_cartouches HOL-Analysis\} \<^smallskip> Update the same for all application sessions based on \<^verbatim>\HOL-Analysis\ --- using its image as starting point (for reduced resource requirements): - @{verbatim [display] \isabelle update -u mixfix_cartouches -b HOL-Analysis -B HOL-Analysis\} + @{verbatim [display] \ isabelle update -u mixfix_cartouches -b HOL-Analysis -B HOL-Analysis\} \<^smallskip> Update sessions that build on \<^verbatim>\HOL-Proofs\, which need to be run separately with special options as follows: - @{verbatim [display] \isabelle update -u mixfix_cartouches -l HOL-Proofs -B HOL-Proofs + @{verbatim [display] \ isabelle update -u mixfix_cartouches -l HOL-Proofs -B HOL-Proofs -o record_proofs=2\} \<^smallskip> See also the end of \secref{sec:tool-dump} for hints on increasing @@ -846,19 +846,19 @@ text \ All sessions of the Isabelle distribution: - @{verbatim [display] \isabelle sessions -a\} + @{verbatim [display] \ isabelle sessions -a\} \<^medskip> Sessions that are based on \<^verbatim>\ZF\ (and required by it): - @{verbatim [display] \isabelle sessions -B ZF\} + @{verbatim [display] \ isabelle sessions -B ZF\} \<^medskip> All sessions of Isabelle/AFP (based in directory \<^path>\AFP\): - @{verbatim [display] \isabelle sessions -D AFP/thys\} + @{verbatim [display] \ isabelle sessions -D AFP/thys\} \<^medskip> Sessions required by Isabelle/AFP (based in directory \<^path>\AFP\): - @{verbatim [display] \isabelle sessions -R -D AFP/thys\} + @{verbatim [display] \ isabelle sessions -R -D AFP/thys\} \ @@ -955,7 +955,7 @@ \<^verbatim>\-J\, but option \<^verbatim>\-T\ to disable the default ``quick check'' of \<^verbatim>\rsync\ (which only inspects file sizes and date stamps); existing heaps are deleted: - @{verbatim [display] \ isabelle sync -A: -T -H testmachine:test/isabelle_afp\} + @{verbatim [display] \ isabelle sync -A: -T -H testmachine:test/isabelle_afp\} \ end