src/HOL/Auth/Message.thy
changeset 16796 140f1e0ea846
parent 16417 9bc16273c2d4
child 16818 2b82259cc7b2
--- a/src/HOL/Auth/Message.thy	Wed Jul 13 15:06:04 2005 +0200
+++ b/src/HOL/Auth/Message.thy	Wed Jul 13 15:06:20 2005 +0200
@@ -84,11 +84,11 @@
 lemma parts_mono: "G\<subseteq>H ==> parts(G) \<subseteq> parts(H)"
 apply auto
 apply (erule parts.induct) 
-apply (auto dest: Fst Snd Body) 
+apply (blast dest: Fst Snd Body)+
 done
 
 
-(*Equations hold because constructors are injective; cannot prove for all f*)
+text{*Equations hold because constructors are injective; cannot prove for all f*}
 lemma Friend_image_eq [simp]: "(Friend x \<in> Friend`A) = (x:A)"
 by auto