use the noted theorem whenever possible, also in 'BNF_Def'
theory All_Symmetricimports Messagebegintext {* 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