# HG changeset patch # User haftmann # Date 1481984520 -3600 # Node ID 2155c0c1ecb6f785acf989e26ae311e18b34f264 # Parent 142ac30b68fe72894067ba3a6e3fd0941ef9119b renewed and spread FIXME tags on watering bin interpretation, which got partially lost in 9f089287687b diff -r 142ac30b68fe -r 2155c0c1ecb6 src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Sat Dec 17 15:22:00 2016 +0100 +++ b/src/HOL/Library/Multiset.thy Sat Dec 17 15:22:00 2016 +0100 @@ -526,9 +526,11 @@ 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) + \ \FIXME: avoid junk stemming from type class interpretation\ interpretation subset_mset: ordered_ab_semigroup_monoid_add_imp_le "op +" 0 "op -" "op \#" "op <#" by standard + \ \FIXME: avoid junk stemming from type class interpretation\ lemma mset_subset_eqI: "(\a. count A a \ count B a) \ A \# B" @@ -547,6 +549,7 @@ interpretation subset_mset: ordered_cancel_comm_monoid_diff "op +" 0 "op \#" "op <#" "op -" by standard (simp, fact mset_subset_eq_exists_conv) + \ \FIXME: avoid junk stemming from type class interpretation\ declare subset_mset.add_diff_assoc[simp] subset_mset.add_diff_assoc2[simp] @@ -684,8 +687,7 @@ by arith show "class.semilattice_inf op \# op \# op \#" by standard (auto simp add: multiset_inter_def subseteq_mset_def) -qed - \ \FIXME: avoid junk stemming from type class interpretation\ +qed \ \FIXME: avoid junk stemming from type class interpretation\ definition sup_subset_mset :: "'a multiset \ 'a multiset \ 'a multiset"(infixl "\#" 70) where "sup_subset_mset A B = A + (B - A)" \ \FIXME irregular fact name\ @@ -696,12 +698,12 @@ by arith show "class.semilattice_sup op \# op \# op \#" by standard (auto simp add: sup_subset_mset_def subseteq_mset_def) -qed - \ \FIXME: avoid junk stemming from type class interpretation\ +qed \ \FIXME: avoid junk stemming from type class interpretation\ interpretation subset_mset: bounded_lattice_bot "op \#" "op \#" "op \#" "op \#" "{#}" by standard auto + \ \FIXME: avoid junk stemming from type class interpretation\ subsubsection \Additional intersection facts\ @@ -1161,7 +1163,7 @@ by (intro cSup_least) (auto intro: mset_subset_eq_count ge) finally show "count (Sup A) x \ count X x" . qed -qed +qed \ \FIXME: avoid junk stemming from type class interpretation\ lemma set_mset_Inf: assumes "A \ {}" @@ -1239,7 +1241,7 @@ fix A B C :: "'a multiset" show "A \# (B \# C) = A \# B \# (A \# C)" by (intro multiset_eqI) simp_all -qed +qed \ \FIXME: avoid junk stemming from type class interpretation\ subsubsection \Filter (with comprehension syntax)\