src/HOL/Library/Code_Char.thy
author haftmann
Tue, 01 Jun 2010 10:30:53 +0200
changeset 37221 4d984bc33c66
parent 33226 a5eba0447559
child 37434 7a3610dca96b
permissions -rw-r--r--
added Scala code setup
     1 (*  Title:      HOL/Library/Code_Char.thy
     2     Author:     Florian Haftmann
     3 *)
     4 
     5 header {* Code generation of pretty characters (and strings) *}
     6 
     7 theory Code_Char
     8 imports List Code_Evaluation Main
     9 begin
    10 
    11 code_type char
    12   (SML "char")
    13   (OCaml "char")
    14   (Haskell "Char")
    15   (Scala "Char")
    16 
    17 setup {*
    18   fold String_Code.add_literal_char ["SML", "OCaml", "Haskell", "Scala"] 
    19   #> String_Code.add_literal_list_string "Haskell"
    20 *}
    21 
    22 code_instance char :: eq
    23   (Haskell -)
    24 
    25 code_reserved SML
    26   char
    27 
    28 code_reserved OCaml
    29   char
    30 
    31 code_reserved Scala
    32   char
    33 
    34 code_const "eq_class.eq \<Colon> char \<Rightarrow> char \<Rightarrow> bool"
    35   (SML "!((_ : char) = _)")
    36   (OCaml "!((_ : char) = _)")
    37   (Haskell infixl 4 "==")
    38   (Scala infixl 5 "==")
    39 
    40 code_const "Code_Evaluation.term_of \<Colon> char \<Rightarrow> term"
    41   (Eval "HOLogic.mk'_char/ (IntInf.fromInt/ (Char.ord/ _))")
    42 
    43 
    44 definition implode :: "string \<Rightarrow> String.literal" where
    45   "implode = STR"
    46 
    47 primrec explode :: "String.literal \<Rightarrow> string" where
    48   "explode (STR s) = s"
    49 
    50 lemma [code]:
    51   "literal_case f s = f (explode s)"
    52   "literal_rec f s = f (explode s)"
    53   by (cases s, simp)+
    54 
    55 code_reserved SML String
    56 
    57 code_const implode
    58   (SML "String.implode")
    59   (OCaml "failwith/ \"implode\"")
    60   (Haskell "_")
    61   (Scala "List.toString((_))")
    62 
    63 code_const explode
    64   (SML "String.explode")
    65   (OCaml "failwith/ \"explode\"")
    66   (Haskell "_")
    67   (Scala "List.fromString((_))")
    68 
    69 end