src/HOL/Library/Multiset.thy
changeset 55811 aa1acc25126b
parent 55808 488c3e8282c8
child 55913 c1409c103b77
--- a/src/HOL/Library/Multiset.thy	Fri Feb 28 22:00:13 2014 +0100
+++ b/src/HOL/Library/Multiset.thy	Fri Feb 28 17:54:52 2014 +0100
@@ -2314,7 +2314,7 @@
 
 lemma card_of_set_of:
 "(card_of {M. set_of M \<subseteq> A}, card_of {as. set as \<subseteq> A}) \<in> ordLeq"
-apply(rule card_of_ordLeqI2[of _ multiset_of]) using multiset_of_surj by auto
+apply(rule surj_imp_ordLeq[of _ multiset_of]) using multiset_of_surj by auto
 
 lemma nat_sum_induct:
 assumes "\<And>n1 n2. (\<And> m1 m2. m1 + m2 < n1 + n2 \<Longrightarrow> phi m1 m2) \<Longrightarrow> phi n1 n2"