--- a/src/HOL/Auth/Guard/Guard.thy Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/Auth/Guard/Guard.thy Mon Mar 01 13:40:23 2010 +0100
@@ -76,7 +76,7 @@
subsection{*guarded sets*}
-constdefs Guard :: "nat => key set => msg set => bool"
+definition Guard :: "nat => key set => msg set => bool" where
"Guard n Ks H == ALL X. X:H --> X:guard n Ks"
subsection{*basic facts about @{term Guard}*}
@@ -241,7 +241,7 @@
subsection{*list corresponding to "decrypt"*}
-constdefs decrypt' :: "msg list => key => msg => msg list"
+definition decrypt' :: "msg list => key => msg => msg list" where
"decrypt' l K Y == Y # remove l (Crypt K Y)"
declare decrypt'_def [simp]