src/HOL/UNITY/Lift.thy
changeset 10064 1a77667b21ef
parent 6718 e869ff059252
--- a/src/HOL/UNITY/Lift.thy	Fri Sep 22 17:25:09 2000 +0200
+++ b/src/HOL/UNITY/Lift.thy	Sat Sep 23 16:02:01 2000 +0200
@@ -108,6 +108,10 @@
          {(s,s'). s' = s (|floor := floor s - #1|)
 		       & ~ stop s & ~ up s & floor s ~: req s}"
 
+  (*This action is omitted from prior treatments, which therefore are
+    unrealistic: nobody asks the lift to do anything!  But adding this
+    action invalidates many of the existing progress arguments: various
+    "ensures" properties fail.*)
   button_press  :: "(state*state) set"
     "button_press ==
          {(s,s'). EX n. s' = s (|req := insert n (req s)|)
@@ -119,7 +123,8 @@
     "Lift == mk_program ({s. floor s = Min & ~ up s & move s & stop s &
 		          ~ open s & req s = {}},
 			 {request_act, open_act, close_act,
-			  req_up, req_down, move_up, move_down})"
+			  req_up, req_down, move_up, move_down},
+			 UNIV)"
 
 
   (** Invariants **)