src/Doc/System/Sessions.thy
changeset 66748 3efac90a11a7
parent 66745 e7ac579b883c
child 66759 918f15c9367a
--- a/src/Doc/System/Sessions.thy	Mon Oct 02 13:40:51 2017 +0200
+++ b/src/Doc/System/Sessions.thy	Mon Oct 02 13:45:36 2017 +0200
@@ -417,6 +417,14 @@
   @{verbatim [display] \<open>isabelle build -b -g main\<close>}
 
   \<^smallskip>
+  Build all descendants (and requirements) of \<^verbatim>\<open>FOL\<close> and \<^verbatim>\<open>ZF\<close>:
+  @{verbatim [display] \<open>isabelle build -B FOL -B ZF\<close>}
+
+  \<^smallskip>
+  Build all sessions where sources have changed (ignoring heaps):
+  @{verbatim [display] \<open>isabelle build -a -S\<close>}
+
+  \<^smallskip>
   Provide a general overview of the status of all Isabelle sessions, without
   building anything:
   @{verbatim [display] \<open>isabelle build -a -n -v\<close>}