src/HOL/Auth/Smartcard/EventSC.thy
changeset 21404 eb85850d3eb7
parent 20768 1d478c2d621f
child 26302 68b073052e8c
--- a/src/HOL/Auth/Smartcard/EventSC.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/Auth/Smartcard/EventSC.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -25,7 +25,7 @@
  secureM :: "bool"(*assumption of secure means between agents and their cards*)
 
 abbreviation
-  insecureM :: bool (*certain protocols make no assumption of secure means*)
+  insecureM :: bool where (*certain protocols make no assumption of secure means*)
   "insecureM == \<not>secureM"