doc-src/TutorialI/Protocol/Message.thy
changeset 32265 fa8872f21ac3
parent 32149 ef59550a55d3
child 32960 69916a850301
equal deleted inserted replaced
32264:0be31453f698 32265:fa8872f21ac3
   839   DEPENDS UPON "X" REFERRING TO THE FRADULENT MESSAGE *)
   839   DEPENDS UPON "X" REFERRING TO THE FRADULENT MESSAGE *)
   840 
   840 
   841 (*Apply rules to break down assumptions of the form
   841 (*Apply rules to break down assumptions of the form
   842   Y \<in> parts(insert X H)  and  Y \<in> analz(insert X H)
   842   Y \<in> parts(insert X H)  and  Y \<in> analz(insert X H)
   843 *)
   843 *)
       
   844 fun impOfSubs th = th RSN (2, @{thm rev_subsetD})
       
   845 
   844 val Fake_insert_tac = 
   846 val Fake_insert_tac = 
   845     dresolve_tac [impOfSubs Fake_analz_insert,
   847     dresolve_tac [impOfSubs Fake_analz_insert,
   846                   impOfSubs Fake_parts_insert] THEN'
   848                   impOfSubs Fake_parts_insert] THEN'
   847     eresolve_tac [asm_rl, thm"synth.Inj"];
   849     eresolve_tac [asm_rl, thm"synth.Inj"];
   848 
   850