doc-src/System/Thy/Misc.thy
changeset 41511 2fe62d602681
parent 40800 330eb65c9469
child 41512 8445396e1e39
equal deleted inserted replaced
41510:75c6c4069938 41511:2fe62d602681
   279 
   279 
   280 
   280 
   281 section {* Output the version identifier of the Isabelle distribution *}
   281 section {* Output the version identifier of the Isabelle distribution *}
   282 
   282 
   283 text {*
   283 text {*
   284   The @{tool_def version} utility outputs the full version string of
   284   The @{tool_def version} utility displays Isabelle version information:
   285   the Isabelle distribution being used, e.g.\ ``@{verbatim
   285 \begin{ttbox}
   286   "Isabelle2008: June 2008"}.  There are no options nor arguments.
   286 Usage: isabelle version [OPTIONS]
       
   287 
       
   288   Options are:
       
   289     -i           short identification (derived from Mercurial id)
       
   290 
       
   291   Display Isabelle version information.
       
   292 \end{ttbox}
       
   293 
       
   294   \medskip The default is to output the full version string of the
       
   295   Isabelle distribution, e.g.\ ``@{verbatim "Isabelle2008: June 2008"}.
       
   296 
       
   297   The @{verbatim "-i"} option produces a short identification derived
       
   298   from the Mercurial id of the @{setting ISABELLE_HOME} directory.
   287 *}
   299 *}
   288 
   300 
   289 
   301 
   290 section {* Convert XML to YXML *}
   302 section {* Convert XML to YXML *}
   291 
   303