equal
deleted
inserted
replaced
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, |