diff -r ecf80e37ed1a -r 8e2355ddce1b src/HOL/Library/AList.thy --- a/src/HOL/Library/AList.thy Wed Aug 18 23:04:58 2021 +0200 +++ b/src/HOL/Library/AList.thy Thu Aug 19 12:31:06 2021 +0200 @@ -424,7 +424,7 @@ qed lemma graph_map_of: "Map.graph (map_of al) = set (clearjunk al)" - by (metis distinct_clearjunk graph_map_of_if_distinct_ran map_of_clearjunk) + by (metis distinct_clearjunk graph_map_of_if_distinct_dom map_of_clearjunk) lemma clearjunk_update: "clearjunk (update k v al) = update k v (clearjunk al)" by (induct al rule: clearjunk.induct) (simp_all add: delete_update)