equal
deleted
inserted
replaced
783 be pulled out using the @{text analz_insert} rules\<close> |
783 be pulled out using the @{text analz_insert} rules\<close> |
784 |
784 |
785 lemmas pushKeys = |
785 lemmas pushKeys = |
786 insert_commute [of "Key K" "Agent C"] |
786 insert_commute [of "Key K" "Agent C"] |
787 insert_commute [of "Key K" "Nonce N"] |
787 insert_commute [of "Key K" "Nonce N"] |
788 insert_commute [of "Key K" "Number N"] |
|
789 insert_commute [of "Key K" "Hash X"] |
|
790 insert_commute [of "Key K" "MPair X Y"] |
788 insert_commute [of "Key K" "MPair X Y"] |
791 insert_commute [of "Key K" "Crypt X K'"] |
789 insert_commute [of "Key K" "Crypt X K'"] |
792 for K C N X Y K' |
790 for K C N X Y K' |
793 |
791 |
794 lemmas pushCrypts = |
792 lemmas pushCrypts = |
795 insert_commute [of "Crypt X K" "Agent C"] |
793 insert_commute [of "Crypt X K" "Agent C"] |
796 insert_commute [of "Crypt X K" "Agent C"] |
794 insert_commute [of "Crypt X K" "Agent C"] |
797 insert_commute [of "Crypt X K" "Nonce N"] |
795 insert_commute [of "Crypt X K" "Nonce N"] |
798 insert_commute [of "Crypt X K" "Number N"] |
|
799 insert_commute [of "Crypt X K" "Hash X'"] |
|
800 insert_commute [of "Crypt X K" "MPair X' Y"] |
796 insert_commute [of "Crypt X K" "MPair X' Y"] |
801 for X K C N X' Y |
797 for X K C N X' Y |
802 |
798 |
803 text\<open>Cannot be added with @{text "[simp]"} -- messages should not always be |
799 text\<open>Cannot be added with @{text "[simp]"} -- messages should not always be |
804 re-ordered.\<close> |
800 re-ordered.\<close> |