doc-src/System/Thy/Sessions.thy
changeset 48903 1621b3f26095
parent 48814 d488a5f25bf6
child 48916 f45ccc0d1ace
equal deleted inserted replaced
48902:44a6967240b7 48903:1621b3f26095
   187     -b           build heap images
   187     -b           build heap images
   188     -c           clean build
   188     -c           clean build
   189     -d DIR       include session directory
   189     -d DIR       include session directory
   190     -g NAME      select session group NAME
   190     -g NAME      select session group NAME
   191     -j INT       maximum number of parallel jobs (default 1)
   191     -j INT       maximum number of parallel jobs (default 1)
       
   192     -l           list session source files
   192     -n           no build -- test dependencies only
   193     -n           no build -- test dependencies only
   193     -o OPTION    override session configuration OPTION
   194     -o OPTION    override session configuration OPTION
   194                  (via NAME=VAL or NAME)
   195                  (via NAME=VAL or NAME)
   195     -s           system build mode: produce output in ISABELLE_HOME
   196     -s           system build mode: produce output in ISABELLE_HOME
   196     -v           verbose
   197     -v           verbose
   263   means that resulting heap images and log files are stored in
   264   means that resulting heap images and log files are stored in
   264   @{verbatim "$ISABELLE_HOME/heaps"} instead of the default location
   265   @{verbatim "$ISABELLE_HOME/heaps"} instead of the default location
   265   @{setting ISABELLE_OUTPUT} (which is normally in @{setting
   266   @{setting ISABELLE_OUTPUT} (which is normally in @{setting
   266   ISABELLE_HOME_USER}, i.e.\ the user's home directory).
   267   ISABELLE_HOME_USER}, i.e.\ the user's home directory).
   267 
   268 
   268   \medskip Option @{verbatim "-v"} enables verbose mode.
   269   \medskip Option @{verbatim "-v"} increases the general level of
       
   270   verbosity.  Option @{verbatim "-l"} lists the source files that
       
   271   contribute to a session.
   269 *}
   272 *}
   270 
   273 
   271 subsubsection {* Examples *}
   274 subsubsection {* Examples *}
   272 
   275 
   273 text {*
   276 text {*