src/Doc/System/Scala.thy
changeset 72103 7b318273a4aa
parent 71907 64c9628b39fc
child 72197 957bf00eff2a
equal deleted inserted replaced
72101:c65614b556b2 72103:7b318273a4aa
   200 
   200 
   201 subsection \<open>Invoking functions in Isabelle/ML\<close>
   201 subsection \<open>Invoking functions in Isabelle/ML\<close>
   202 
   202 
   203 text \<open>
   203 text \<open>
   204   Isabelle/PIDE provides a protocol to invoke registered Scala functions in
   204   Isabelle/PIDE provides a protocol to invoke registered Scala functions in
   205   ML: this requires a proper PIDE session context, e.g.\ within the Prover IDE
   205   ML: this works both within the Prover IDE and in batch builds.
   206   or in batch builds via option @{system_option pide_session}.
       
   207 
   206 
   208   The subsequent ML antiquotations refer to Scala functions in a
   207   The subsequent ML antiquotations refer to Scala functions in a
   209   formally-checked manner.
   208   formally-checked manner.
   210 
   209 
   211   \begin{matharray}{rcl}
   210   \begin{matharray}{rcl}