src/HOL/SET_Protocol/Message_SET.thy
changeset 36866 426d5781bb25
parent 35703 29cb504abbb5
child 41413 64cd30d6b0b8
--- a/src/HOL/SET_Protocol/Message_SET.thy	Wed May 12 15:25:58 2010 +0200
+++ b/src/HOL/SET_Protocol/Message_SET.thy	Wed May 12 16:44:49 2010 +0200
@@ -93,10 +93,10 @@
 by (simp add: nat_of_agent_def inj_on_def curry_def prod_encode_eq split: agent.split) 
 
 
-constdefs
+definition
   (*Keys useful to decrypt elements of a message set*)
   keysFor :: "msg set => key set"
-  "keysFor H == invKey ` {K. \<exists>X. Crypt K X \<in> H}"
+  where "keysFor H = invKey ` {K. \<exists>X. Crypt K X \<in> H}"
 
 subsubsection{*Inductive definition of all "parts" of a message.*}