src/HOL/Auth/KerberosV.thy
changeset 76290 64d29ebb7d3d
parent 69597 ff784d5a5bfb
child 76299 0ad6f6508274
equal deleted inserted replaced
76289:a6cc15ec45b2 76290:64d29ebb7d3d
   776 (*A fresh authK cannot be associated with any other
   776 (*A fresh authK cannot be associated with any other
   777   (with respect to a given trace). *)
   777   (with respect to a given trace). *)
   778 lemma Auth_fresh_not_AKcryptSK:
   778 lemma Auth_fresh_not_AKcryptSK:
   779      "\<lbrakk> Key authK \<notin> used evs; evs \<in> kerbV \<rbrakk>
   779      "\<lbrakk> Key authK \<notin> used evs; evs \<in> kerbV \<rbrakk>
   780       \<Longrightarrow> \<not> AKcryptSK authK servK evs"
   780       \<Longrightarrow> \<not> AKcryptSK authK servK evs"
   781 apply (unfold AKcryptSK_def)
   781 unfolding AKcryptSK_def
   782 apply (erule rev_mp)
   782 apply (erule rev_mp)
   783 apply (erule kerbV.induct)
   783 apply (erule kerbV.induct)
   784 apply (frule_tac [7] Says_ticket_parts)
   784 apply (frule_tac [7] Says_ticket_parts)
   785 apply (frule_tac [5] Says_ticket_parts, simp_all, blast)
   785 apply (frule_tac [5] Says_ticket_parts, simp_all, blast)
   786 done
   786 done
   819 done
   819 done
   820 
   820 
   821 text\<open>Long term keys are not issued as servKeys\<close>
   821 text\<open>Long term keys are not issued as servKeys\<close>
   822 lemma shrK_not_AKcryptSK:
   822 lemma shrK_not_AKcryptSK:
   823      "evs \<in> kerbV \<Longrightarrow> \<not> AKcryptSK K (shrK A) evs"
   823      "evs \<in> kerbV \<Longrightarrow> \<not> AKcryptSK K (shrK A) evs"
   824 apply (unfold AKcryptSK_def)
   824 unfolding AKcryptSK_def
   825 apply (erule kerbV.induct)
   825 apply (erule kerbV.induct)
   826 apply (frule_tac [7] Says_ticket_parts)
   826 apply (frule_tac [7] Says_ticket_parts)
   827 apply (frule_tac [5] Says_ticket_parts, auto)
   827 apply (frule_tac [5] Says_ticket_parts, auto)
   828 done
   828 done
   829 
   829