src/Doc/System/Scala.thy
changeset 74656 0659536b150b
parent 74071 b25b7c264a93
child 74661 591303cc04c2
equal deleted inserted replaced
74655:cd674ebf6cac 74656:0659536b150b
   276   Options are:
   276   Options are:
   277     -D DIR       project directory (default: "$ISABELLE_HOME_USER/scala_project")
   277     -D DIR       project directory (default: "$ISABELLE_HOME_USER/scala_project")
   278     -L           make symlinks to original source files
   278     -L           make symlinks to original source files
   279     -f           force update of existing directory
   279     -f           force update of existing directory
   280 
   280 
   281   Setup Gradle project for Isabelle/Scala/jEdit --- to support Scala IDEs
   281   Setup Maven project for Isabelle/Scala/jEdit --- to support common IDEs
   282   such as IntelliJ IDEA.\<close>}
   282   such as IntelliJ IDEA.\<close>}
   283 
   283 
   284   The generated configuration is for Gradle\<^footnote>\<open>\<^url>\<open>https://gradle.org\<close>\<close>, but the
   284   The generated configuration is for Maven\<^footnote>\<open>\<^url>\<open>https://maven.apache.org\<close>\<close>, but
   285   main purpose is to import it into common Scala IDEs, such as IntelliJ
   285   the main purpose is to import it into common IDEs, such as IntelliJ
   286   IDEA\<^footnote>\<open>\<^url>\<open>https://www.jetbrains.com/idea\<close>\<close>. This allows to explore the
   286   IDEA\<^footnote>\<open>\<^url>\<open>https://www.jetbrains.com/idea\<close>\<close>. This allows to explore the
   287   sources with static analysis and other hints in real-time.
   287   sources with static analysis and other hints in real-time.
   288 
   288 
   289   The generated files refer to physical file-system locations, using the path
   289   The generated files refer to physical file-system locations, using the path
   290   notation of the underlying OS platform. Thus the project needs to be
   290   notation of the underlying OS platform. Thus the project needs to be