src/HOL/Auth/Guard/Extensions.thy
changeset 44890 22f665a2e91c
parent 41775 6214816d79d3
child 45600 1bbbac9a0cb0
--- a/src/HOL/Auth/Guard/Extensions.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Auth/Guard/Extensions.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -198,7 +198,7 @@
 
 lemma parts_invKey [rule_format,dest]:"X:parts {Y} ==>
 X:analz (insert (Crypt K Y) H) --> X ~:analz H --> Key (invKey K):analz H"
-by (erule parts.induct, (fastsimp dest: parts.Fst parts.Snd parts.Body)+)
+by (erule parts.induct, (fastforce dest: parts.Fst parts.Snd parts.Body)+)
 
 lemma in_analz: "Y:analz H ==> EX X. X:H & Y:parts {X}"
 by (erule analz.induct, auto intro: parts.Fst parts.Snd parts.Body)