src/HOL/Library/Multiset.thy
changeset 35273 51692ec1b220
parent 35268 04673275441a
child 35308 359e0fd38a92
--- a/src/HOL/Library/Multiset.thy	Mon Feb 22 09:15:10 2010 +0100
+++ b/src/HOL/Library/Multiset.thy	Mon Feb 22 09:15:11 2010 +0100
@@ -1206,11 +1206,14 @@
 
 subsubsection {* Partial-order properties *}
 
-definition less_multiset :: "'a\<Colon>order multiset \<Rightarrow> 'a multiset \<Rightarrow> bool" (infix "\<subset>#" 50) where
-  "M' \<subset># M \<longleftrightarrow> (M', M) \<in> mult {(x', x). x' < x}"
+definition less_multiset :: "'a\<Colon>order multiset \<Rightarrow> 'a multiset \<Rightarrow> bool" (infix "<#" 50) where
+  "M' <# M \<longleftrightarrow> (M', M) \<in> mult {(x', x). x' < x}"
 
-definition le_multiset :: "'a\<Colon>order multiset \<Rightarrow> 'a multiset \<Rightarrow> bool" (infix "\<subseteq>#" 50) where
-  "M' \<subseteq># M \<longleftrightarrow> M' \<subset># M \<or> M' = M"
+definition le_multiset :: "'a\<Colon>order multiset \<Rightarrow> 'a multiset \<Rightarrow> bool" (infix "<=#" 50) where
+  "M' <=# M \<longleftrightarrow> M' <# M \<or> M' = M"
+
+notation (xsymbol) less_multiset (infix "\<subset>#" 50)
+notation (xsymbol) le_multiset (infix "\<subseteq>#" 50)
 
 interpretation multiset_order: order le_multiset less_multiset
 proof -