src/HOL/Auth/Event.thy
changeset 58305 57752a91eec4
parent 53428 3083c611ec40
child 58310 91ea607a34d8
--- a/src/HOL/Auth/Event.thy	Thu Sep 11 18:54:36 2014 +0200
+++ b/src/HOL/Auth/Event.thy	Thu Sep 11 18:54:36 2014 +0200
@@ -15,7 +15,7 @@
 consts  (*Initial states of agents -- parameter of the construction*)
   initState :: "agent => msg set"
 
-datatype
+datatype_new
   event = Says  agent agent msg
         | Gets  agent       msg
         | Notes agent       msg