src/HOL/Library/Multiset.thy
changeset 63290 9ac558ab0906
parent 63195 f3f08c0d4aaf
child 63310 caaacf37943f
--- a/src/HOL/Library/Multiset.thy	Sat Jun 11 17:40:52 2016 +0200
+++ b/src/HOL/Library/Multiset.thy	Sat Jun 11 16:22:42 2016 +0200
@@ -1562,16 +1562,13 @@
 
 subsection \<open>Big operators\<close>
 
-no_notation times (infixl "*" 70)
-no_notation Groups.one ("1")
-
 locale comm_monoid_mset = comm_monoid
 begin
 
 definition F :: "'a multiset \<Rightarrow> 'a"
-  where eq_fold: "F M = fold_mset f 1 M"
-
-lemma empty [simp]: "F {#} = 1"
+  where eq_fold: "F M = fold_mset f \<^bold>1 M"
+
+lemma empty [simp]: "F {#} = \<^bold>1"
   by (simp add: eq_fold)
 
 lemma singleton [simp]: "F {#x#} = x"
@@ -1581,7 +1578,7 @@
   show ?thesis by (simp add: eq_fold)
 qed
 
-lemma union [simp]: "F (M + N) = F M * F N"
+lemma union [simp]: "F (M + N) = F M \<^bold>* F N"
 proof -
   interpret comp_fun_commute f
     by standard (simp add: fun_eq_iff left_commute)
@@ -1599,9 +1596,6 @@
 lemma in_mset_fold_plus_iff[iff]: "x \<in># fold_mset (op +) M NN \<longleftrightarrow> x \<in># M \<or> (\<exists>N. N \<in># NN \<and> x \<in># N)"
   by (induct NN) auto
 
-notation times (infixl "*" 70)
-notation Groups.one ("1")
-
 context comm_monoid_add
 begin