src/Doc/System/Basics.thy
changeset 51434 e19a22974c72
parent 51057 a22b134f862e
child 51932 f196352201d6
equal deleted inserted replaced
51429:48eb29821bd9 51434:e19a22974c72
   218   command line.  The optional @{setting ML_PLATFORM} may specify the
   218   command line.  The optional @{setting ML_PLATFORM} may specify the
   219   binary format of ML heap images, which is useful for cross-platform
   219   binary format of ML heap images, which is useful for cross-platform
   220   installations.  The value of @{setting ML_IDENTIFIER} is
   220   installations.  The value of @{setting ML_IDENTIFIER} is
   221   automatically obtained by composing the values of @{setting
   221   automatically obtained by composing the values of @{setting
   222   ML_SYSTEM}, @{setting ML_PLATFORM} and the Isabelle version values.
   222   ML_SYSTEM}, @{setting ML_PLATFORM} and the Isabelle version values.
       
   223 
       
   224   \item[@{setting_def ISABELLE_POLYML}@{text "\<^sup>*"}] is @{verbatim true}
       
   225   for @{setting ML_SYSTEM} values derived from Poly/ML, as opposed to
       
   226   SML/NJ where it is empty.  This is particularly useful with the
       
   227   build option @{system_option condition}
       
   228   (\secref{sec:system-options}) to restrict big sessions to something
       
   229   that SML/NJ can still handle.
   223 
   230 
   224   \item[@{setting_def ISABELLE_JDK_HOME}] needs to point to a full JDK
   231   \item[@{setting_def ISABELLE_JDK_HOME}] needs to point to a full JDK
   225   (Java Development Kit) installation with @{verbatim javac} and
   232   (Java Development Kit) installation with @{verbatim javac} and
   226   @{verbatim jar} executables.  This is essential for Isabelle/Scala
   233   @{verbatim jar} executables.  This is essential for Isabelle/Scala
   227   and other JVM-based tools to work properly.  Note that conventional
   234   and other JVM-based tools to work properly.  Note that conventional