src/Doc/System/Environment.thy
changeset 66733 9180953b976b
parent 66732 e566fb4d43d4
child 66789 feb36b73a7f0
equal deleted inserted replaced
66732:e566fb4d43d4 66733:9180953b976b
   171   images, which is useful for cross-platform installations. The value of
   171   images, which is useful for cross-platform installations. The value of
   172   @{setting ML_IDENTIFIER} is automatically obtained by composing the values
   172   @{setting ML_IDENTIFIER} is automatically obtained by composing the values
   173   of @{setting ML_SYSTEM}, @{setting ML_PLATFORM} and the Isabelle version
   173   of @{setting ML_SYSTEM}, @{setting ML_PLATFORM} and the Isabelle version
   174   values.
   174   values.
   175 
   175 
   176   \<^descr>[@{setting_def ISABELLE_JDK_HOME}] needs to point to a full JDK (Java
   176   \<^descr>[@{setting_def ISABELLE_JDK_HOME}] points to a full JDK (Java Development
   177   Development Kit) installation with \<^verbatim>\<open>javac\<close> and \<^verbatim>\<open>jar\<close> executables. This is
   177   Kit) installation with \<^verbatim>\<open>javac\<close> and \<^verbatim>\<open>jar\<close> executables. Note that
   178   essential for Isabelle/Scala and other JVM-based tools to work properly.
   178   conventional \<^verbatim>\<open>JAVA_HOME\<close> points to the JRE (Java Runtime Environment), not
   179   Note that conventional \<^verbatim>\<open>JAVA_HOME\<close> usually points to the JRE (Java Runtime
   179   the JDK.
   180   Environment), not JDK.
   180 
       
   181   \<^descr>[@{setting_def ISABELLE_JAVA_PLATFORM}] identifies the hardware and
       
   182   operating system platform for the Java installation of Isabelle. That is
       
   183   usually the (native) 64 bit variant: \<^verbatim>\<open>x86_64-linux\<close>, \<^verbatim>\<open>x86_64-darwin\<close>,
       
   184   \<^verbatim>\<open>x86_64-windows\<close>.
   181 
   185 
   182   \<^descr>[@{setting_def ISABELLE_PATH}] is a list of directories (separated by
   186   \<^descr>[@{setting_def ISABELLE_PATH}] is a list of directories (separated by
   183   colons) where Isabelle logic images may reside. When looking up heaps files,
   187   colons) where Isabelle logic images may reside. When looking up heaps files,
   184   the value of @{setting ML_IDENTIFIER} is appended to each component
   188   the value of @{setting ML_IDENTIFIER} is appended to each component
   185   internally.
   189   internally.