src/HOL/Auth/Shared.thy
changeset 18749 31c2af8b0c60
parent 17744 3007c82f17ca
child 20048 a7964311f1fb
equal deleted inserted replaced
18748:1d7b0830a8a7 18749:31c2af8b0c60
    35 
    35 
    36 
    36 
    37 subsection{*Basic properties of shrK*}
    37 subsection{*Basic properties of shrK*}
    38 
    38 
    39 (*Injectiveness: Agents' long-term keys are distinct.*)
    39 (*Injectiveness: Agents' long-term keys are distinct.*)
    40 declare inj_shrK [THEN inj_eq, iff]
    40 lemmas shrK_injective = inj_shrK [THEN inj_eq]
       
    41 declare shrK_injective [iff]
    41 
    42 
    42 lemma invKey_K [simp]: "invKey K = K"
    43 lemma invKey_K [simp]: "invKey K = K"
    43 apply (insert isSym_keys)
    44 apply (insert isSym_keys)
    44 apply (simp add: symKeys_def) 
    45 apply (simp add: symKeys_def) 
    45 done
    46 done