src/Doc/System/Scala.thy
changeset 79059 ae682b2aab03
parent 79058 f13390b2c1ee
child 79724 54d0f6edfe3a
--- a/src/Doc/System/Scala.thy	Sat Nov 25 16:13:08 2023 +0100
+++ b/src/Doc/System/Scala.thy	Sat Nov 25 16:49:48 2023 +0100
@@ -96,27 +96,6 @@
 \<close>
 
 
-subsection \<open>Scala script wrapper\<close>
-
-text \<open>
-  The executable @{executable "$ISABELLE_HOME/bin/isabelle_scala_script"}
-  allows to run Isabelle/Scala source files stand-alone programs, by using a
-  suitable ``hash-bang'' line and executable file permissions. For example:
-  @{verbatim [display, indent = 2] \<open>#!/usr/bin/env isabelle_scala_script\<close>}
-  @{scala [display, indent = 2]
-\<open>val options = isabelle.Options.init()
-Console.println("browser_info = " + options.bool("browser_info"))
-Console.println("document = " + options.string("document"))\<close>}
-
-  This assumes that the executable may be found via the @{setting PATH} from
-  the process environment: this is the case when Isabelle settings are active,
-  e.g.\ in the context of the main Isabelle tool wrapper
-  \secref{sec:isabelle-tool}. Alternatively, the full
-  \<^file>\<open>$ISABELLE_HOME/bin/isabelle_scala_script\<close> may be specified in expanded
-  form.
-\<close>
-
-
 subsection \<open>Scala compiler \label{sec:tool-scalac}\<close>
 
 text \<open>