src/Doc/System/Basics.thy
changeset 54705 0dff3326d12a
parent 54683 cf48ddc266e5
child 54937 ce4bf91331e7
equal deleted inserted replaced
54704:ea71549629e2 54705:0dff3326d12a
    93   distribution already contains a global settings file with sensible
    93   distribution already contains a global settings file with sensible
    94   defaults for most variables.  When installing the system, only a few
    94   defaults for most variables.  When installing the system, only a few
    95   of these may have to be adapted (probably @{setting ML_SYSTEM}
    95   of these may have to be adapted (probably @{setting ML_SYSTEM}
    96   etc.).
    96   etc.).
    97   
    97   
    98   \item The file @{verbatim "$ISABELLE_HOME_USER/etc/settings"} (if it
    98   \item The file @{file_unchecked "$ISABELLE_HOME_USER/etc/settings"} (if it
    99   exists) is run in the same way as the site default settings. Note
    99   exists) is run in the same way as the site default settings. Note
   100   that the variable @{setting ISABELLE_HOME_USER} has already been set
   100   that the variable @{setting ISABELLE_HOME_USER} has already been set
   101   before --- usually to something like @{verbatim
   101   before --- usually to something like @{verbatim
   102   "$USER_HOME/.isabelle/IsabelleXXXX"}.
   102   "$USER_HOME/.isabelle/IsabelleXXXX"}.
   103   
   103   
   164   determined from the Isabelle executable that has been invoked.  Do
   164   determined from the Isabelle executable that has been invoked.  Do
   165   not attempt to set @{setting ISABELLE_HOME} yourself from the shell!
   165   not attempt to set @{setting ISABELLE_HOME} yourself from the shell!
   166   
   166   
   167   \item[@{setting_def ISABELLE_HOME_USER}] is the user-specific
   167   \item[@{setting_def ISABELLE_HOME_USER}] is the user-specific
   168   counterpart of @{setting ISABELLE_HOME}. The default value is
   168   counterpart of @{setting ISABELLE_HOME}. The default value is
   169   relative to @{verbatim "$USER_HOME/.isabelle"}, under rare
   169   relative to @{file_unchecked "$USER_HOME/.isabelle"}, under rare
   170   circumstances this may be changed in the global setting file.
   170   circumstances this may be changed in the global setting file.
   171   Typically, the @{setting ISABELLE_HOME_USER} directory mimics
   171   Typically, the @{setting ISABELLE_HOME_USER} directory mimics
   172   @{setting ISABELLE_HOME} to some extend. In particular, site-wide
   172   @{setting ISABELLE_HOME} to some extend. In particular, site-wide
   173   defaults may be overridden by a private @{verbatim
   173   defaults may be overridden by a private @{verbatim
   174   "$ISABELLE_HOME_USER/etc/settings"}.
   174   "$ISABELLE_HOME_USER/etc/settings"}.
   245   ML system and Isabelle version identifier is appended here, too.
   245   ML system and Isabelle version identifier is appended here, too.
   246   
   246   
   247   \item[@{setting_def ISABELLE_BROWSER_INFO}] is the directory where
   247   \item[@{setting_def ISABELLE_BROWSER_INFO}] is the directory where
   248   theory browser information (HTML text, graph data, and printable
   248   theory browser information (HTML text, graph data, and printable
   249   documents) is stored (see also \secref{sec:info}).  The default
   249   documents) is stored (see also \secref{sec:info}).  The default
   250   value is @{verbatim "$ISABELLE_HOME_USER/browser_info"}.
   250   value is @{file_unchecked "$ISABELLE_HOME_USER/browser_info"}.
   251   
   251   
   252   \item[@{setting_def ISABELLE_LOGIC}] specifies the default logic to
   252   \item[@{setting_def ISABELLE_LOGIC}] specifies the default logic to
   253   load if none is given explicitely by the user.  The default value is
   253   load if none is given explicitely by the user.  The default value is
   254   @{verbatim HOL}.
   254   @{verbatim HOL}.
   255   
   255   
   275   for displaying @{verbatim dvi} files.
   275   for displaying @{verbatim dvi} files.
   276   
   276   
   277   \item[@{setting_def ISABELLE_TMP_PREFIX}@{text "\<^sup>*"}] is the
   277   \item[@{setting_def ISABELLE_TMP_PREFIX}@{text "\<^sup>*"}] is the
   278   prefix from which any running @{executable "isabelle-process"}
   278   prefix from which any running @{executable "isabelle-process"}
   279   derives an individual directory for temporary files.  The default is
   279   derives an individual directory for temporary files.  The default is
   280   somewhere in @{verbatim "/tmp"}.
   280   somewhere in @{file_unchecked "/tmp"}.
   281   
   281   
   282   \end{description}
   282   \end{description}
   283 *}
   283 *}
   284 
   284 
   285 
   285 
   323 
   323 
   324   The root of component initialization is @{setting ISABELLE_HOME}
   324   The root of component initialization is @{setting ISABELLE_HOME}
   325   itself.  After initializing all of its sub-components recursively,
   325   itself.  After initializing all of its sub-components recursively,
   326   @{setting ISABELLE_HOME_USER} is included in the same manner (if
   326   @{setting ISABELLE_HOME_USER} is included in the same manner (if
   327   that directory exists).  This allows to install private components
   327   that directory exists).  This allows to install private components
   328   via @{verbatim "$ISABELLE_HOME_USER/etc/components"}, although it is
   328   via @{file_unchecked "$ISABELLE_HOME_USER/etc/components"}, although it is
   329   often more convenient to do that programmatically via the
   329   often more convenient to do that programmatically via the
   330   \verb,init_component, shell function in the \verb,etc/settings,
   330   \verb,init_component, shell function in the \verb,etc/settings,
   331   script of \verb,$ISABELLE_HOME_USER, (or any other component
   331   script of \verb,$ISABELLE_HOME_USER, (or any other component
   332   directory).  For example:
   332   directory).  For example:
   333 \begin{ttbox}
   333 \begin{ttbox}