changeset 16417 | 9bc16273c2d4 |
parent 11310 | 51e70b7bc315 |
child 23925 | ee98c2528a8f |
--- a/doc-src/TutorialI/Protocol/Event.thy Fri Jun 17 11:35:35 2005 +0200 +++ b/doc-src/TutorialI/Protocol/Event.thy Fri Jun 17 16:12:49 2005 +0200 @@ -11,8 +11,8 @@ stores are visible to him *) -theory Event = Message -files ("Event_lemmas.ML"): +theory Event imports Message +uses ("Event_lemmas.ML") begin consts (*Initial states of agents -- parameter of the construction*) initState :: "agent => msg set"