src/HOL/Auth/Message.thy
changeset 32117 0762b9ad83df
parent 30607 c3d1590debd8
child 32149 ef59550a55d3
equal deleted inserted replaced
32116:045e7ca3ea74 32117:0762b9ad83df
   853 
   853 
   854 (*Analysis of Fake cases.  Also works for messages that forward unknown parts,
   854 (*Analysis of Fake cases.  Also works for messages that forward unknown parts,
   855   but this application is no longer necessary if analz_insert_eq is used.
   855   but this application is no longer necessary if analz_insert_eq is used.
   856   Abstraction over i is ESSENTIAL: it delays the dereferencing of claset
   856   Abstraction over i is ESSENTIAL: it delays the dereferencing of claset
   857   DEPENDS UPON "X" REFERRING TO THE FRADULENT MESSAGE *)
   857   DEPENDS UPON "X" REFERRING TO THE FRADULENT MESSAGE *)
       
   858 
       
   859 fun impOfSubs th = th RSN (2, @{thm rev_subsetD})
   858 
   860 
   859 (*Apply rules to break down assumptions of the form
   861 (*Apply rules to break down assumptions of the form
   860   Y \<in> parts(insert X H)  and  Y \<in> analz(insert X H)
   862   Y \<in> parts(insert X H)  and  Y \<in> analz(insert X H)
   861 *)
   863 *)
   862 val Fake_insert_tac = 
   864 val Fake_insert_tac =