src/Doc/System/Scala.thy
changeset 74057 22ad3ac2152c
parent 74053 54a11c37d5bc
child 74071 b25b7c264a93
equal deleted inserted replaced
74056:fb8d5c0133c9 74057:22ad3ac2152c
   163 
   163 
   164     \<^item> \<^verbatim>\<open>title\<close> (required) is a human-readable description of the module, used
   164     \<^item> \<^verbatim>\<open>title\<close> (required) is a human-readable description of the module, used
   165     in printed messages.
   165     in printed messages.
   166 
   166 
   167     \<^item> \<^verbatim>\<open>module\<close> specifies a \<^verbatim>\<open>jar\<close> file name for the output module, as result
   167     \<^item> \<^verbatim>\<open>module\<close> specifies a \<^verbatim>\<open>jar\<close> file name for the output module, as result
   168     of compiling the specified sources (and resources). If this is absent,
   168     of the specified sources (and resources). If this is absent (or
   169     there is no build process, but contributing sources may still be given,
   169     \<^verbatim>\<open>no_build\<close> is set, as described below), there is no implicit build
   170     possibly together with \<^verbatim>\<open>no_module\<close> as described below.
   170     process. The contributing sources might be given nonetheless, notably for
   171 
   171     @{tool scala_project} (\secref{sec:tool-scala-project}), which includes
   172     \<^item> \<^verbatim>\<open>no_module\<close> means that there is no build process, but the specified
   172     Scala/Java sources of components, while suppressing \<^verbatim>\<open>jar\<close> modules (to
   173     \<^verbatim>\<open>jar\<close> is provided by other means. This is relevant for @{tool
   173     avoid duplication of program content).
   174     scala_project} (\secref{sec:tool-scala-project}), which includes all
   174 
   175     Scala/Java sources of components, but suppresses \<^verbatim>\<open>jar\<close> modules to avoid
   175     \<^item> \<^verbatim>\<open>no_build\<close> is a Boolean property, with default \<^verbatim>\<open>false\<close>. If set to
   176     duplication of content.
   176     \<^verbatim>\<open>true\<close>, the implicit build process for the given \<^verbatim>\<open>module\<close> is \<^emph>\<open>omitted\<close>
       
   177     --- it is assumed to be provided by other means.
   177 
   178 
   178     \<^item> \<^verbatim>\<open>scalac_options\<close> and \<^verbatim>\<open>javac_options\<close> augment the default settings
   179     \<^item> \<^verbatim>\<open>scalac_options\<close> and \<^verbatim>\<open>javac_options\<close> augment the default settings
   179     @{setting_ref ISABELLE_SCALAC_OPTIONS} and @{setting_ref
   180     @{setting_ref ISABELLE_SCALAC_OPTIONS} and @{setting_ref
   180     ISABELLE_JAVAC_OPTIONS} for this component; option syntax follows the
   181     ISABELLE_JAVAC_OPTIONS} for this component; option syntax follows the
   181     regular command-line tools \<^verbatim>\<open>scalac\<close> and \<^verbatim>\<open>javac\<close>, respectively.
   182     regular command-line tools \<^verbatim>\<open>scalac\<close> and \<^verbatim>\<open>javac\<close>, respectively.