src/HOL/Auth/Smartcard/EventSC.thy
changeset 46471 2289a3869c88
parent 45605 a89b4bc311a5
child 53428 3083c611ec40
equal deleted inserted replaced
46470:b0331b0d33a3 46471:2289a3869c88
   235 
   235 
   236 
   236 
   237 text{*Elimination rules: derive contradictions from old Says events containing
   237 text{*Elimination rules: derive contradictions from old Says events containing
   238   items known to be fresh*}
   238   items known to be fresh*}
   239 lemmas knows_Spy_partsEs =
   239 lemmas knows_Spy_partsEs =
   240      Says_imp_knows_Spy [THEN parts.Inj, THEN revcut_rl]
   240      Says_imp_knows_Spy [THEN parts.Inj, elim_format]
   241      parts.Body [THEN revcut_rl]
   241      parts.Body [elim_format]
   242 
   242 
   243 
   243 
   244 
   244 
   245 subsection{*Knowledge of Agents*}
   245 subsection{*Knowledge of Agents*}
   246 
   246