src/HOL/Library/Multiset.thy
changeset 40210 aee7ef725330
parent 39533 91a0ff0ff237
child 40250 8792b0b89dcf
--- a/src/HOL/Library/Multiset.thy	Wed Oct 27 08:58:03 2010 +0200
+++ b/src/HOL/Library/Multiset.thy	Wed Oct 27 16:40:31 2010 +0200
@@ -837,11 +837,11 @@
 context linorder
 begin
 
-lemma multiset_of_insort_key [simp]:
+lemma multiset_of_insort [simp]:
   "multiset_of (insort_key k x xs) = {#x#} + multiset_of xs"
   by (induct xs) (simp_all add: ac_simps)
  
-lemma multiset_of_sort_key [simp]:
+lemma multiset_of_sort [simp]:
   "multiset_of (sort_key k xs) = multiset_of xs"
   by (induct xs) (simp_all add: ac_simps)