src/HOL/Library/Multiset.thy
changeset 60400 a8a31b9ebff5
parent 60397 f8a513fedb31
child 60495 d7ff0a1df90a
child 60500 903bb1495239
--- a/src/HOL/Library/Multiset.thy	Wed Jun 10 13:44:46 2015 +0200
+++ b/src/HOL/Library/Multiset.thy	Wed Jun 10 15:50:17 2015 +0200
@@ -281,10 +281,10 @@
 subsubsection {* Pointwise ordering induced by count *}
 
 definition subseteq_mset :: "'a multiset \<Rightarrow> 'a multiset \<Rightarrow> bool" (infix "<=#" 50) where
-"subseteq_mset A B \<equiv> (\<forall>a. count A a \<le> count B a)"
+"subseteq_mset A B = (\<forall>a. count A a \<le> count B a)"
 
 definition subset_mset :: "'a multiset \<Rightarrow> 'a multiset \<Rightarrow> bool" (infix "<#" 50) where
-"subset_mset A B \<equiv> (A <=# B \<and> A \<noteq> B)"
+"subset_mset A B = (A <=# B \<and> A \<noteq> B)"
 
 notation subseteq_mset (infix "\<le>#" 50)
 notation (xsymbols) subseteq_mset (infix "\<subseteq>#" 50)