src/Doc/System/Sessions.thy
changeset 77563 cbb49fe8e5a2
parent 77554 4465d9dff448
child 77572 7c0c5bce3e60
--- a/src/Doc/System/Sessions.thy	Tue Mar 07 16:23:48 2023 +0100
+++ b/src/Doc/System/Sessions.thy	Tue Mar 07 22:17:47 2023 +0100
@@ -570,7 +570,7 @@
   database of the given session. Its command-line usage is:
 
   @{verbatim [display]
-\<open>Usage: isabelle log [OPTIONS] [SESSIONS ...]
+\<open>Usage: isabelle build_log [OPTIONS] [SESSIONS ...]
 
   Options are:
     -H REGEX     filter messages by matching against head
@@ -628,16 +628,16 @@
 text \<open>
   Print messages from theory \<^verbatim>\<open>HOL.Nat\<close> of session \<^verbatim>\<open>HOL\<close>, using Unicode
   rendering of Isabelle symbols and a margin of 100 characters:
-  @{verbatim [display] \<open>  isabelle log -T HOL.Nat -U -m 100 HOL\<close>}
+  @{verbatim [display] \<open>  isabelle build_log -T HOL.Nat -U -m 100 HOL\<close>}
 
   Print warnings about ambiguous input (inner syntax) of session
   \<^verbatim>\<open>HOL-Library\<close>, which is built beforehand:
   @{verbatim [display] \<open>  isabelle build HOL-Library
-  isabelle log -H "Warning" -M "Ambiguous input" HOL-Library\<close>}
+  isabelle build_log -H "Warning" -M "Ambiguous input" HOL-Library\<close>}
 
   Print all errors from all sessions, e.g. from a partial build of
   Isabelle/AFP:
-  @{verbatim [display] \<open>  isabelle log -H "Error" $(isabelle sessions -a -d AFP/thys)\<close>}
+  @{verbatim [display] \<open>  isabelle build_log -H "Error" $(isabelle sessions -a -d AFP/thys)\<close>}
 \<close>