src/HOL/Auth/Shared.thy
author paulson
Wed, 21 Aug 1996 13:25:27 +0200
changeset 1934 58573e7041b4
child 1943 20574dca5a3e
permissions -rw-r--r--
Separation of theory Event into two parts: Shared for general shared-key material NS_Shared for the Needham-Schroeder shared-key protocol
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1934
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     1
(*  Title:      HOL/Auth/Shared
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     2
    ID:         $Id$
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     4
    Copyright   1996  University of Cambridge
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     5
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     6
Theory of Shared Keys (common to all symmetric-key protocols)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     7
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     8
Server keys; initial states of agents; new nonces and keys; function "sees" 
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
     9
*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    10
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    11
Shared = Message + List + 
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    12
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    13
consts
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    14
  serverKey    :: agent => key  (*symmetric keys*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    15
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    16
rules
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    17
  isSym_serverKey "isSymKey (serverKey A)"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    18
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    19
consts  (*Initial states of agents -- parameter of the construction*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    20
  initState :: agent => msg set
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    21
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    22
primrec initState agent
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    23
        (*Server knows all keys; other agents know only their own*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    24
  initState_Server  "initState Server     = Key `` range serverKey"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    25
  initState_Friend  "initState (Friend i) = {Key (serverKey (Friend i))}"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    26
  initState_Enemy   "initState Enemy  = {Key (serverKey Enemy)}"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    27
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    28
datatype  (*Messages, and components of agent stores*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    29
  event = Says agent agent msg
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    30
        | Notes agent msg
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    31
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    32
consts  
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    33
  sees1 :: [agent, event] => msg set
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    34
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    35
primrec sees1 event
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    36
           (*First agent recalls all that it says, but NOT everything
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    37
             that is sent to it; it must note such things if/when received*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    38
  sees1_Says  "sees1 A (Says A' B X)  = (if A:{A',Enemy} then {X} else {})"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    39
          (*part of A's internal state*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    40
  sees1_Notes "sees1 A (Notes A' X)   = (if A=A' then {X} else {})"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    41
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    42
consts  
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    43
  sees :: [agent, event list] => msg set
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    44
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    45
primrec sees list
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    46
        (*Initial knowledge includes all public keys and own private key*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    47
  sees_Nil  "sees A []       = initState A"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    48
  sees_Cons "sees A (ev#evs) = sees1 A ev Un sees A evs"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    49
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    50
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    51
(*Agents generate "random" nonces.  Different traces always yield
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    52
  different nonces.  Same applies for keys.*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    53
consts
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    54
  newN :: "event list => nat"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    55
  newK :: "event list => key"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    56
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    57
rules
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    58
  inj_serverKey "inj serverKey"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    59
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    60
  inj_newN   "inj newN"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    61
  fresh_newN "Nonce (newN evs) ~: parts (initState B)" 
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    62
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    63
  inj_newK   "inj newK"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    64
  fresh_newK "Key (newK evs) ~: parts (initState B)" 
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    65
  isSym_newK "isSymKey (newK evs)"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    66
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    67
end