src/Doc/Codegen/Computations.thy
changeset 76659 2afbd514b654
parent 74584 c14787d73db6
child 76987 4c275405faae
equal deleted inserted replaced
76658:e60fd6257abe 76659:2afbd514b654
   239 
   239 
   240   
   240   
   241 subsection \<open>Pitfalls concerning input terms\<close>
   241 subsection \<open>Pitfalls concerning input terms\<close>
   242 
   242 
   243 text \<open>
   243 text \<open>
   244     \<^descr> \<open>No polymorphims.\<close> Input terms must be monomorphic: compilation
   244     \<^descr> \<open>No polymorphism.\<close> Input terms must be monomorphic: compilation
   245       to ML requires dedicated choice of monomorphic types.
   245       to ML requires dedicated choice of monomorphic types.
   246 
   246 
   247     \<^descr> \<open>No abstractions.\<close> Only constants and applications are admissible
   247     \<^descr> \<open>No abstractions.\<close> Only constants and applications are admissible
   248       as input; abstractions are not possible.  In theory, the
   248       as input; abstractions are not possible.  In theory, the
   249       compilation schema could be extended to cover abstractions also,
   249       compilation schema could be extended to cover abstractions also,