adapted proof
authorhaftmann
Mon, 21 Sep 2009 15:56:15 +0200
changeset 32695 66ae4e8b1309
parent 32694 0264f360438d
child 32696 46a20c74bd91
adapted proof
src/HOL/Auth/Guard/Extensions.thy
--- a/src/HOL/Auth/Guard/Extensions.thy	Mon Sep 21 15:35:24 2009 +0200
+++ b/src/HOL/Auth/Guard/Extensions.thy	Mon Sep 21 15:56:15 2009 +0200
@@ -11,7 +11,9 @@
 
 header {*Extensions to Standard Theories*}
 
-theory Extensions imports "../Event" begin
+theory Extensions
+imports "../Event"
+begin
 
 subsection{*Extensions to Theory @{text Set}*}
 
@@ -173,7 +175,7 @@
 subsubsection{*lemmas on analz*}
 
 lemma analz_UnI1 [intro]: "X:analz G ==> X:analz (G Un H)"
-by (subgoal_tac "G <= G Un H", auto dest: analz_mono)
+  by (subgoal_tac "G <= G Un H") (blast dest: analz_mono)+
 
 lemma analz_sub: "[| X:analz G; G <= H |] ==> X:analz H"
 by (auto dest: analz_mono)