src/HOL/Code_Setup.thy
changeset 25534 d0b74fdd6067
parent 24844 98c006a30218
child 25860 844ab7ace3db
equal deleted inserted replaced
25533:0140cc7b26ad 25534:d0b74fdd6067
    89 code_type bool
    89 code_type bool
    90   (SML "bool")
    90   (SML "bool")
    91   (OCaml "bool")
    91   (OCaml "bool")
    92   (Haskell "Bool")
    92   (Haskell "Bool")
    93 
    93 
    94 code_instance bool :: eq
       
    95   (Haskell -)
       
    96 
       
    97 code_const "op = \<Colon> bool \<Rightarrow> bool \<Rightarrow> bool"
       
    98   (Haskell infixl 4 "==")
       
    99 
       
   100 code_const True and False and Not and "op &" and "op |" and If
    94 code_const True and False and Not and "op &" and "op |" and If
   101   (SML "true" and "false" and "not"
    95   (SML "true" and "false" and "not"
   102     and infixl 1 "andalso" and infixl 0 "orelse"
    96     and infixl 1 "andalso" and infixl 0 "orelse"
   103     and "!(if (_)/ then (_)/ else (_))")
    97     and "!(if (_)/ then (_)/ else (_))")
   104   (OCaml "true" and "false" and "not"
    98   (OCaml "true" and "false" and "not"