src/HOL/Auth/KerberosV.thy
changeset 76290 64d29ebb7d3d
parent 69597 ff784d5a5bfb
child 76299 0ad6f6508274
--- a/src/HOL/Auth/KerberosV.thy	Thu Oct 13 16:00:22 2022 +0100
+++ b/src/HOL/Auth/KerberosV.thy	Thu Oct 13 16:09:31 2022 +0100
@@ -778,7 +778,7 @@
 lemma Auth_fresh_not_AKcryptSK:
      "\<lbrakk> Key authK \<notin> used evs; evs \<in> kerbV \<rbrakk>
       \<Longrightarrow> \<not> AKcryptSK authK servK evs"
-apply (unfold AKcryptSK_def)
+unfolding AKcryptSK_def
 apply (erule rev_mp)
 apply (erule kerbV.induct)
 apply (frule_tac [7] Says_ticket_parts)
@@ -821,7 +821,7 @@
 text\<open>Long term keys are not issued as servKeys\<close>
 lemma shrK_not_AKcryptSK:
      "evs \<in> kerbV \<Longrightarrow> \<not> AKcryptSK K (shrK A) evs"
-apply (unfold AKcryptSK_def)
+unfolding AKcryptSK_def
 apply (erule kerbV.induct)
 apply (frule_tac [7] Says_ticket_parts)
 apply (frule_tac [5] Says_ticket_parts, auto)