src/Doc/System/Sessions.thy
changeset 64265 8eb6365f5916
parent 63827 b24d0e53dd03
child 64308 b00508facb4f
equal deleted inserted replaced
64264:42138702d6ec 64265:8eb6365f5916
   255   @{verbatim [display]
   255   @{verbatim [display]
   256 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   256 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   257 
   257 
   258   Options are:
   258   Options are:
   259     -D DIR       include session directory and select its sessions
   259     -D DIR       include session directory and select its sessions
       
   260     -N           cyclic shuffling of NUMA CPU nodes (performance tuning)
   260     -R           operate on requirements of selected sessions
   261     -R           operate on requirements of selected sessions
   261     -X NAME      exclude sessions from group NAME and all descendants
   262     -X NAME      exclude sessions from group NAME and all descendants
   262     -a           select all sessions
   263     -a           select all sessions
   263     -b           build heap images
   264     -b           build heap images
   264     -c           clean build
   265     -c           clean build
   347   Option \<^verbatim>\<open>-j\<close> specifies the maximum number of parallel build jobs (prover
   348   Option \<^verbatim>\<open>-j\<close> specifies the maximum number of parallel build jobs (prover
   348   processes). Each prover process is subject to a separate limit of parallel
   349   processes). Each prover process is subject to a separate limit of parallel
   349   worker threads, cf.\ system option @{system_option_ref threads}.
   350   worker threads, cf.\ system option @{system_option_ref threads}.
   350 
   351 
   351   \<^medskip>
   352   \<^medskip>
       
   353   Option \<^verbatim>\<open>-N\<close> enables cyclic shuffling of NUMA CPU nodes. This may help
       
   354   performance tuning on Linux servers with separate CPU/memory modules.
       
   355 
       
   356   \<^medskip>
   352   Option \<^verbatim>\<open>-s\<close> enables \<^emph>\<open>system mode\<close>, which means that resulting heap images
   357   Option \<^verbatim>\<open>-s\<close> enables \<^emph>\<open>system mode\<close>, which means that resulting heap images
   353   and log files are stored in @{path "$ISABELLE_HOME/heaps"} instead of the
   358   and log files are stored in @{path "$ISABELLE_HOME/heaps"} instead of the
   354   default location @{setting ISABELLE_OUTPUT} (which is normally in @{setting
   359   default location @{setting ISABELLE_OUTPUT} (which is normally in @{setting
   355   ISABELLE_HOME_USER}, i.e.\ the user's home directory).
   360   ISABELLE_HOME_USER}, i.e.\ the user's home directory).
   356 
   361