| changeset 25534 | d0b74fdd6067 |
| parent 24844 | 98c006a30218 |
| child 25860 | 844ab7ace3db |
--- a/src/HOL/Code_Setup.thy Wed Dec 05 14:15:39 2007 +0100 +++ b/src/HOL/Code_Setup.thy Wed Dec 05 14:15:45 2007 +0100 @@ -91,12 +91,6 @@ (OCaml "bool") (Haskell "Bool") -code_instance bool :: eq - (Haskell -) - -code_const "op = \<Colon> bool \<Rightarrow> bool \<Rightarrow> bool" - (Haskell infixl 4 "==") - code_const True and False and Not and "op &" and "op |" and If (SML "true" and "false" and "not" and infixl 1 "andalso" and infixl 0 "orelse"