changeset 58318 | f95754ca7082 |
parent 57492 | 74bf65a1910a |
child 59788 | 6f7b6adac439 |
--- a/src/ZF/Induct/Multiset.thy Thu Sep 11 20:01:29 2014 +0200 +++ b/src/ZF/Induct/Multiset.thy Thu Sep 11 21:11:03 2014 +0200 @@ -61,7 +61,7 @@ "MCollect(M, P) == funrestrict(M, {x \<in> mset_of(M). P(x)})" definition - (* Counts the number of occurences of an element in a multiset *) + (* Counts the number of occurrences of an element in a multiset *) mcount :: "[i, i] => i" where "mcount(M, a) == if a \<in> mset_of(M) then M`a else 0"