src/HOL/SET_Protocol/Public_SET.thy
changeset 35416 d8d7d1b785af
parent 35068 544867142ea4
child 36866 426d5781bb25
--- a/src/HOL/SET_Protocol/Public_SET.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/SET_Protocol/Public_SET.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -161,21 +161,19 @@
 
 subsection{*Encryption Primitives*}
 
-constdefs
-
-  EXcrypt :: "[key,key,msg,msg] => msg"
+definition EXcrypt :: "[key,key,msg,msg] => msg" where
   --{*Extra Encryption*}
     (*K: the symmetric key   EK: the public encryption key*)
     "EXcrypt K EK M m ==
        {|Crypt K {|M, Hash m|}, Crypt EK {|Key K, m|}|}"
 
-  EXHcrypt :: "[key,key,msg,msg] => msg"
+definition EXHcrypt :: "[key,key,msg,msg] => msg" where
   --{*Extra Encryption with Hashing*}
     (*K: the symmetric key   EK: the public encryption key*)
     "EXHcrypt K EK M m ==
        {|Crypt K {|M, Hash m|}, Crypt EK {|Key K, m, Hash M|}|}"
 
-  Enc :: "[key,key,key,msg] => msg"
+definition Enc :: "[key,key,key,msg] => msg" where
   --{*Simple Encapsulation with SIGNATURE*}
     (*SK: the sender's signing key
       K: the symmetric key
@@ -183,7 +181,7 @@
     "Enc SK K EK M ==
        {|Crypt K (sign SK M), Crypt EK (Key K)|}"
 
-  EncB :: "[key,key,key,msg,msg] => msg"
+definition EncB :: "[key,key,key,msg,msg] => msg" where
   --{*Encapsulation with Baggage.  Keys as above, and baggage b.*}
     "EncB SK K EK M b == 
        {|Enc SK K EK {|M, Hash b|}, b|}"