equal
deleted
inserted
replaced
293 typically contains the keywords of the target language. It can be |
293 typically contains the keywords of the target language. It can be |
294 extended manually, thus avoiding accidental overwrites, using the |
294 extended manually, thus avoiding accidental overwrites, using the |
295 @{command_def "code_reserved"} command: |
295 @{command_def "code_reserved"} command: |
296 \<close> |
296 \<close> |
297 |
297 |
298 code_reserved %quote "\<SMLdummy>" bool true false andalso |
298 code_reserved %quotett ("\<SMLdummy>") bool true false andalso |
299 |
299 |
300 text \<open> |
300 text \<open> |
301 \noindent Next, we try to map HOL pairs to SML pairs, using the |
301 \noindent Next, we try to map HOL pairs to SML pairs, using the |
302 infix ``\<^verbatim>\<open>*\<close>'' type constructor and parentheses: |
302 infix ``\<^verbatim>\<open>*\<close>'' type constructor and parentheses: |
303 \<close> |
303 \<close> |
386 code_printing %quotett code_module "Errno" \<rightharpoonup> (Haskell) |
386 code_printing %quotett code_module "Errno" \<rightharpoonup> (Haskell) |
387 \<open>module Errno(errno) where |
387 \<open>module Errno(errno) where |
388 |
388 |
389 errno i = error ("Error number: " ++ show i)\<close> |
389 errno i = error ("Error number: " ++ show i)\<close> |
390 |
390 |
391 code_reserved %quotett Haskell Errno |
391 code_reserved %quotett (Haskell) Errno |
392 |
392 |
393 text \<open> |
393 text \<open> |
394 \noindent Such named modules are then prepended to every |
394 \noindent Such named modules are then prepended to every |
395 generated code. Inspect such code in order to find out how |
395 generated code. Inspect such code in order to find out how |
396 this behaves with respect to a particular |
396 this behaves with respect to a particular |