src/HOL/Auth/Smartcard/Smartcard.thy
changeset 32631 2489e3c3562b
parent 32149 ef59550a55d3
child 32960 69916a850301
equal deleted inserted replaced
32630:133e4a6474e3 32631:2489e3c3562b
     1 (*  ID:         $Id$
     1 (* Author:     Giampaolo Bella, Catania University
     2     Author:     Giampaolo Bella, Catania University
       
     3 *)
     2 *)
     4 
     3 
     5 header{*Theory of smartcards*}
     4 header{*Theory of smartcards*}
     6 
     5 
     7 theory Smartcard imports EventSC begin
     6 theory Smartcard
       
     7 imports EventSC All_Symmetric
       
     8 begin
     8 
     9 
     9 text{*  
    10 text{*  
    10 As smartcards handle long-term (symmetric) keys, this theoy extends and 
    11 As smartcards handle long-term (symmetric) keys, this theoy extends and 
    11 supersedes theory Private.thy
    12 supersedes theory Private.thy
    12 
    13 
    39   pairK_disj_shrK [iff]: "pairK(A,B) \<noteq> shrK P"
    40   pairK_disj_shrK [iff]: "pairK(A,B) \<noteq> shrK P"
    40   pairK_disj_pin [iff]:  "pairK(A,B) \<noteq> pin P"
    41   pairK_disj_pin [iff]:  "pairK(A,B) \<noteq> pin P"
    41   shrK_disj_crdK [iff]:  "shrK P \<noteq> crdK C"
    42   shrK_disj_crdK [iff]:  "shrK P \<noteq> crdK C"
    42   shrK_disj_pin [iff]:  "shrK P \<noteq> pin Q"
    43   shrK_disj_pin [iff]:  "shrK P \<noteq> pin Q"
    43   crdK_disj_pin [iff]:   "crdK C \<noteq> pin P"
    44   crdK_disj_pin [iff]:   "crdK C \<noteq> pin P"
    44 
       
    45 
       
    46 text{*All keys are symmetric*}
       
    47 defs  all_symmetric_def: "all_symmetric == True"
       
    48 
       
    49 lemma isSym_keys: "K \<in> symKeys"	
       
    50 by (simp add: symKeys_def all_symmetric_def invKey_symmetric) 
       
    51 
       
    52 
    45 
    53 constdefs
    46 constdefs
    54   legalUse :: "card => bool" ("legalUse (_)")
    47   legalUse :: "card => bool" ("legalUse (_)")
    55   "legalUse C == C \<notin> stolen"
    48   "legalUse C == C \<notin> stolen"
    56 
    49