src/HOL/Library/Multiset.thy
changeset 61566 c3d6e570ccef
parent 61424 c3658c18b7bc
child 61585 a9599d3d7610
--- a/src/HOL/Library/Multiset.thy	Wed Nov 04 08:13:49 2015 +0100
+++ b/src/HOL/Library/Multiset.thy	Wed Nov 04 08:13:52 2015 +0100
@@ -1060,7 +1060,7 @@
   "mset_set = folding.F (\<lambda>x M. {#x#} + M) {#}"
 
 interpretation mset_set!: folding "\<lambda>x M. {#x#} + M" "{#}"
-where
+rewrites
   "folding.F (\<lambda>x M. {#x#} + M) {#} = mset_set"
 proof -
   interpret comp_fun_commute "\<lambda>x M. {#x#} + M"
@@ -1223,7 +1223,7 @@
   where "msetsum = comm_monoid_mset.F plus 0"
 
 sublocale msetsum!: comm_monoid_mset plus 0
-  where "comm_monoid_mset.F plus 0 = msetsum"
+  rewrites "comm_monoid_mset.F plus 0 = msetsum"
 proof -
   show "comm_monoid_mset plus 0" ..
   from msetsum_def show "comm_monoid_mset.F plus 0 = msetsum" ..
@@ -1281,7 +1281,7 @@
   where "msetprod = comm_monoid_mset.F times 1"
 
 sublocale msetprod!: comm_monoid_mset times 1
-  where "comm_monoid_mset.F times 1 = msetprod"
+  rewrites "comm_monoid_mset.F times 1 = msetprod"
 proof -
   show "comm_monoid_mset times 1" ..
   show "comm_monoid_mset.F times 1 = msetprod" using msetprod_def ..