src/Doc/System/Sessions.thy
changeset 73774 734d5d3fbd9d
parent 73743 813a08dff3fd
child 73777 52e43a93d51f
equal deleted inserted replaced
73773:ac7f41b66e1b 73774:734d5d3fbd9d
   324 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   324 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   325 
   325 
   326   Options are:
   326   Options are:
   327     -B NAME      include session NAME and all descendants
   327     -B NAME      include session NAME and all descendants
   328     -D DIR       include session directory and select its sessions
   328     -D DIR       include session directory and select its sessions
       
   329     -L FILE      append syslog messages to given FILE
   329     -N           cyclic shuffling of NUMA CPU nodes (performance tuning)
   330     -N           cyclic shuffling of NUMA CPU nodes (performance tuning)
   330     -P DIR       enable HTML/PDF presentation in directory (":" for default)
   331     -P DIR       enable HTML/PDF presentation in directory (":" for default)
   331     -R           refer to requirements of selected sessions
   332     -R           refer to requirements of selected sessions
   332     -S           soft build: only observe changes of sources, not heap images
   333     -S           soft build: only observe changes of sources, not heap images
   333     -X NAME      exclude sessions from group NAME and all descendants
   334     -X NAME      exclude sessions from group NAME and all descendants
   458   \<^medskip>
   459   \<^medskip>
   459   Option \<^verbatim>\<open>-v\<close> increases the general level of verbosity. Option \<^verbatim>\<open>-l\<close> lists
   460   Option \<^verbatim>\<open>-v\<close> increases the general level of verbosity. Option \<^verbatim>\<open>-l\<close> lists
   460   the source files that contribute to a session.
   461   the source files that contribute to a session.
   461 
   462 
   462   \<^medskip>
   463   \<^medskip>
       
   464   Option \<^verbatim>\<open>-L\<close>~\<open>FILE\<close> appends syslog messages to the given file. Such messages
       
   465   can be produced in Isabelle/ML via formal \<^ML>\<open>Output.system_message\<close> or
       
   466   informal \<^ML>\<open>Output.physical_stderr\<close>.
       
   467 
       
   468   \<^medskip>
   463   Option \<^verbatim>\<open>-k\<close> specifies a newly proposed keyword for outer syntax (multiple
   469   Option \<^verbatim>\<open>-k\<close> specifies a newly proposed keyword for outer syntax (multiple
   464   uses allowed). The theory sources are checked for conflicts wrt.\ this
   470   uses allowed). The theory sources are checked for conflicts wrt.\ this
   465   hypothetical change of syntax, e.g.\ to reveal occurrences of identifiers
   471   hypothetical change of syntax, e.g.\ to reveal occurrences of identifiers
   466   that need to be quoted.
   472   that need to be quoted.
   467 \<close>
   473 \<close>