src/HOL/Auth/Shared.thy
changeset 13956 8fe7e12290e1
parent 13926 6e62e5357a10
child 14126 28824746d046
--- a/src/HOL/Auth/Shared.thy	Mon May 05 15:55:56 2003 +0200
+++ b/src/HOL/Auth/Shared.thy	Mon May 05 18:22:01 2003 +0200
@@ -242,7 +242,7 @@
      REPEAT_FIRST (resolve_tac [refl, conjI]))
 *}
 
-subsection{*Specialized rewriting for analz_insert_freshK*}
+subsection{*Specialized Rewriting for Theorems About @{term analz} and Image*}
 
 lemma subset_Compl_range: "A <= - (range shrK) ==> shrK x \<notin> A"
 by blast
@@ -250,7 +250,7 @@
 lemma insert_Key_singleton: "insert (Key K) H = Key ` {K} \<union> H"
 by blast
 
-lemma insert_Key_image: "insert (Key K) (Key`KK \<union> C) = Key ` (insert K KK) \<union> C"
+lemma insert_Key_image: "insert (Key K) (Key`KK \<union> C) = Key`(insert K KK) \<union> C"
 by blast
 
 (** Reverse the normal simplification of "image" to build up (not break down)