src/HOL/Auth/Recur.thy
changeset 62343 24106dc44def
parent 61956 38b73f7940af
child 67613 ce654b0e6d69
--- a/src/HOL/Auth/Recur.thy	Wed Feb 17 21:51:55 2016 +0100
+++ b/src/HOL/Auth/Recur.thy	Wed Feb 17 21:51:56 2016 +0100
@@ -337,7 +337,7 @@
          RB \<in> responses evs |]
      ==> (Key K \<in> parts{RB} | Key K \<in> analz H)"
 apply (erule rev_mp, erule responses.induct)
-apply (simp_all del: image_insert
+apply (simp_all del: image_insert parts_image
              add: analz_image_freshK_simps resp_analz_image_freshK_lemma)
 txt\<open>Simplification using two distinct treatments of "image"\<close>
 apply (simp add: parts_insert2, blast)
@@ -389,7 +389,7 @@
 apply (erule respond.induct)
 apply (frule_tac [2] respond_imp_responses)
 apply (frule_tac [2] respond_imp_not_used)
-apply (simp_all del: image_insert
+apply (simp_all del: image_insert parts_image
                 add: analz_image_freshK_simps split_ifs shrK_in_analz_respond
                      resp_analz_image_freshK parts_insert2)
 txt\<open>Base case of respond\<close>