src/HOL/More_List.thy
changeset 45993 3ca49a4bcc9f
parent 45990 b7b905b23b2a
child 46033 6fc579c917b8
--- a/src/HOL/More_List.thy	Tue Dec 27 09:15:26 2011 +0100
+++ b/src/HOL/More_List.thy	Tue Dec 27 09:15:26 2011 +0100
@@ -8,16 +8,6 @@
 
 hide_const (open) Finite_Set.fold
 
-text {* Repairing code generator setup *}
-
-declare (in lattice) Inf_fin_set_fold [code_unfold del]
-declare (in lattice) Sup_fin_set_fold [code_unfold del]
-declare (in linorder) Min_fin_set_fold [code_unfold del]
-declare (in linorder) Max_fin_set_fold [code_unfold del]
-declare (in complete_lattice) Inf_set_fold [code_unfold del]
-declare (in complete_lattice) Sup_set_fold [code_unfold del]
-
-
 text {* Fold combinator with canonical argument order *}
 
 primrec fold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'a list \<Rightarrow> 'b \<Rightarrow> 'b" where
@@ -238,7 +228,7 @@
 proof -
   interpret comp_fun_idem "sup :: 'a \<Rightarrow> 'a \<Rightarrow> 'a"
     by (fact comp_fun_idem_sup)
-  show ?thesis by (simp add: Sup_fold_sup fold_set sup_commute)
+  show ?thesis by (simp add: Sup_fold_sup fold_set_fold sup_commute)
 qed
 
 lemma (in complete_lattice) Sup_set_foldr [code_unfold]: