src/Doc/System/Sessions.thy
changeset 77616 29effd67d8a8
parent 77572 7c0c5bce3e60
child 77647 c14db5d67400
--- a/src/Doc/System/Sessions.thy	Sat Mar 11 14:19:09 2023 +0100
+++ b/src/Doc/System/Sessions.thy	Sat Mar 11 14:49:53 2023 +0100
@@ -326,7 +326,8 @@
     -b           include $ISABELLE_BUILD_OPTIONS
     -g OPTION    get value of OPTION
     -l           list options
-    -x FILE      export to FILE in YXML format
+    -t TAGS      restrict list to given tags (comma-separated)
+    -x FILE      export options to FILE in YXML format
 
   Report Isabelle system options, augmented by MORE_OPTIONS given as
   arguments NAME=VAL or NAME.\<close>}
@@ -338,7 +339,8 @@
   of @{setting ISABELLE_BUILD_OPTIONS}, cf.\ \secref{sec:tool-build}.
 
   Option \<^verbatim>\<open>-g\<close> prints the value of the given option. Option \<^verbatim>\<open>-l\<close> lists all
-  options with their declaration and current value.
+  options with their declaration and current value. Option \<^verbatim>\<open>-t\<close> restricts the
+  listing to given tags (as comma-separated list), e.g. \<^verbatim>\<open>-t build,document\<close>.
 
   Option \<^verbatim>\<open>-x\<close> specifies a file to export the result in YXML format, instead
   of printing it in human-readable form.