src/HOL/Auth/TLS.thy
changeset 3519 ab0a9fbed4c0
parent 3515 d8a71f6eaf40
child 3672 56e4365a0c99
--- a/src/HOL/Auth/TLS.thy	Mon Jul 14 12:44:09 1997 +0200
+++ b/src/HOL/Auth/TLS.thy	Mon Jul 14 12:47:21 1997 +0200
@@ -13,7 +13,7 @@
 Server, who is in charge of all public keys.
 
 The model assumes that no fraudulent certificates are present, but it does
-assume that some private keys are lost to the spy.
+assume that some private keys are to the spy.
 
 Abstracted from "The TLS Protocol, Version 1.0" by Tim Dierks and Christopher
 Allen, Transport Layer Security Working Group, 21 May 1997,
@@ -56,14 +56,8 @@
   (*Clashes with pubK and priK are impossible, but this axiom is needed.*)
   clientK_range "range clientK <= Compl (range serverK)"
 
-  (*Spy has access to his own key for spoof messages, but Server is secure*)
-  Spy_in_lost     "Spy: lost"
-  Server_not_lost "Server ~: lost"
 
-
-consts  lost :: agent set        (*No need for it to be a variable*)
-	tls  :: event list set
-
+consts    tls :: event list set
 inductive tls
   intrs 
     Nil  (*Initial trace is empty*)
@@ -71,7 +65,7 @@
 
     Fake (*The spy, an active attacker, MAY say anything he CAN say.*)
          "[| evs: tls;  B ~= Spy;  
-             X: synth (analz (sees lost Spy evs)) |]
+             X: synth (analz (sees Spy evs)) |]
           ==> Says Spy B X # evs : tls"
 
     SpyKeys (*The spy may apply clientK & serverK to nonces he's found*)