src/Doc/System/Server.thy
changeset 68957 eef4e983fd9d
parent 68947 ea804c814693
child 69464 2323dce4a0db
equal deleted inserted replaced
68956:122c0d6cb790 68957:eef4e983fd9d
   475   error messages in particular. These occur routinely with \<^verbatim>\<open>ERROR\<close> or
   475   error messages in particular. These occur routinely with \<^verbatim>\<open>ERROR\<close> or
   476   \<^verbatim>\<open>FAILED\<close> replies, but also as initial command syntax errors (which are
   476   \<^verbatim>\<open>FAILED\<close> replies, but also as initial command syntax errors (which are
   477   omitted in the command specifications below).
   477   omitted in the command specifications below).
   478 
   478 
   479   \<^item> \<^bold>\<open>type\<close>~\<open>theory_progress = {kind:\<close>~\<^verbatim>\<open>"writeln"\<close>\<open>, message: string, theory:
   479   \<^item> \<^bold>\<open>type\<close>~\<open>theory_progress = {kind:\<close>~\<^verbatim>\<open>"writeln"\<close>\<open>, message: string, theory:
   480   string, session: string}\<close> reports formal progress in loading theories (e.g.\
   480   string, session: string, percentage?: int}\<close> reports formal progress in
   481   when building a session image). Apart from a regular output message, it also
   481   loading theories (e.g.\ when building a session image). Apart from a regular
   482   reveals the formal theory name (e.g.\ \<^verbatim>\<open>"HOL.Nat"\<close>) and session name (e.g.\
   482   output message, it also reveals the formal theory name (e.g.\ \<^verbatim>\<open>"HOL.Nat"\<close>)
   483   \<^verbatim>\<open>"HOL"\<close>). Note that some rare theory names lack a proper session prefix,
   483   and session name (e.g.\ \<^verbatim>\<open>"HOL"\<close>). Note that some rare theory names lack a
   484   e.g.\ theory \<^verbatim>\<open>"Main"\<close> in session \<^verbatim>\<open>"HOL"\<close>.
   484   proper session prefix, e.g.\ theory \<^verbatim>\<open>"Main"\<close> in session \<^verbatim>\<open>"HOL"\<close>. The
       
   485   optional percentage has the same meaning as in \<^bold>\<open>type\<close>~\<open>node_status\<close> below.
   485 
   486 
   486   \<^item> \<^bold>\<open>type\<close>~\<open>timing = {elapsed: double, cpu: double, gc: double}\<close> refers to
   487   \<^item> \<^bold>\<open>type\<close>~\<open>timing = {elapsed: double, cpu: double, gc: double}\<close> refers to
   487   common Isabelle timing information in seconds, usually with a precision of
   488   common Isabelle timing information in seconds, usually with a precision of
   488   three digits after the point (whole milliseconds).
   489   three digits after the point (whole milliseconds).
   489 
   490