src/Doc/System/Server.thy
changeset 67922 9e668ae81f97
parent 67921 1722384ffd4a
child 67923 3e072441c96a
equal deleted inserted replaced
67921:1722384ffd4a 67922:9e668ae81f97
   630   \<^bold>\<open>type\<close> \<open>session_build_args =\<close> \\
   630   \<^bold>\<open>type\<close> \<open>session_build_args =\<close> \\
   631   \quad\<open>{session: string,\<close> \\
   631   \quad\<open>{session: string,\<close> \\
   632   \quad~~\<open>preferences?: string,\<close> & \<^bold>\<open>default:\<close> server preferences \\
   632   \quad~~\<open>preferences?: string,\<close> & \<^bold>\<open>default:\<close> server preferences \\
   633   \quad~~\<open>options?: [string],\<close> \\
   633   \quad~~\<open>options?: [string],\<close> \\
   634   \quad~~\<open>dirs?: [string],\<close> \\
   634   \quad~~\<open>dirs?: [string],\<close> \\
   635   \quad~~\<open>all_known?: bool,\<close> \\
   635   \quad~~\<open>include_sessions: [string],\<close> \\
   636   \quad~~\<open>system_mode?: bool,\<close> \\
   636   \quad~~\<open>system_mode?: bool,\<close> \\
   637   \quad~~\<open>verbose?: bool}\<close> \\[2ex]
   637   \quad~~\<open>verbose?: bool}\<close> \\[2ex]
   638   \end{tabular}
   638   \end{tabular}
   639 
   639 
   640   \begin{tabular}{ll}
   640   \begin{tabular}{ll}
   692   The \<open>dirs\<close> field specifies additional directories for session ROOT and ROOTS
   692   The \<open>dirs\<close> field specifies additional directories for session ROOT and ROOTS
   693   files (\secref{sec:session-root}). This augments the name space of available
   693   files (\secref{sec:session-root}). This augments the name space of available
   694   sessions; see also option \<^verbatim>\<open>-d\<close> in @{tool build}.
   694   sessions; see also option \<^verbatim>\<open>-d\<close> in @{tool build}.
   695 
   695 
   696   \<^medskip>
   696   \<^medskip>
   697   The \<open>all_known\<close> field set to \<^verbatim>\<open>true\<close> includes all sessions from reachable
   697   The \<open>include_sessions\<close> field specifies sessions whose theories should be
   698   ROOT entries into the name space of theories. This is relevant for proper
   698   included in the overall name space of session-qualified theory names. This
   699   session-qualified names, instead of referring to theory file names. The
   699   corresponds to a \<^bold>\<open>sessions\<close> specification in ROOT files
   700   option enables the \<^verbatim>\<open>use_theories\<close> command
   700   (\secref{sec:session-root}). It enables the \<^verbatim>\<open>use_theories\<close> command
   701   (\secref{sec:command-use-theories}) to refer to arbitrary theories from
   701   (\secref{sec:command-use-theories}) to refer to sources from other sessions
   702   other sessions, but considerable time is required to explore all accessible
   702   in a robust manner, instead of relying on directory locations.
   703   session directories and theory dependencies.
       
   704 
   703 
   705   \<^medskip>
   704   \<^medskip>
   706   The \<open>system_mode\<close> field set to \<^verbatim>\<open>true\<close> stores resulting session images and
   705   The \<open>system_mode\<close> field set to \<^verbatim>\<open>true\<close> stores resulting session images and
   707   log files in @{path "$ISABELLE_HOME/heaps"} instead of the default location
   706   log files in @{path "$ISABELLE_HOME/heaps"} instead of the default location
   708   @{setting ISABELLE_OUTPUT} (which is normally in @{setting
   707   @{setting ISABELLE_OUTPUT} (which is normally in @{setting
   987   context of an already started session for Isabelle/HOL (see also
   986   context of an already started session for Isabelle/HOL (see also
   988   \secref{sec:command-session-start}):
   987   \secref{sec:command-session-start}):
   989   @{verbatim [display] \<open>use_theories {"session_id": ..., "theories": ["~~/src/HOL/Isar_Examples/Drinker"]}\<close>}
   988   @{verbatim [display] \<open>use_theories {"session_id": ..., "theories": ["~~/src/HOL/Isar_Examples/Drinker"]}\<close>}
   990 
   989 
   991   \<^medskip>
   990   \<^medskip>
   992   Process some example theories that import other theories via
       
   993   session-qualified theory names:
       
   994 
       
   995   @{verbatim [display] \<open>session_start {"session": "HOL", "all_known": true}
       
   996 use_theories {"session_id": ..., "theories": ["~~/src/HOL/Unix/Unix"]}
       
   997 session_stop {"session_id": ...}\<close>}
       
   998 
       
   999   The option \<open>all_known\<close> has been used here to the full name space of
       
  1000   session-qualified theory names accessible in this session. This is also the
       
  1001   default in Isabelle/jEdit, although it requires significant startup time.
       
  1002 
       
  1003   \<^medskip>
       
  1004   Process some example theories in the context of their (single) parent
   991   Process some example theories in the context of their (single) parent
  1005   session:
   992   session:
  1006 
   993 
  1007   @{verbatim [display] \<open>session_start {"session": "HOL-Library"}
   994   @{verbatim [display] \<open>session_start {"session": "HOL-Library"}
  1008 use_theories {"session_id": ..., "theories": ["~~/src/HOL/Unix/Unix"]}
   995 use_theories {"session_id": ..., "theories": ["~~/src/HOL/Unix/Unix"]}
  1009 session_stop {"session_id": ...}\<close>}
   996 session_stop {"session_id": ...}\<close>}
       
   997 
       
   998   \<^medskip>
       
   999   Process some example theories that import other theories via
       
  1000   session-qualified theory names:
       
  1001 
       
  1002   @{verbatim [display] \<open>session_start {"session": "HOL", "include_sessions": ["HOL-Unix"]}
       
  1003 use_theories {"session_id": ..., "theories": ["HOL-Unix.Unix"]}
       
  1004 session_stop {"session_id": ...}\<close>}
  1010 \<close>
  1005 \<close>
  1011 
  1006 
  1012 end
  1007 end