diff -r 45eee631ea4f -r ad43b3ab06e4 src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Wed Jan 20 13:16:58 2016 +0100 +++ b/src/HOL/Library/Multiset.thy Wed Jan 20 17:14:53 2016 +0100 @@ -271,12 +271,23 @@ definition subset_mset :: "'a multiset \ 'a multiset \ bool" (infix "\#" 50) where "A \# B = (A \# B \ A \ B)" +abbreviation (input) supseteq_mset :: "'a multiset \ 'a multiset \ bool" where + "supseteq_mset A B == B \# A" + +abbreviation (input) supset_mset :: "'a multiset \ 'a multiset \ bool" where + "supset_mset A B == B \# A" + notation (input) - subseteq_mset (infix "\#" 50) + subseteq_mset (infix "\#" 50) and + supseteq_mset (infix "\#" 50) and + supseteq_mset (infix "\#" 50) and + supset_mset (infix "\#" 50) notation (ASCII) subseteq_mset (infix "<=#" 50) and - subset_mset (infix "<#" 50) + subset_mset (infix "<#" 50) and + supseteq_mset (infix ">=#" 50) and + supset_mset (infix ">#" 50) interpretation subset_mset: ordered_ab_semigroup_add_imp_le "op +" "op -" "op \#" "op \#" by standard (auto simp add: subset_mset_def subseteq_mset_def multiset_eq_iff intro: order_trans antisym)