author | wenzelm |
Wed, 30 Dec 2015 18:24:36 +0100 | |
changeset 61985 | a63a11b09335 |
parent 61830 | 4f5ab843cf5b |
child 62145 | 5b946c81dfbf |
permissions | -rw-r--r-- |
32631 | 1 |
theory All_Symmetric |
2 |
imports Message |
|
3 |
begin |
|
1944 | 4 |
|
61830 | 5 |
text \<open>All keys are symmetric\<close> |
1944 | 6 |
|
32631 | 7 |
defs all_symmetric_def: "all_symmetric \<equiv> True" |
14145
2e31b8cc8788
ZhouGollmann: new example (fair non-repudiation protocol)
paulson
parents:
13922
diff
changeset
|
8 |
|
32631 | 9 |
lemma isSym_keys: "K \<in> symKeys" |
10 |
by (simp add: symKeys_def all_symmetric_def invKey_symmetric) |
|
18886 | 11 |
|
32631 | 12 |
end |