src/HOL/Library/AList_Impl.thy
changeset 46171 19f68d7671f0
parent 46133 d9fe85d3d2cd
equal deleted inserted replaced
46170:1b2e882f42d2 46171:19f68d7671f0
   691 lemma distinct_map_default:
   691 lemma distinct_map_default:
   692   assumes "distinct (map fst xs)"
   692   assumes "distinct (map fst xs)"
   693   shows "distinct (map fst (map_default k v f xs))"
   693   shows "distinct (map fst (map_default k v f xs))"
   694 using assms by (induct xs) (auto simp add: dom_map_default)
   694 using assms by (induct xs) (auto simp add: dom_map_default)
   695 
   695 
   696 hide_const (open) map_entry
   696 hide_const (open) update updates delete restrict clearjunk merge compose map_entry
   697 
   697 
   698 end
   698 end