src/Doc/System/Sessions.thy
changeset 66737 2edc0c42c883
parent 66671 41b64e53b6a1
child 66745 e7ac579b883c
equal deleted inserted replaced
66736:148891036469 66737:2edc0c42c883
   278   \<^verbatim>\<open>isabelle.Build.build\<close>.\<close>
   278   \<^verbatim>\<open>isabelle.Build.build\<close>.\<close>
   279   @{verbatim [display]
   279   @{verbatim [display]
   280 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   280 \<open>Usage: isabelle build [OPTIONS] [SESSIONS ...]
   281 
   281 
   282   Options are:
   282   Options are:
       
   283     -B NAME      include session NAME and all descendants
   283     -D DIR       include session directory and select its sessions
   284     -D DIR       include session directory and select its sessions
   284     -N           cyclic shuffling of NUMA CPU nodes (performance tuning)
   285     -N           cyclic shuffling of NUMA CPU nodes (performance tuning)
   285     -R           operate on requirements of selected sessions
   286     -R           operate on requirements of selected sessions
   286     -X NAME      exclude sessions from group NAME and all descendants
   287     -X NAME      exclude sessions from group NAME and all descendants
   287     -a           select all sessions
   288     -a           select all sessions
   327   more options \<^verbatim>\<open>-g\<close>~\<open>NAME\<close>. Option \<^verbatim>\<open>-a\<close> selects all sessions. The build tool
   328   more options \<^verbatim>\<open>-g\<close>~\<open>NAME\<close>. Option \<^verbatim>\<open>-a\<close> selects all sessions. The build tool
   328   takes session dependencies into account: the set of selected sessions is
   329   takes session dependencies into account: the set of selected sessions is
   329   completed by including all ancestors.
   330   completed by including all ancestors.
   330 
   331 
   331   \<^medskip>
   332   \<^medskip>
       
   333   One or more options \<^verbatim>\<open>-B\<close>~\<open>NAME\<close> specify base sessions. All descendants
       
   334   are included.
       
   335 
       
   336   \<^medskip>
   332   One or more options \<^verbatim>\<open>-x\<close>~\<open>NAME\<close> specify sessions to be excluded. All
   337   One or more options \<^verbatim>\<open>-x\<close>~\<open>NAME\<close> specify sessions to be excluded. All
   333   descendents of excluded sessions are removed from the selection as specified
   338   descendents of excluded sessions are removed from the selection as specified
   334   above. Option \<^verbatim>\<open>-X\<close> is analogous to this, but excluded sessions are
   339   above. Option \<^verbatim>\<open>-X\<close> is analogous to this, but excluded sessions are
   335   specified by session group membership.
   340   specified by session group membership.
   336 
   341 
   448   session structure. It supports three main operations via options \<^verbatim>\<open>-I\<close>,
   453   session structure. It supports three main operations via options \<^verbatim>\<open>-I\<close>,
   449   \<^verbatim>\<open>-M\<close>, \<^verbatim>\<open>-U\<close>. Its command-line usage is: @{verbatim [display]
   454   \<^verbatim>\<open>-M\<close>, \<^verbatim>\<open>-U\<close>. Its command-line usage is: @{verbatim [display]
   450 \<open>Usage: isabelle imports [OPTIONS] [SESSIONS ...]
   455 \<open>Usage: isabelle imports [OPTIONS] [SESSIONS ...]
   451 
   456 
   452   Options are:
   457   Options are:
       
   458     -B NAME      include session NAME and all descendants
   453     -D DIR       include session directory and select its sessions
   459     -D DIR       include session directory and select its sessions
   454     -I           operation: report potential session imports
   460     -I           operation: report potential session imports
   455     -M           operation: Mercurial repository check for theory files
   461     -M           operation: Mercurial repository check for theory files
   456     -R           operate on requirements of selected sessions
   462     -R           operate on requirements of selected sessions
   457     -U           operation: update theory imports to use session qualifiers
   463     -U           operation: update theory imports to use session qualifiers
   467   Maintain theory imports wrt. session structure. At least one operation
   473   Maintain theory imports wrt. session structure. At least one operation
   468   needs to be specified (see options -I -M -U).\<close>}
   474   needs to be specified (see options -I -M -U).\<close>}
   469 
   475 
   470   \<^medskip>
   476   \<^medskip>
   471   The selection of sessions and session directories works as for @{tool build}
   477   The selection of sessions and session directories works as for @{tool build}
   472   via options \<^verbatim>\<open>-D\<close>, \<^verbatim>\<open>-R\<close>, \<^verbatim>\<open>-X\<close>, \<^verbatim>\<open>-a\<close>, \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-g\<close>, \<^verbatim>\<open>-x\<close> (see
   478   via options \<^verbatim>\<open>-B\<close>, \<^verbatim>\<open>-D\<close>, \<^verbatim>\<open>-R\<close>, \<^verbatim>\<open>-X\<close>, \<^verbatim>\<open>-a\<close>, \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-g\<close>, \<^verbatim>\<open>-x\<close> (see
   473   \secref{sec:tool-build}).
   479   \secref{sec:tool-build}).
   474 
   480 
   475   \<^medskip>
   481   \<^medskip>
   476   Option \<^verbatim>\<open>-o\<close> overrides Isabelle system options as for @{tool build}
   482   Option \<^verbatim>\<open>-o\<close> overrides Isabelle system options as for @{tool build}
   477   (see \secref{sec:tool-build}).
   483   (see \secref{sec:tool-build}).