src/Doc/System/Sessions.thy
changeset 59891 9ce697050455
parent 59446 4427f04fca57
child 59892 2a616319c171
--- a/src/Doc/System/Sessions.thy	Wed Apr 01 13:32:32 2015 +0200
+++ b/src/Doc/System/Sessions.thy	Wed Apr 01 15:41:08 2015 +0200
@@ -284,6 +284,7 @@
     -d DIR       include session directory
     -g NAME      select session group NAME
     -j INT       maximum number of parallel jobs (default 1)
+    -k KEYWORD   check theory sources for conflicts with proposed keywords
     -l           list session source files
     -n           no build -- test dependencies only
     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
@@ -369,7 +370,12 @@
   \medskip Option @{verbatim "-v"} increases the general level of
   verbosity.  Option @{verbatim "-l"} lists the source files that
   contribute to a session.
-\<close>
+
+  \medskip Option @{verbatim "-k"} specifies a newly proposed keyword for
+  outer syntax (multiple uses allowed). The theory sources are checked for
+  conflicts wrt.\ this hypothetical change of syntax, e.g.\ to reveal
+  occurrences of identifiers that need to be quoted.\<close>
+
 
 subsubsection \<open>Examples\<close>