diff -r 067210a08a22 -r b0f89998c2a1 src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Wed Apr 12 09:27:43 2017 +0200 +++ b/src/HOL/Library/Multiset.thy Wed Apr 12 09:27:47 2017 +0200 @@ -503,10 +503,10 @@ subsubsection \Pointwise ordering induced by count\ definition subseteq_mset :: "'a multiset \ 'a multiset \ bool" (infix "\#" 50) - where "A \# B = (\a. count A a \ count B a)" + where "A \# B \ (\a. count A a \ count B a)" definition subset_mset :: "'a multiset \ 'a multiset \ bool" (infix "\#" 50) - where "A \# B = (A \# B \ A \ B)" + where "A \# B \ A \# B \ A \ B" abbreviation (input) supseteq_mset :: "'a multiset \ 'a multiset \ bool" (infix "\#" 50) where "supseteq_mset A B \ B \# A"