# HG changeset patch # User nipkow # Date 1591177461 -7200 # Node ID 4c5778d8a53df6e81dfe4198c0aba4101072c904 # Parent 435cdc77211019bbf5915aac7bf44c7916e0cc8e should have been copied across from Set.thy as well for better printing diff -r 435cdc772110 -r 4c5778d8a53d src/HOL/Library/Multiset.thy --- a/src/HOL/Library/Multiset.thy Sat May 30 11:48:35 2020 +0000 +++ b/src/HOL/Library/Multiset.thy Wed Jun 03 11:44:21 2020 +0200 @@ -189,6 +189,11 @@ "\x\#A. P" \ "CONST Multiset.Ball A (\x. P)" "\x\#A. P" \ "CONST Multiset.Bex A (\x. P)" +print_translation \ + [Syntax_Trans.preserve_binder_abs2_tr' \<^const_syntax>\Multiset.Ball\ \<^syntax_const>\_MBall\, + Syntax_Trans.preserve_binder_abs2_tr' \<^const_syntax>\Multiset.Bex\ \<^syntax_const>\_MBex\] +\ \ \to avoid eta-contraction of body\ + lemma count_eq_zero_iff: "count M x = 0 \ x \# M" by (auto simp add: set_mset_def)