src/Doc/System/Server.thy
changeset 71925 bf085daea304
parent 71521 e977609c30eb
child 72515 c7038c397ae3
equal deleted inserted replaced
71924:e5df9c8d9d4b 71925:bf085daea304
   513   connections and may be shared by different clients, as long as the internal
   513   connections and may be shared by different clients, as long as the internal
   514   session identifier is known.
   514   session identifier is known.
   515 
   515 
   516   \<^item> \<^bold>\<open>type\<close> \<open>node = {node_name: string, theory_name: string}\<close> represents the
   516   \<^item> \<^bold>\<open>type\<close> \<open>node = {node_name: string, theory_name: string}\<close> represents the
   517   internal node name of a theory. The \<open>node_name\<close> is derived from the
   517   internal node name of a theory. The \<open>node_name\<close> is derived from the
   518   canonical theory file-name (e.g.\ \<^verbatim>\<open>"~~/src/HOL/ex/Seq.thy"\<close> after
   518   canonical theory file-name (e.g.\ \<^verbatim>\<open>"~~/src/HOL/Examples/Seq.thy"\<close> after
   519   normalization within the file-system). The \<open>theory_name\<close> is the
   519   normalization within the file-system). The \<open>theory_name\<close> is the
   520   session-qualified theory name (e.g.\ \<^verbatim>\<open>HOL-ex.Seq\<close>).
   520   session-qualified theory name (e.g.\ \<^verbatim>\<open>HOL-Examples.Seq\<close>).
   521 
   521 
   522   \<^item> \<^bold>\<open>type\<close> \<open>node_status = {ok: bool, total: int, unprocessed: int, running:
   522   \<^item> \<^bold>\<open>type\<close> \<open>node_status = {ok: bool, total: int, unprocessed: int, running:
   523   int, warned: int, failed: int, finished: int, canceled: bool, consolidated:
   523   int, warned: int, failed: int, finished: int, canceled: bool, consolidated:
   524   bool, percentage: int}\<close> represents a formal theory node status of the PIDE
   524   bool, percentage: int}\<close> represents a formal theory node status of the PIDE
   525   document model as follows.
   525   document model as follows.
   973 
   973 
   974   \<^medskip>
   974   \<^medskip>
   975   The \<open>master_dir\<close> field specifies the master directory of imported theories:
   975   The \<open>master_dir\<close> field specifies the master directory of imported theories:
   976   it acts like the ``current working directory'' for locating theory files.
   976   it acts like the ``current working directory'' for locating theory files.
   977   This is irrelevant for \<open>theories\<close> with an absolute path name (e.g.\
   977   This is irrelevant for \<open>theories\<close> with an absolute path name (e.g.\
   978   \<^verbatim>\<open>"~~/src/HOL/ex/Seq.thy"\<close>) or session-qualified theory name (e.g.\
   978   \<^verbatim>\<open>"~~/src/HOL/Examples/Seq.thy"\<close>) or session-qualified theory name (e.g.\
   979   \<^verbatim>\<open>"HOL-ex/Seq"\<close>).
   979   \<^verbatim>\<open>"HOL-Examples.Seq"\<close>).
   980 
   980 
   981   \<^medskip>
   981   \<^medskip>
   982   The \<open>pretty_margin\<close> field specifies the line width for pretty-printing. The
   982   The \<open>pretty_margin\<close> field specifies the line width for pretty-printing. The
   983   default is suitable for classic console output. Formatting happens at the
   983   default is suitable for classic console output. Formatting happens at the
   984   end of \<^verbatim>\<open>use_theories\<close>, when all prover messages are exported to the client.
   984   end of \<^verbatim>\<open>use_theories\<close>, when all prover messages are exported to the client.
  1024 
  1024 
  1025 text \<open>
  1025 text \<open>
  1026   Process some example theory from the Isabelle distribution, within the
  1026   Process some example theory from the Isabelle distribution, within the
  1027   context of an already started session for Isabelle/HOL (see also
  1027   context of an already started session for Isabelle/HOL (see also
  1028   \secref{sec:command-session-start}):
  1028   \secref{sec:command-session-start}):
  1029   @{verbatim [display] \<open>use_theories {"session_id": ..., "theories": ["~~/src/HOL/ex/Seq"]}\<close>}
  1029   @{verbatim [display] \<open>use_theories {"session_id": ..., "theories": ["~~/src/HOL/Examples/Seq"]}\<close>}
  1030 
  1030 
  1031   \<^medskip>
  1031   \<^medskip>
  1032   Process some example theories in the context of their (single) parent
  1032   Process some example theories in the context of their (single) parent
  1033   session:
  1033   session:
  1034 
  1034