src/HOL/Library/DAList_Multiset.thy
changeset 60515 484559628038
parent 60495 d7ff0a1df90a
child 60679 ade12ef2773c
equal deleted inserted replaced
60514:78a82c37b4b2 60515:484559628038
   265     unfolding mset_less_eq_Bag0 by auto
   265     unfolding mset_less_eq_Bag0 by auto
   266 qed
   266 qed
   267 
   267 
   268 declare multiset_inter_def [code]
   268 declare multiset_inter_def [code]
   269 declare sup_subset_mset_def [code]
   269 declare sup_subset_mset_def [code]
   270 declare multiset_of.simps [code]
   270 declare mset.simps [code]
   271 
   271 
   272 
   272 
   273 fun fold_impl :: "('a \<Rightarrow> nat \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'b \<Rightarrow> ('a \<times> nat) list \<Rightarrow> 'b"
   273 fun fold_impl :: "('a \<Rightarrow> nat \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'b \<Rightarrow> ('a \<times> nat) list \<Rightarrow> 'b"
   274 where
   274 where
   275   "fold_impl fn e ((a,n) # ms) = (fold_impl fn ((fn a n) e) ms)"
   275   "fold_impl fn e ((a,n) # ms) = (fold_impl fn ((fn a n) e) ms)"