src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy
changeset 65919 b6d458915f1b
parent 64850 fc9265882329
child 66014 2f45f4abf0a9
--- a/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy	Wed May 24 16:35:18 2017 +0200
+++ b/src/HOL/Codegenerator_Test/Generate_Efficient_Datastructures.thy	Thu May 25 14:38:41 2017 +0200
@@ -55,20 +55,6 @@
   or implemented for RBT trees.
 *)
 
-export_code _ checking SML OCaml? Haskell?
-
-(* Extra setup to make Scala happy *)
-(* If the compilation fails with an error "ambiguous implicit values",
-   read \<section>7.1 in the Code Generation Manual *)
-
-lemma [code]:
-  "(gfp :: ('a :: complete_linorder \<Rightarrow> 'a) \<Rightarrow> 'a) f = Sup {u. u \<le> f u}"
-unfolding gfp_def by blast
-
-lemma [code]:
-  "(lfp :: ('a :: complete_linorder \<Rightarrow> 'a) \<Rightarrow> 'a) f = Inf {u. f u \<le> u}"
-unfolding lfp_def by blast
-
-export_code _ checking Scala?
+export_code _ checking SML OCaml? Haskell? Scala
 
 end