src/HOL/Auth/Smartcard/EventSC.thy
changeset 20768 1d478c2d621f
parent 18886 9f27383426db
child 21404 eb85850d3eb7
--- a/src/HOL/Auth/Smartcard/EventSC.thy	Thu Sep 28 23:42:32 2006 +0200
+++ b/src/HOL/Auth/Smartcard/EventSC.thy	Thu Sep 28 23:42:35 2006 +0200
@@ -24,10 +24,9 @@
  cloned  :: "card set"   (* cloned smart cards*)
  secureM :: "bool"(*assumption of secure means between agents and their cards*)
 
-syntax
+abbreviation
   insecureM :: bool (*certain protocols make no assumption of secure means*)
-translations
-  "insecureM" == "\<not>secureM"
+  "insecureM == \<not>secureM"
 
 
 text{*Spy has access to his own key for spoof messages, but Server is secure*}