src/HOL/Auth/Public.thy
changeset 3683 aafe719dff14
parent 3519 ab0a9fbed4c0
child 5183 89f162de39cf
--- a/src/HOL/Auth/Public.thy	Wed Sep 17 16:40:52 1997 +0200
+++ b/src/HOL/Auth/Public.thy	Thu Sep 18 13:24:04 1997 +0200
@@ -26,7 +26,7 @@
   initState_Friend  "initState (Friend i) =    
  		         insert (Key (priK (Friend i))) (Key `` range pubK)"
   initState_Spy     "initState Spy        =    
- 		         (Key``invKey``pubK``lost) Un (Key `` range pubK)"
+ 		         (Key``invKey``pubK``bad) Un (Key `` range pubK)"
 
 
 rules