src/HOL/Auth/Public.thy
changeset 11287 0103ee3082bf
parent 11270 a315a3862bb4
child 13922 75ae4244a596
equal deleted inserted replaced
11286:5116d92c6a83 11287:0103ee3082bf
    35   inj_pubK:        "inj pubK"
    35   inj_pubK:        "inj pubK"
    36   priK_neq_pubK:   "priK A ~= pubK B"
    36   priK_neq_pubK:   "priK A ~= pubK B"
    37 
    37 
    38 use "Public_lemmas.ML"
    38 use "Public_lemmas.ML"
    39 
    39 
       
    40 lemma [simp]: "K \\<in> symKeys ==> invKey K = K"
       
    41 by (simp add: symKeys_def)
       
    42 
    40 (*Specialized methods*)
    43 (*Specialized methods*)
    41 
    44 
    42 method_setup possibility = {*
    45 method_setup possibility = {*
    43     Method.ctxt_args (fn ctxt =>
    46     Method.ctxt_args (fn ctxt =>
    44         Method.METHOD (fn facts =>
    47         Method.METHOD (fn facts =>