diff -r 2008f1cf3030 -r f0a927235162 src/HOL/Finite_Set.thy --- a/src/HOL/Finite_Set.thy Sat Mar 15 03:37:22 2014 +0100 +++ b/src/HOL/Finite_Set.thy Sat Mar 15 08:31:33 2014 +0100 @@ -395,7 +395,7 @@ by (auto simp add: finite_conv_nat_seg_image) then have "fst ` (A \ B) = fst ` f ` {i::nat. i < n}" by simp with `B \ {}` have "A = (fst \ f) ` {i::nat. i < n}" - by (simp add: image_compose) + by (simp add: image_comp) then have "\n f. A = f ` {i::nat. i < n}" by blast then show ?thesis by (auto simp add: finite_conv_nat_seg_image) @@ -409,7 +409,7 @@ by (auto simp add: finite_conv_nat_seg_image) then have "snd ` (A \ B) = snd ` f ` {i::nat. i < n}" by simp with `A \ {}` have "B = (snd \ f) ` {i::nat. i < n}" - by (simp add: image_compose) + by (simp add: image_comp) then have "\n f. B = f ` {i::nat. i < n}" by blast then show ?thesis by (auto simp add: finite_conv_nat_seg_image)