diff -r 57861bd0a3e1 -r 21995f5e8126 src/Doc/System/Scala.thy --- a/src/Doc/System/Scala.thy Thu Jan 16 16:15:25 2020 +0100 +++ b/src/Doc/System/Scala.thy Thu Jan 16 16:35:17 2020 +0100 @@ -97,8 +97,8 @@ section \Project setup for common Scala IDEs\ text \ - The @{tool_def scala_project} tool creates a Gradle project configuration - for Isabelle/Scala/jEdit: + The @{tool_def scala_project} tool creates a project configuration for + Isabelle/Scala/jEdit: @{verbatim [display] \Usage: isabelle scala_project [OPTIONS] PROJECT_DIR @@ -108,23 +108,23 @@ Setup Gradle project for Isabelle/Scala/jEdit --- to support Scala IDEs such as IntelliJ IDEA.\} - The generated project configuration is for Gradle\<^footnote>\\<^url>\https://gradle.org\\, - but the main purpose is to import it into common Scala IDEs, such as - IntelliJ IDEA\<^footnote>\\<^url>\https://www.jetbrains.com/idea\\. This allows to explore - the sources with static analysis and other hints in real-time. + The generated configuration is for Gradle\<^footnote>\\<^url>\https://gradle.org\\, but the + main purpose is to import it into common Scala IDEs, such as IntelliJ + IDEA\<^footnote>\\<^url>\https://www.jetbrains.com/idea\\. This allows to explore the + sources with static analysis and other hints in real-time. The specified project directory must not exist yet. The generated files - refer to physical file locations, using the path notation of the underlying - OS platform. Thus the project needs to be recreated whenever the Isabelle - installation is changed or moved. + refer to physical file-system locations, using the path notation of the + underlying OS platform. Thus the project needs to be recreated whenever the + Isabelle installation is changed or moved. \<^medskip> By default, Scala sources are \<^emph>\copied\ from the Isabelle distribution and editing them within the IDE has no permanent effect. - Alternatively, option \<^verbatim>\-l\ may be used to produce symlinks to the original - files: this allows to develop Isabelle/Scala/jEdit within an external Scala - IDE. Note that building the result always requires \<^verbatim>\isabelle jedit -b\ on - the command-line. + Option \<^verbatim>\-l\ produces \<^emph>\symlinks\ to the original files: this allows to + develop Isabelle/Scala/jEdit within an external Scala IDE. Note that + building the result always requires \<^verbatim>\isabelle jedit -b\ on the + command-line. \ end