src/Doc/System/Sessions.thy
changeset 72876 626fcaebd049
parent 72769 4dcd05a26795
child 72878 80465b791f95
equal deleted inserted replaced
72875:847c6fb05a21 72876:626fcaebd049
   507   anything yet:
   507   anything yet:
   508   @{verbatim [display] \<open>isabelle build -D '$AFP' -R -v -n\<close>}
   508   @{verbatim [display] \<open>isabelle build -D '$AFP' -R -v -n\<close>}
   509 \<close>
   509 \<close>
   510 
   510 
   511 
   511 
       
   512 section \<open>Print messages from build database \label{sec:tool-log}\<close>
       
   513 
       
   514 text \<open>
       
   515   The @{tool_def "log"} tool prints prover messages from the build
       
   516   database of the given session. Its command-line usage is:
       
   517 
       
   518   @{verbatim [display]
       
   519 \<open>Usage: isabelle log [OPTIONS] SESSION
       
   520 
       
   521   Options are:
       
   522     -T NAME      restrict to given theories (multiple options possible)
       
   523     -U           output Unicode symbols
       
   524     -m MARGIN    margin for pretty printing (default: 76.0)
       
   525     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
       
   526 
       
   527   Print messages from the build database of the given session, without any
       
   528   checks against current sources: results from a failed build can be
       
   529   printed as well.\<close>}
       
   530 
       
   531   The specified session database is taken as is, independently of the current
       
   532   session structure and theories sources. The order of messages follows the
       
   533   source positions of source files; thus the erratic evaluation of parallel
       
   534   processing rarely matters. There is \<^emph>\<open>no\<close> implicit build process involved,
       
   535   so it is possible to retrieve error messages from a failed session as well.
       
   536 
       
   537   \<^medskip> Option \<^verbatim>\<open>-o\<close> allows to change system options, as in @{tool build}
       
   538   (\secref{sec:tool-build}). This may affect the storage space for the build
       
   539   database, notably via @{system_option system_heaps}, or @{system_option
       
   540   build_database_server} and its relatives.
       
   541 
       
   542   \<^medskip> Option \<^verbatim>\<open>-T\<close> restricts output to given theories: multiple entries are
       
   543   possible by repeating this option on the command-line. The default is to
       
   544   refer to \<^emph>\<open>all\<close> theories that were used in original session build process.
       
   545 
       
   546   \<^medskip> Options \<^verbatim>\<open>-m\<close> and \<^verbatim>\<open>-U\<close> modify pretty printing and output of Isabelle
       
   547   symbols. The default is for an old-fashioned ASCII terminal at 80 characters
       
   548   per line (76 + 4 characters to prefix warnings or errors).
       
   549 \<close>
       
   550 
       
   551 subsubsection \<open>Examples\<close>
       
   552 
       
   553 text \<open>
       
   554   Print messages from theory \<^verbatim>\<open>HOL.Nat\<close> of session \<^verbatim>\<open>HOL\<close>, using Unicode
       
   555   rendering of Isabelle symbols and a margin of 100 characters:
       
   556   @{verbatim [display] \<open>isabelle log -T HOL.Nat -U -m 100 HOL\<close>}
       
   557 \<close>
       
   558 
       
   559 
   512 section \<open>Retrieve theory exports \label{sec:tool-export}\<close>
   560 section \<open>Retrieve theory exports \label{sec:tool-export}\<close>
   513 
   561 
   514 text \<open>
   562 text \<open>
   515   The @{tool_def "export"} tool retrieves theory exports from the session
   563   The @{tool_def "export"} tool retrieves theory exports from the session
   516   database. Its command-line usage is: @{verbatim [display]
   564   database. Its command-line usage is: @{verbatim [display]