src/Doc/Classes/Classes.thy
changeset 69660 2bc2a8599369
parent 69597 ff784d5a5bfb
child 76987 4c275405faae
equal deleted inserted replaced
69659:07025152dd80 69660:2bc2a8599369
   586   "example = pow_int 10 (-2)"
   586   "example = pow_int 10 (-2)"
   587 
   587 
   588 text \<open>
   588 text \<open>
   589   \<^noindent> This maps to Haskell as follows:
   589   \<^noindent> This maps to Haskell as follows:
   590 \<close>
   590 \<close>
   591 text %quotetypewriter \<open>
   591 text %quote \<open>
   592   @{code_stmts example (Haskell)}
   592   @{code_stmts example (Haskell)}
   593 \<close>
   593 \<close>
   594 
   594 
   595 text \<open>
   595 text \<open>
   596   \<^noindent> The code in SML has explicit dictionary passing:
   596   \<^noindent> The code in SML has explicit dictionary passing:
   597 \<close>
   597 \<close>
   598 text %quotetypewriter \<open>
   598 text %quote \<open>
   599   @{code_stmts example (SML)}
   599   @{code_stmts example (SML)}
   600 \<close>
   600 \<close>
   601 
   601 
   602 
   602 
   603 text \<open>
   603 text \<open>
   604   \<^noindent> In Scala, implicits are used as dictionaries:
   604   \<^noindent> In Scala, implicits are used as dictionaries:
   605 \<close>
   605 \<close>
   606 text %quotetypewriter \<open>
   606 text %quote \<open>
   607   @{code_stmts example (Scala)}
   607   @{code_stmts example (Scala)}
   608 \<close>
   608 \<close>
   609 
   609 
   610 
   610 
   611 subsection \<open>Inspecting the type class universe\<close>
   611 subsection \<open>Inspecting the type class universe\<close>