src/HOL/Metis_Examples/Message.thy
changeset 62390 842917225d56
parent 61984 cdea44c775fa
child 63167 0909deb8059b
equal deleted inserted replaced
62380:29800666e526 62390:842917225d56
   458                analz (insert (Crypt K X) H) =
   458                analz (insert (Crypt K X) H) =
   459                insert (Crypt K X) (analz (insert X H))"
   459                insert (Crypt K X) (analz (insert X H))"
   460 by (intro equalityI lemma1 lemma2)
   460 by (intro equalityI lemma1 lemma2)
   461 
   461 
   462 text{*Case analysis: either the message is secure, or it is not! Effective,
   462 text{*Case analysis: either the message is secure, or it is not! Effective,
   463 but can cause subgoals to blow up! Use with @{text "split_if"}; apparently
   463 but can cause subgoals to blow up! Use with @{text "if_split"}; apparently
   464 @{text "split_tac"} does not cope with patterns such as @{term"analz (insert
   464 @{text "split_tac"} does not cope with patterns such as @{term"analz (insert
   465 (Crypt K X) H)"} *}
   465 (Crypt K X) H)"} *}
   466 lemma analz_Crypt_if [simp]:
   466 lemma analz_Crypt_if [simp]:
   467      "analz (insert (Crypt K X) H) =
   467      "analz (insert (Crypt K X) H) =
   468           (if (Key (invKey K) \<in> analz H)
   468           (if (Key (invKey K) \<in> analz H)