src/HOL/Library/RBT_Set.thy
changeset 54263 c4159fe6fa46
parent 53955 436649a2ed62
child 55565 f663fc1e653b
--- a/src/HOL/Library/RBT_Set.thy	Tue Nov 05 09:45:00 2013 +0100
+++ b/src/HOL/Library/RBT_Set.thy	Tue Nov 05 09:45:02 2013 +0100
@@ -756,7 +756,8 @@
 declare Inf_Set_fold[folded Inf'_def, code]
 
 lemma INFI_Set_fold [code]:
-  "INFI (Set t) f = fold_keys (inf \<circ> f) t top"
+  fixes f :: "_ \<Rightarrow> 'a::complete_lattice"
+  shows "INFI (Set t) f = fold_keys (inf \<circ> f) t top"
 proof -
   have "comp_fun_commute ((inf :: 'a \<Rightarrow> 'a \<Rightarrow> 'a) \<circ> f)" 
     by default (auto simp add: fun_eq_iff ac_simps)
@@ -796,7 +797,8 @@
 declare Sup_Set_fold[folded Sup'_def, code]
 
 lemma SUPR_Set_fold [code]:
-  "SUPR (Set t) f = fold_keys (sup \<circ> f) t bot"
+  fixes f :: "_ \<Rightarrow> 'a::complete_lattice"
+  shows "SUPR (Set t) f = fold_keys (sup \<circ> f) t bot"
 proof -
   have "comp_fun_commute ((sup :: 'a \<Rightarrow> 'a \<Rightarrow> 'a) \<circ> f)" 
     by default (auto simp add: fun_eq_iff ac_simps)