src/Doc/System/Scala.thy
changeset 72759 bd5ee3148132
parent 72332 319dd5c618a5
child 73419 22f3f2117ed7
equal deleted inserted replaced
72758:9d0951e24e61 72759:bd5ee3148132
   241 
   241 
   242 
   242 
   243 subsubsection \<open>Examples\<close>
   243 subsubsection \<open>Examples\<close>
   244 
   244 
   245 text \<open>
   245 text \<open>
   246   Invoke a predefined Scala function that is the identity on type
   246   Invoke the predefined Scala function \<^scala_function>\<open>echo\<close>:
   247   \<^ML_type>\<open>string\<close>:
       
   248 \<close>
   247 \<close>
   249 
   248 
   250 ML \<open>
   249 ML \<open>
   251   val s = "test";
   250   val s = "test";
   252   val s' = \<^scala>\<open>echo\<close> s;
   251   val s' = \<^scala>\<open>echo\<close> s;