src/HOLCF/IOA/Modelcheck/Cockpit.thy
changeset 17244 0b2ff9541727
parent 10127 86269867de34
child 19764 372065f34795
--- a/src/HOLCF/IOA/Modelcheck/Cockpit.thy	Sat Sep 03 16:49:48 2005 +0200
+++ b/src/HOLCF/IOA/Modelcheck/Cockpit.thy	Sat Sep 03 16:50:22 2005 +0200
@@ -1,43 +1,49 @@
 
-Cockpit = MuIOAOracle +
+(* $Id$ *)
+
+theory Cockpit
+imports MuIOAOracle
+begin
 
 datatype 'a action = Alarm 'a | Info 'a | Ack 'a
 datatype event = NONE | PonR | Eng | Fue
 
 
-(*This cockpit automaton is a deeply simplified version of the
+text {*
+  This cockpit automaton is a deeply simplified version of the
   control component of a helicopter alarm system considered in a study
   of ESG.  Some properties will be proved by using model checker
-  mucke.*)
+  mucke. *}
 
 automaton cockpit =
   signature
-    actions event action
+    actions "event action"
     inputs "Alarm a"
-    outputs "Ack a","Info a"
+    outputs "Ack a", "Info a"
   states
     APonR_incl :: bool
     info :: event
-  initially "info=NONE & ~APonR_incl"
+  initially "info = NONE & ~APonR_incl"
   transitions
     "Alarm a"
-      post info:="if (a=NONE) then info else a",
-        APonR_incl:="if (a=PonR) then True else APonR_incl"
+      post info := "if (a=NONE) then info else a",
+        APonR_incl := "if (a=PonR) then True else APonR_incl"
     "Info a"
       pre "(a=info)"
     "Ack a"
       pre "(a=PonR --> APonR_incl) & (a=NONE --> ~APonR_incl)"
-      post info:="NONE",APonR_incl:="if (a=PonR) then False else APonR_incl"
+      post info := "NONE",
+        APonR_incl := "if (a=PonR) then False else APonR_incl"
 
 automaton cockpit_hide = hide_action "Info a" in cockpit
 
-
-(*Subsequent automata express the properties to be proved, see also
-  Cockpit.ML*)
+text {*
+  Subsequent automata express the properties to be proved, see also
+  Cockpit.ML *}
 
 automaton Al_before_Ack =
   signature
-    actions event action
+    actions "event action"
     inputs "Alarm a"
     outputs "Ack a"
   states
@@ -52,7 +58,7 @@
 
 automaton Info_while_Al =
   signature
-    actions event action
+    actions "event action"
     inputs "Alarm a"
     outputs "Ack a", "Info i"
   states
@@ -69,7 +75,7 @@
 
 automaton Info_before_Al =
   signature
-    actions event action
+    actions "event action"
     inputs "Alarm a"
     outputs "Ack a", "Info i"
   states
@@ -83,4 +89,6 @@
     "Ack a"
       post info_at_NONE:="True"
 
+ML {* use_legacy_bindings (the_context ()) *}
+
 end