| changeset 32631 | 2489e3c3562b | 
| parent 28098 | c92850d2d16c | 
| child 61830 | 4f5ab843cf5b | 
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Auth/All_Symmetric.thy Mon Sep 21 15:33:40 2009 +0200 @@ -0,0 +1,12 @@ +theory All_Symmetric +imports Message +begin + +text {* All keys are symmetric *} + +defs all_symmetric_def: "all_symmetric \<equiv> True" + +lemma isSym_keys: "K \<in> symKeys" + by (simp add: symKeys_def all_symmetric_def invKey_symmetric) + +end