src/Doc/System/Server.thy
changeset 67940 b4e80f062fbf
parent 67938 da44f151f716
child 67941 49a34b2fa788
equal deleted inserted replaced
67939:544a7a21298e 67940:b4e80f062fbf
   875   argument: & \<open>use_theories_arguments\<close> \\
   875   argument: & \<open>use_theories_arguments\<close> \\
   876   regular result: & \<^verbatim>\<open>OK\<close> \<open>use_theories_results\<close> \\
   876   regular result: & \<^verbatim>\<open>OK\<close> \<open>use_theories_results\<close> \\
   877   \end{tabular}
   877   \end{tabular}
   878 
   878 
   879   \begin{tabular}{ll}
   879   \begin{tabular}{ll}
   880   \<^bold>\<open>type\<close> \<open>theory_name = string | {name: string, pos: position}\<close> \\
       
   881   \end{tabular}
       
   882 
       
   883   \begin{tabular}{ll}
       
   884   \<^bold>\<open>type\<close> \<open>use_theories_arguments =\<close> \\
   880   \<^bold>\<open>type\<close> \<open>use_theories_arguments =\<close> \\
   885   \quad\<open>{session_id: uuid,\<close> \\
   881   \quad\<open>{session_id: uuid,\<close> \\
   886   \quad~~\<open>theories: [theory_name],\<close> \\
   882   \quad~~\<open>theories: [string],\<close> \\
   887   \quad~~\<open>master_dir?: string,\<close> \\
   883   \quad~~\<open>master_dir?: string,\<close> \\
   888   \quad~~\<open>pretty_margin?: double\<close> & \<^bold>\<open>default:\<close> \<^verbatim>\<open>76\<close> \\
   884   \quad~~\<open>pretty_margin?: double\<close> & \<^bold>\<open>default:\<close> \<^verbatim>\<open>76\<close> \\
   889   \quad~~\<open>unicode_symbols?: bool}\<close> \\[2ex]
   885   \quad~~\<open>unicode_symbols?: bool}\<close> \\[2ex]
   890   \end{tabular}
   886   \end{tabular}
   891 
   887 
   923   The \<open>session_id\<close> is the identifier provided by the server, when the session
   919   The \<open>session_id\<close> is the identifier provided by the server, when the session
   924   was created (possibly on a different client connection).
   920   was created (possibly on a different client connection).
   925 
   921 
   926   \<^medskip>
   922   \<^medskip>
   927   The \<open>theories\<close> field specifies theory names as in theory \<^theory_text>\<open>imports\<close> or in
   923   The \<open>theories\<close> field specifies theory names as in theory \<^theory_text>\<open>imports\<close> or in
   928   ROOT \<^bold>\<open>theories\<close>. An explicit source position for these theory name
   924   ROOT \<^bold>\<open>theories\<close>.
   929   specifications may be given, which is occasionally useful for precise error
       
   930   locations.
       
   931 
   925 
   932   \<^medskip> The \<open>master_dir\<close> field specifies the master directory of imported
   926   \<^medskip> The \<open>master_dir\<close> field specifies the master directory of imported
   933   theories: it acts like the ``current working directory'' for locating theory
   927   theories: it acts like the ``current working directory'' for locating theory
   934   files. This may be omitted if all entries of \<open>theories\<close> use a
   928   files. This may be omitted if all entries of \<open>theories\<close> use a
   935   session-qualified theory name (e.g.\ \<^verbatim>\<open>"HOL-Library.AList"\<close>) or absolute
   929   session-qualified theory name (e.g.\ \<^verbatim>\<open>"HOL-Library.AList"\<close>) or absolute