src/Doc/System/Server.thy
changeset 67931 f7917c15b566
parent 67927 0b70405b3969
child 67937 91eb307511bb
equal deleted inserted replaced
67930:7dff1186daf3 67931:f7917c15b566
   464   Isabelle symbols, see @{ML_type Symbol.symbol} in Isabelle/ML @{cite
   464   Isabelle symbols, see @{ML_type Symbol.symbol} in Isabelle/ML @{cite
   465   "isabelle-implementation"}. The position \<open>id\<close> belongs to the representation
   465   "isabelle-implementation"}. The position \<open>id\<close> belongs to the representation
   466   of command transactions in the Isabelle/PIDE protocol: it normally does not
   466   of command transactions in the Isabelle/PIDE protocol: it normally does not
   467   occur in externalized positions.
   467   occur in externalized positions.
   468 
   468 
   469   \<^item> \<^bold>\<open>type\<close>~\<open>message = {kind?: string, message: string, pos?: position}\<close> where
   469   \<^item> \<^bold>\<open>type\<close>~\<open>message = {kind: string, message: string, pos?: position}\<close> where
   470   the \<open>kind\<close> provides some hint about the role and importance of the message.
   470   the \<open>kind\<close> provides some hint about the role and importance of the message.
   471   The main message kinds are \<^verbatim>\<open>writeln\<close> (for regular output), \<^verbatim>\<open>warning\<close>,
   471   The main message kinds are \<^verbatim>\<open>writeln\<close> (for regular output), \<^verbatim>\<open>warning\<close>,
   472   \<^verbatim>\<open>error\<close>. Messages without explicit kind can be treated like \<^verbatim>\<open>writeln\<close>.
   472   \<^verbatim>\<open>error\<close>.
   473 
   473 
   474   \<^item> \<^bold>\<open>type\<close>~\<open>error_message = {kind:\<close>~\<^verbatim>\<open>"error"\<close>\<open>, message: string}\<close> refers to
   474   \<^item> \<^bold>\<open>type\<close>~\<open>error_message = {kind:\<close>~\<^verbatim>\<open>"error"\<close>\<open>, message: string}\<close> refers to
   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).
   979 
   979 
   980   \<^item> \<open>status\<close>: the overall node status, e.g.\ see the visualization in the
   980   \<^item> \<open>status\<close>: the overall node status, e.g.\ see the visualization in the
   981   \<open>Theories\<close> panel of Isabelle/jEdit @{cite "isabelle-jedit"};
   981   \<open>Theories\<close> panel of Isabelle/jEdit @{cite "isabelle-jedit"};
   982 
   982 
   983   \<^item> \<open>messages\<close>: the main bulk of prover messages produced in this theory
   983   \<^item> \<open>messages\<close>: the main bulk of prover messages produced in this theory
   984   (\<^verbatim>\<open>writeln\<close>, \<^verbatim>\<open>warning\<close>, \<^verbatim>\<open>error\<close>, etc.).
   984   (with kind \<^verbatim>\<open>writeln\<close>, \<^verbatim>\<open>warning\<close>, \<^verbatim>\<open>error\<close>).
   985 \<close>
   985 \<close>
   986 
   986 
   987 
   987 
   988 subsubsection \<open>Examples\<close>
   988 subsubsection \<open>Examples\<close>
   989 
   989