src/HOL/Finite_Set.thy
changeset 56154 f0a927235162
parent 55096 916b2ac758f4
child 56166 9a241bc276cd
--- 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 \<times> B) = fst ` f ` {i::nat. i < n}" by simp
   with `B \<noteq> {}` have "A = (fst \<circ> f) ` {i::nat. i < n}"
-    by (simp add: image_compose)
+    by (simp add: image_comp)
   then have "\<exists>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 \<times> B) = snd ` f ` {i::nat. i < n}" by simp
   with `A \<noteq> {}` have "B = (snd \<circ> f) ` {i::nat. i < n}"
-    by (simp add: image_compose)
+    by (simp add: image_comp)
   then have "\<exists>n f. B = f ` {i::nat. i < n}" by blast
   then show ?thesis
     by (auto simp add: finite_conv_nat_seg_image)