src/HOL/Auth/Guard/Auth_Guard_Shared.thy
author immler
Thu, 24 Sep 2015 14:29:08 +0200
changeset 61243 44b2d133063e
parent 58889 5b7a9633cfa8
child 61830 4f5ab843cf5b
permissions -rw-r--r--
exchange uniform limit and integral
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
32632
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
     1
(*  Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
1944
ea0f573b222b ROOT file for Auth directory
paulson
parents:
diff changeset
     2
    Copyright   1996  University of Cambridge
ea0f573b222b ROOT file for Auth directory
paulson
parents:
diff changeset
     3
*)
ea0f573b222b ROOT file for Auth directory
paulson
parents:
diff changeset
     4
58889
5b7a9633cfa8 modernized header uniformly as section;
wenzelm
parents: 32632
diff changeset
     5
section {* Blanqui's "guard" concept: protocol-independent secrecy *}
1944
ea0f573b222b ROOT file for Auth directory
paulson
parents:
diff changeset
     6
32632
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
     7
theory Auth_Guard_Shared
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
     8
imports
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
     9
  "Guard_OtwayRees"
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
    10
  "Guard_Yahalom"
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
    11
begin
14145
2e31b8cc8788 ZhouGollmann: new example (fair non-repudiation protocol)
paulson
parents: 13922
diff changeset
    12
32632
8ae912371831 added session entry point theories
haftmann
parents: 28098
diff changeset
    13
end