src/Doc/System/Environment.thy
changeset 69854 cc0b3e177b49
parent 69593 3dda49e08b9d
child 71578 d59d557f4ee0
equal deleted inserted replaced
69853:f7c9a1be333f 69854:cc0b3e177b49
   179   \<^path>\<open>$ISABELLE_HOME_USER/browser_info\<close>. For ``system build mode'' (see
   179   \<^path>\<open>$ISABELLE_HOME_USER/browser_info\<close>. For ``system build mode'' (see
   180   \secref{sec:tool-build}), @{setting_def ISABELLE_BROWSER_INFO_SYSTEM} is
   180   \secref{sec:tool-build}), @{setting_def ISABELLE_BROWSER_INFO_SYSTEM} is
   181   used instead; its default is \<^path>\<open>$ISABELLE_HOME/browser_info\<close>.
   181   used instead; its default is \<^path>\<open>$ISABELLE_HOME/browser_info\<close>.
   182 
   182 
   183   \<^descr>[@{setting_def ISABELLE_HEAPS}] is the directory where session heap images,
   183   \<^descr>[@{setting_def ISABELLE_HEAPS}] is the directory where session heap images,
   184   log files, and build databases are stored; its default is \<^path>\<open>$ISABELLE_HOME_USER/heaps\<close>. For ``system build mode'' (see
   184   log files, and build databases are stored; its default is
   185   \secref{sec:tool-build}), @{setting_def ISABELLE_HEAPS_SYSTEM} is used
   185   \<^path>\<open>$ISABELLE_HOME_USER/heaps\<close>. If @{system_option system_heaps} is
   186   instead; its default is \<^path>\<open>$ISABELLE_HOME/heaps\<close>.
   186   \<^verbatim>\<open>true\<close>, @{setting_def ISABELLE_HEAPS_SYSTEM} is used instead; its default
       
   187   is \<^path>\<open>$ISABELLE_HOME/heaps\<close>. See also \secref{sec:tool-build}.
   187 
   188 
   188   \<^descr>[@{setting_def ISABELLE_LOGIC}] specifies the default logic to load if none
   189   \<^descr>[@{setting_def ISABELLE_LOGIC}] specifies the default logic to load if none
   189   is given explicitely by the user. The default value is \<^verbatim>\<open>HOL\<close>.
   190   is given explicitely by the user. The default value is \<^verbatim>\<open>HOL\<close>.
   190 
   191 
   191   \<^descr>[@{setting_def ISABELLE_LINE_EDITOR}] specifies the line editor for the
   192   \<^descr>[@{setting_def ISABELLE_LINE_EDITOR}] specifies the line editor for the
   408     -l NAME      logic session name (default ISABELLE_LOGIC)
   409     -l NAME      logic session name (default ISABELLE_LOGIC)
   409     -m MODE      add print mode for output
   410     -m MODE      add print mode for output
   410     -n           no build of session image on startup
   411     -n           no build of session image on startup
   411     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   412     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   412     -r           bootstrap from raw Poly/ML
   413     -r           bootstrap from raw Poly/ML
   413     -s           system build mode for session image
       
   414 
   414 
   415   Build a logic session image and run the raw Isabelle ML process
   415   Build a logic session image and run the raw Isabelle ML process
   416   in interactive mode, with line editor ISABELLE_LINE_EDITOR.\<close>}
   416   in interactive mode, with line editor ISABELLE_LINE_EDITOR.\<close>}
   417 
   417 
   418   \<^medskip>
   418   \<^medskip>
   426   relevant for Isabelle/Pure development.
   426   relevant for Isabelle/Pure development.
   427 
   427 
   428   \<^medskip>
   428   \<^medskip>
   429   Options \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-m\<close>, \<^verbatim>\<open>-o\<close> have the same meaning as for @{tool process}
   429   Options \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-m\<close>, \<^verbatim>\<open>-o\<close> have the same meaning as for @{tool process}
   430   (\secref{sec:tool-process}).
   430   (\secref{sec:tool-process}).
   431 
       
   432   Option \<^verbatim>\<open>-s\<close> has the same meaning as for @{tool build}
       
   433   (\secref{sec:tool-build}).
       
   434 
   431 
   435   \<^medskip>
   432   \<^medskip>
   436   The Isabelle/ML process is run through the line editor that is specified via
   433   The Isabelle/ML process is run through the line editor that is specified via
   437   the settings variable @{setting ISABELLE_LINE_EDITOR} (e.g.\
   434   the settings variable @{setting ISABELLE_LINE_EDITOR} (e.g.\
   438   @{executable_def rlwrap} for GNU readline); the fall-back is to use plain
   435   @{executable_def rlwrap} for GNU readline); the fall-back is to use plain