tidied
authorpaulson
Wed, 20 Sep 2006 15:11:46 +0200
changeset 20648 742c30fc3fcb
parent 20647 680b58597f65
child 20649 5079b9ee1ef5
tidied
src/HOL/Auth/Message.thy
--- a/src/HOL/Auth/Message.thy	Wed Sep 20 14:02:41 2006 +0200
+++ b/src/HOL/Auth/Message.thy	Wed Sep 20 15:11:46 2006 +0200
@@ -941,8 +941,7 @@
      "X \<in> synth (analz H) ==> parts{X} \<subseteq> synth (analz H) \<union> parts H";
 apply (rule subset_trans) 
  apply (erule_tac [2] Fake_parts_insert)
-apply (rule parts_mono)  
-apply (blast intro: elim:); 
+apply (rule parts_mono, blast)
 done
 
 lemmas Fake_parts_sing_imp_Un = Fake_parts_sing [THEN [2] rev_subsetD]