src/Doc/System/Scala.thy
changeset 53576 793a429c63e7
parent 52116 abf9fcfa65cf
child 53982 f0ee92285221
--- a/src/Doc/System/Scala.thy	Wed Sep 11 23:32:47 2013 +0200
+++ b/src/Doc/System/Scala.thy	Thu Sep 12 13:23:54 2013 +0200
@@ -61,10 +61,10 @@
 
   This allows to compile further Scala modules, depending on existing
   Isabelle/Scala functionality.  The resulting class or jar files can
-  be added to the @{setting CLASSPATH} via the @{verbatim classpath}
-  Bash function that is provided by the Isabelle process environment.
-  Thus add-on components can register themselves in a modular manner,
-  see also \secref{sec:components}.
+  be added to the Java classpath the @{verbatim classpath} Bash
+  function that is provided by the Isabelle process environment.  Thus
+  add-on components can register themselves in a modular manner, see
+  also \secref{sec:components}.
 
   Note that jEdit (\secref{sec:tool-jedit}) has its own mechanisms for
   adding plugin components, which needs special attention since