src/HOL/Library/Multiset.thy
changeset 40210 aee7ef725330
parent 39533 91a0ff0ff237
child 40250 8792b0b89dcf
equal deleted inserted replaced
40208:54e5e8e0b2a4 40210:aee7ef725330
   835 qed
   835 qed
   836 
   836 
   837 context linorder
   837 context linorder
   838 begin
   838 begin
   839 
   839 
   840 lemma multiset_of_insort_key [simp]:
   840 lemma multiset_of_insort [simp]:
   841   "multiset_of (insort_key k x xs) = {#x#} + multiset_of xs"
   841   "multiset_of (insort_key k x xs) = {#x#} + multiset_of xs"
   842   by (induct xs) (simp_all add: ac_simps)
   842   by (induct xs) (simp_all add: ac_simps)
   843  
   843  
   844 lemma multiset_of_sort_key [simp]:
   844 lemma multiset_of_sort [simp]:
   845   "multiset_of (sort_key k xs) = multiset_of xs"
   845   "multiset_of (sort_key k xs) = multiset_of xs"
   846   by (induct xs) (simp_all add: ac_simps)
   846   by (induct xs) (simp_all add: ac_simps)
   847 
   847 
   848 text {*
   848 text {*
   849   This lemma shows which properties suffice to show that a function
   849   This lemma shows which properties suffice to show that a function