src/Doc/System/Sessions.thy
changeset 76107 4dedb6e2dac2
parent 76089 13ae8dff47b6
child 76110 0605eb327e60
--- a/src/Doc/System/Sessions.thy	Sat Sep 10 15:48:36 2022 +0200
+++ b/src/Doc/System/Sessions.thy	Sat Sep 10 16:12:52 2022 +0200
@@ -865,6 +865,7 @@
     -R           refer to requirements of selected sessions
     -X NAME      exclude sessions from group NAME and all descendants
     -a           select all sessions
+    -b           follow session build dependencies (default: source imports)
     -d DIR       include session directory
     -g NAME      select session group NAME
     -x NAME      exclude session NAME and all descendants
@@ -884,7 +885,15 @@
   @{verbatim [display] \<open>  isabelle sessions -a\<close>}
 
   \<^medskip>
-  Sessions that are based on \<^verbatim>\<open>ZF\<close> (and required by it):
+  Sessions that are imported by \<^verbatim>\<open>ZF\<close>:
+  @{verbatim [display] \<open>  isabelle sessions ZF\<close>}
+
+  \<^medskip>
+  Sessions that are required to build \<^verbatim>\<open>ZF\<close>:
+  @{verbatim [display] \<open>  isabelle sessions -b ZF\<close>}
+
+  \<^medskip>
+  Sessions that are based on \<^verbatim>\<open>ZF\<close> (and imported by it):
   @{verbatim [display] \<open>  isabelle sessions -B ZF\<close>}
 
   \<^medskip>