doc-src/System/Thy/Basics.thy
changeset 36196 cbb9ee265cdd
parent 33952 5e9ddf000d97
child 38253 3d4e521014f7
equal deleted inserted replaced
36195:9c098598db2a 36196:cbb9ee265cdd
   160   changed in the global setting file.  Typically, the @{setting
   160   changed in the global setting file.  Typically, the @{setting
   161   ISABELLE_HOME_USER} directory mimics @{setting ISABELLE_HOME} to
   161   ISABELLE_HOME_USER} directory mimics @{setting ISABELLE_HOME} to
   162   some extend. In particular, site-wide defaults may be overridden by
   162   some extend. In particular, site-wide defaults may be overridden by
   163   a private @{verbatim "$ISABELLE_HOME_USER/etc/settings"}.
   163   a private @{verbatim "$ISABELLE_HOME_USER/etc/settings"}.
   164   
   164   
       
   165   \item[@{setting_def ISABELLE_PLATFORM}@{text "\<^sup>*"}] is automatically
       
   166   set to a symbolic identifier for the underlying hardware and
       
   167   operating system.  The Isabelle platform identification always
       
   168   refers to the 32 bit variant, even this is a 64 bit machine.  Note
       
   169   that the ML or Java runtime may have a different idea, depending on
       
   170   which binaries are actually run.
       
   171 
       
   172   \item[@{setting_def ISABELLE_PLATFORM64}@{text "\<^sup>*"}] is similar to
       
   173   @{setting ISABELLE_PLATFORM} but refers to the proper 64 bit variant
       
   174   on a platform that supports this; the value is empty for 32 bit.
       
   175 
   165   \item[@{setting_def ISABELLE_PROCESS}@{text "\<^sup>*"}, @{setting
   176   \item[@{setting_def ISABELLE_PROCESS}@{text "\<^sup>*"}, @{setting
   166   ISABELLE_TOOL}@{text "\<^sup>*"}] are automatically set to the full path
   177   ISABELLE_TOOL}@{text "\<^sup>*"}] are automatically set to the full path
   167   names of the @{executable "isabelle-process"} and @{executable
   178   names of the @{executable "isabelle-process"} and @{executable
   168   isabelle} executables, respectively.  Thus other tools and scripts
   179   isabelle} executables, respectively.  Thus other tools and scripts
   169   need not assume that the @{"file" "$ISABELLE_HOME/bin"} directory is
   180   need not assume that the @{"file" "$ISABELLE_HOME/bin"} directory is