src/Doc/System/Sessions.thy
changeset 66841 5c32a072ca8b
parent 66759 918f15c9367a
child 66851 c75769065548
equal deleted inserted replaced
66840:0d689d71dbdc 66841:5c32a072ca8b
   278     -X NAME      exclude sessions from group NAME and all descendants
   278     -X NAME      exclude sessions from group NAME and all descendants
   279     -a           select all sessions
   279     -a           select all sessions
   280     -b           build heap images
   280     -b           build heap images
   281     -c           clean build
   281     -c           clean build
   282     -d DIR       include session directory
   282     -d DIR       include session directory
       
   283     -f           fresh build
   283     -g NAME      select session group NAME
   284     -g NAME      select session group NAME
   284     -j INT       maximum number of parallel jobs (default 1)
   285     -j INT       maximum number of parallel jobs (default 1)
   285     -k KEYWORD   check theory sources for conflicts with proposed keywords
   286     -k KEYWORD   check theory sources for conflicts with proposed keywords
   286     -l           list session source files
   287     -l           list session source files
   287     -n           no build -- test dependencies only
   288     -n           no build -- test dependencies only
   361   of sessions, as required for other sessions to continue later on.
   362   of sessions, as required for other sessions to continue later on.
   362 
   363 
   363   \<^medskip>
   364   \<^medskip>
   364   Option \<^verbatim>\<open>-c\<close> cleans all descendants of the selected sessions before
   365   Option \<^verbatim>\<open>-c\<close> cleans all descendants of the selected sessions before
   365   performing the specified build operation.
   366   performing the specified build operation.
       
   367 
       
   368   \<^medskip>
       
   369   Option \<^verbatim>\<open>-f\<close> forces a fresh build of all selected sessions and their
       
   370   requirements.
   366 
   371 
   367   \<^medskip>
   372   \<^medskip>
   368   Option \<^verbatim>\<open>-n\<close> omits the actual build process after the preparatory stage
   373   Option \<^verbatim>\<open>-n\<close> omits the actual build process after the preparatory stage
   369   (including optional cleanup). Note that the return code always indicates the
   374   (including optional cleanup). Note that the return code always indicates the
   370   status of the set of selected sessions.
   375   status of the set of selected sessions.