src/HOL/Auth/Shared.thy
changeset 13507 febb8e5d2a9d
parent 12415 74977582a585
child 13907 2bc462b99e70
equal deleted inserted replaced
13506:acc18a5d2b1a 13507:febb8e5d2a9d
    37 use "Shared_lemmas.ML"
    37 use "Shared_lemmas.ML"
    38 
    38 
    39 (*Lets blast_tac perform this step without needing the simplifier*)
    39 (*Lets blast_tac perform this step without needing the simplifier*)
    40 lemma invKey_shrK_iff [iff]:
    40 lemma invKey_shrK_iff [iff]:
    41      "(Key (invKey K) \<in> X) = (Key K \<in> X)"
    41      "(Key (invKey K) \<in> X) = (Key K \<in> X)"
    42 by auto;
    42 by auto
    43 
    43 
    44 (*Specialized methods*)
    44 (*Specialized methods*)
    45 
    45 
    46 method_setup analz_freshK = {*
    46 method_setup analz_freshK = {*
    47     Method.no_args
    47     Method.no_args