doc-src/System/Thy/Scala.thy
changeset 48815 eed6698b2ba0
parent 48602 342ca8f3197b
equal deleted inserted replaced
48814:d488a5f25bf6 48815:eed6698b2ba0
    44 
    44 
    45   This allows to interact with Isabelle/Scala in TTY mode like this:
    45   This allows to interact with Isabelle/Scala in TTY mode like this:
    46 \begin{alltt}
    46 \begin{alltt}
    47   isabelle scala
    47   isabelle scala
    48   scala> isabelle.Isabelle_System.getenv("ISABELLE_HOME")
    48   scala> isabelle.Isabelle_System.getenv("ISABELLE_HOME")
    49   scala> isabelle.Isabelle_System.find_logics()
    49   scala> val options = isabelle.Options.init()
       
    50   scala> options.bool("browser_info")
    50 \end{alltt}
    51 \end{alltt}
    51 *}
    52 *}
    52 
    53 
    53 
    54 
    54 section {* Scala compiler \label{sec:tool-scalac} *}
    55 section {* Scala compiler \label{sec:tool-scalac} *}