--- a/src/HOL/Auth/KerberosV.thy Thu Sep 28 23:42:32 2006 +0200
+++ b/src/HOL/Auth/KerberosV.thy Thu Sep 28 23:42:35 2006 +0200
@@ -8,33 +8,18 @@
text{*The "u" prefix indicates theorems referring to an updated version of the protocol. The "r" suffix indicates theorems where the confidentiality assumptions are relaxed by the corresponding arguments.*}
-syntax
+abbreviation
Kas :: agent
- Tgs :: agent --{*the two servers are translations...*}
+ "Kas == Server"
-
-translations
- "Kas" == "Server "
- "Tgs" == "Friend 0"
+ Tgs :: agent
+ "Tgs == Friend 0"
axioms
Tgs_not_bad [iff]: "Tgs \<notin> bad"
--{*Tgs is secure --- we already know that Kas is secure*}
-(*The current time is just the length of the trace!*)
-syntax
- CT :: "event list=>nat"
-
- expiredAK :: "[nat, event list] => bool"
-
- expiredSK :: "[nat, event list] => bool"
-
- expiredA :: "[nat, event list] => bool"
-
- valid :: "[nat, nat] => bool" ("valid _ wrt _")
-
-
constdefs
(* authKeys are those contained in an authTicket *)
authKeys :: "event list => key set"
@@ -81,16 +66,22 @@
replylife_LB [iff]: "Suc 0 \<le> replylife"
by blast
-translations
- "CT" == "length "
+abbreviation
+ (*The current time is just the length of the trace!*)
+ CT :: "event list=>nat"
+ "CT == length"
- "expiredAK T evs" == "authKlife + T < CT evs"
+ expiredAK :: "[nat, event list] => bool"
+ "expiredAK T evs == authKlife + T < CT evs"
- "expiredSK T evs" == "servKlife + T < CT evs"
+ expiredSK :: "[nat, event list] => bool"
+ "expiredSK T evs == servKlife + T < CT evs"
- "expiredA T evs" == "authlife + T < CT evs"
+ expiredA :: "[nat, event list] => bool"
+ "expiredA T evs == authlife + T < CT evs"
- "valid T1 wrt T2" == "T1 <= replylife + T2"
+ valid :: "[nat, nat] => bool" ("valid _ wrt _")
+ "valid T1 wrt T2 == T1 <= replylife + T2"
(*---------------------------------------------------------------------*)