src/HOL/Library/Code_Char.thy
author haftmann
Mon, 23 Jul 2012 09:28:03 +0200
changeset 49446 6efff142bb54
parent 43469 85ca44488a29
child 52297 599ff65b85e2
permissions -rw-r--r--
restrict unqualified imports from Haskell Prelude to a small set of fundamental operations
     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 "Prelude.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 :: equal
    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 "HOL.equal \<Colon> char \<Rightarrow> char \<Rightarrow> bool"
    35   (SML "!((_ : char) = _)")
    36   (OCaml "!((_ : char) = _)")
    37   (Haskell infix 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 code_reserved SML String
    48 
    49 code_const implode
    50   (SML "String.implode")
    51   (OCaml "!(let l = _ in let res = String.create (List.length l) in let rec imp i = function | [] -> res | c :: l -> String.set res i c; imp (i + 1) l in imp 0 l)")
    52   (Haskell "_")
    53   (Scala "!(\"\" ++/ _)")
    54 
    55 code_const explode
    56   (SML "String.explode")
    57   (OCaml "!(let s = _ in let rec exp i l = if i < 0 then l else exp (i - 1) (String.get s i :: l) in exp (String.length s - 1) [])")
    58   (Haskell "_")
    59   (Scala "!(_.toList)")
    60 
    61 end