equal
deleted
inserted
replaced
181 |
181 |
182 setup {* |
182 setup {* |
183 fold String_Code.add_literal_string ["SML", "OCaml", "Haskell", "Scala"] |
183 fold String_Code.add_literal_string ["SML", "OCaml", "Haskell", "Scala"] |
184 *} |
184 *} |
185 |
185 |
186 code_instance literal :: eq |
186 code_instance literal :: equal |
187 (Haskell -) |
187 (Haskell -) |
188 |
188 |
189 code_const "eq_class.eq \<Colon> literal \<Rightarrow> literal \<Rightarrow> bool" |
189 code_const "HOL.equal \<Colon> literal \<Rightarrow> literal \<Rightarrow> bool" |
190 (SML "!((_ : string) = _)") |
190 (SML "!((_ : string) = _)") |
191 (OCaml "!((_ : string) = _)") |
191 (OCaml "!((_ : string) = _)") |
192 (Haskell infixl 4 "==") |
192 (Haskell infixl 4 "==") |
193 (Scala infixl 5 "==") |
193 (Scala infixl 5 "==") |
194 |
194 |