src/Doc/System/Scala.thy
changeset 79724 54d0f6edfe3a
parent 79059 ae682b2aab03
equal deleted inserted replaced
79723:aa77ebb2dc16 79724:54d0f6edfe3a
   130   ensures that all provided modules are compiled and packaged (as jars). It is
   130   ensures that all provided modules are compiled and packaged (as jars). It is
   131   also possible to invoke @{tool scala_build} explicitly, with extra options.
   131   also possible to invoke @{tool scala_build} explicitly, with extra options.
   132 
   132 
   133   \<^medskip>
   133   \<^medskip>
   134   The syntax of \<^path>\<open>etc/build.props\<close> follows a regular Java properties
   134   The syntax of \<^path>\<open>etc/build.props\<close> follows a regular Java properties
   135   file\<^footnote>\<open>\<^url>\<open>https://docs.oracle.com/en/java/javase/17/docs/api/java.base/java/util/Properties.html#load(java.io.Reader)\<close>\<close>,
   135   file\<^footnote>\<open>\<^url>\<open>https://docs.oracle.com/en/java/javase/21/docs/api/java.base/java/util/Properties.html#load(java.io.Reader)\<close>\<close>,
   136   but the encoding is \<^verbatim>\<open>UTF-8\<close>, instead of historic \<^verbatim>\<open>ISO 8859-1\<close> from the API
   136   but the encoding is \<^verbatim>\<open>UTF-8\<close>, instead of historic \<^verbatim>\<open>ISO 8859-1\<close> from the API
   137   documentation.
   137   documentation.
   138 
   138 
   139   The subsequent properties are relevant for the Scala/Java build process.
   139   The subsequent properties are relevant for the Scala/Java build process.
   140   Most properties are optional: the default is an empty string (or list). File
   140   Most properties are optional: the default is an empty string (or list). File