src/HOL/Auth/Shared.thy
author paulson
Mon, 23 Sep 1996 18:19:38 +0200
changeset 2012 1b234f1fd9c7
parent 1967 0ff58b41c037
child 2032 1bbf1bdcaf56
permissions -rw-r--r--
Removal of the Notes constructor
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
1943
20574dca5a3e Renaming and simplification
paulson
parents: 1934
diff changeset
    14
  shrK    :: agent => key  (*symmetric keys*)
1965
789c12ea0b30 Stronger proofs; work for Otway-Rees
paulson
parents: 1943
diff changeset
    15
  leaked  :: nat set       (*Friendly agents whose keys have leaked to Enemy*)
1934
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    16
1967
0ff58b41c037 "bad" set simplifies statements of many theorems
paulson
parents: 1965
diff changeset
    17
constdefs     (*Enemy and compromised agents*)
0ff58b41c037 "bad" set simplifies statements of many theorems
paulson
parents: 1965
diff changeset
    18
  bad     :: agent set     "bad == insert Enemy (Friend``leaked)"
0ff58b41c037 "bad" set simplifies statements of many theorems
paulson
parents: 1965
diff changeset
    19
1934
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    20
rules
1943
20574dca5a3e Renaming and simplification
paulson
parents: 1934
diff changeset
    21
  isSym_shrK "isSymKey (shrK A)"
1934
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    22
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    23
consts  (*Initial states of agents -- parameter of the construction*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    24
  initState :: agent => msg set
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    25
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    26
primrec initState agent
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    27
        (*Server knows all keys; other agents know only their own*)
1943
20574dca5a3e Renaming and simplification
paulson
parents: 1934
diff changeset
    28
  initState_Server  "initState Server     = Key `` range shrK"
20574dca5a3e Renaming and simplification
paulson
parents: 1934
diff changeset
    29
  initState_Friend  "initState (Friend i) = {Key (shrK (Friend i))}"
1967
0ff58b41c037 "bad" set simplifies statements of many theorems
paulson
parents: 1965
diff changeset
    30
  initState_Enemy   "initState Enemy      = Key``shrK``bad"
1934
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
datatype  (*Messages, and components of agent stores*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    33
  event = Says agent agent msg
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
consts  
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    36
  sees1 :: [agent, event] => msg set
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    37
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    38
primrec sees1 event
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    39
           (*First agent recalls all that it says, but NOT everything
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    40
             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
    41
  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
    42
          (*part of A's internal state*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    43
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    44
consts  
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    45
  sees :: [agent, event list] => msg set
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    46
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    47
primrec sees list
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    48
        (*Initial knowledge includes all public keys and own private key*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    49
  sees_Nil  "sees A []       = initState A"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    50
  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
    51
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    52
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    53
(*Agents generate "random" nonces.  Different traces always yield
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    54
  different nonces.  Same applies for keys.*)
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    55
consts
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    56
  newN :: "event list => nat"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    57
  newK :: "event list => key"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    58
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    59
rules
1943
20574dca5a3e Renaming and simplification
paulson
parents: 1934
diff changeset
    60
  inj_shrK "inj shrK"
1934
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    61
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    62
  inj_newN   "inj newN"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    63
  fresh_newN "Nonce (newN evs) ~: parts (initState B)" 
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    64
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    65
  inj_newK   "inj newK"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    66
  fresh_newK "Key (newK evs) ~: parts (initState B)" 
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    67
  isSym_newK "isSymKey (newK evs)"
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    68
58573e7041b4 Separation of theory Event into two parts:
paulson
parents:
diff changeset
    69
end