src/Doc/System/Environment.thy
changeset 71904 70442ddbfb15
parent 71903 0da5fb75088a
child 72252 3b17e7688dc6
equal deleted inserted replaced
71903:0da5fb75088a 71904:70442ddbfb15
   246     (with leading \<^verbatim>\<open>/\<close>) or relative to the component's main directory.
   246     (with leading \<^verbatim>\<open>/\<close>) or relative to the component's main directory.
   247 
   247 
   248   The root of component initialization is @{setting ISABELLE_HOME} itself.
   248   The root of component initialization is @{setting ISABELLE_HOME} itself.
   249   After initializing all of its sub-components recursively, @{setting
   249   After initializing all of its sub-components recursively, @{setting
   250   ISABELLE_HOME_USER} is included in the same manner (if that directory
   250   ISABELLE_HOME_USER} is included in the same manner (if that directory
   251   exists). This allows to install private components via \<^path>\<open>$ISABELLE_HOME_USER/etc/components\<close>, although it is often more convenient
   251   exists). This allows to install private components via
   252   to do that programmatically via the \<^bash_function>\<open>init_component\<close> shell function in the
   252   \<^path>\<open>$ISABELLE_HOME_USER/etc/components\<close>, although it is often more
   253   \<^verbatim>\<open>etc/settings\<close> script of \<^verbatim>\<open>$ISABELLE_HOME_USER\<close> (or any other component
   253   convenient to do that programmatically via the
   254   directory). For example:
   254   \<^bash_function>\<open>init_component\<close> shell function in the \<^verbatim>\<open>etc/settings\<close>
       
   255   script of \<^verbatim>\<open>$ISABELLE_HOME_USER\<close> (or any other component directory). For
       
   256   example:
   255   @{verbatim [display] \<open>init_component "$HOME/screwdriver-2.0"\<close>}
   257   @{verbatim [display] \<open>init_component "$HOME/screwdriver-2.0"\<close>}
   256 
   258 
   257   This is tolerant wrt.\ missing component directories, but might produce a
   259   This is tolerant wrt.\ missing component directories, but might produce a
   258   warning.
   260   warning.
   259 
   261