src/Doc/System/Environment.thy
changeset 68514 b20980997cd2
parent 68477 f090b313fdc8
child 68523 ccacc84e0251
equal deleted inserted replaced
68513:88b0e63d58a5 68514:b20980997cd2
    71   variables. Such advanced features should be added only with great care,
    71   variables. Such advanced features should be added only with great care,
    72   though. In particular, external environment references should be kept at a
    72   though. In particular, external environment references should be kept at a
    73   minimum.
    73   minimum.
    74 
    74 
    75   \<^medskip>
    75   \<^medskip>
    76   A few variables are somewhat special, e.g. @{setting_def ISABELLE_TOOL} is
    76   A few variables are somewhat special, e.g.\ @{setting_def ISABELLE_TOOL} is
    77   set automatically to the absolute path name of the @{executable isabelle}
    77   set automatically to the absolute path name of the @{executable isabelle}
    78   executables.
    78   executables.
    79 
    79 
    80   \<^medskip>
    80   \<^medskip>
    81   Note that the settings environment may be inspected with the @{tool getenv}
    81   Note that the settings environment may be inspected with the @{tool getenv}
   205   \<^descr>[@{setting_def ISABELLE_TMP_PREFIX}\<open>\<^sup>*\<close>] is the prefix from which any
   205   \<^descr>[@{setting_def ISABELLE_TMP_PREFIX}\<open>\<^sup>*\<close>] is the prefix from which any
   206   running Isabelle ML process derives an individual directory for temporary
   206   running Isabelle ML process derives an individual directory for temporary
   207   files.
   207   files.
   208 
   208 
   209   \<^descr>[@{setting_def ISABELLE_TOOL_JAVA_OPTIONS}] is passed to the \<^verbatim>\<open>java\<close>
   209   \<^descr>[@{setting_def ISABELLE_TOOL_JAVA_OPTIONS}] is passed to the \<^verbatim>\<open>java\<close>
   210   executable when running Isabelle tools (e.g. @{tool build}). This is
   210   executable when running Isabelle tools (e.g.\ @{tool build}). This is
   211   occasionally helpful to provide more heap space, via additional options like
   211   occasionally helpful to provide more heap space, via additional options like
   212   \<^verbatim>\<open>-Xms1g -Xmx4g\<close>.
   212   \<^verbatim>\<open>-Xms1g -Xmx4g\<close>.
   213 \<close>
   213 \<close>
   214 
   214 
   215 
   215