src/HOL/Auth/Shared.thy
changeset 3472 fb3c38c88c08
parent 3414 804c8a178a7f
child 3512 9dcb4daa15e8
--- a/src/HOL/Auth/Shared.thy	Tue Jul 01 10:38:11 1997 +0200
+++ b/src/HOL/Auth/Shared.thy	Tue Jul 01 10:39:28 1997 +0200
@@ -14,8 +14,8 @@
   shrK    :: agent => key  (*symmetric keys*)
 
 rules
-  (*ALL keys are symmetric*)
-  isSym_keys "isSymKey K"
+  isSym_keys "isSymKey K"	(*All keys are symmetric*)
+  inj_shrK   "inj shrK"		(*No two agents have the same long-term key*)
 
 consts  (*Initial states of agents -- parameter of the construction*)
   initState :: [agent set, agent] => msg set
@@ -61,25 +61,4 @@
     an unspecified finite number.*)
   Key_supply_ax  "finite KK ==> EX K. K ~: KK & Key K ~: used evs"
 
-
-(*Agents generate random (symmetric) keys and nonces.
-  The numeric argument is typically the length of the current trace.
-  An injective pairing function allows multiple keys/nonces to be generated
-	in one protocol round.  A typical candidate for npair(i,j) is
-	2^j(2i+1)
-*)
-
-consts
-  nPair :: "nat*nat => nat"
-  newN  :: "nat => nat"
-  newK  :: "nat => key"
-
-rules
-  inj_shrK        "inj shrK"
-  inj_nPair       "inj nPair"
-  inj_newN        "inj newN"
-  inj_newK        "inj newK"
-
-  newK_neq_shrK   "newK i ~= shrK A" 
-
 end