src/HOL/Library/AList.thy
changeset 69661 a03a63b81f44
parent 69593 3dda49e08b9d
child 73678 78929c029785
--- a/src/HOL/Library/AList.thy	Mon Jan 14 18:33:53 2019 +0000
+++ b/src/HOL/Library/AList.thy	Mon Jan 14 18:35:03 2019 +0000
@@ -82,7 +82,7 @@
   by (simp add: update_conv' map_upd_Some_unfold)
 
 lemma image_update [simp]: "x \<notin> A \<Longrightarrow> map_of (update x y al) ` A = map_of al ` A"
-  by (simp add: update_conv')
+  by (auto simp add: update_conv')
 
 qualified definition updates ::
     "'key list \<Rightarrow> 'val list \<Rightarrow> ('key \<times> 'val) list \<Rightarrow> ('key \<times> 'val) list"