src/HOL/UNITY/Lift_prog.thy
changeset 7880 62fb24e28e5e
parent 7878 43b03d412b82
child 7947 b999c1ab9327
--- a/src/HOL/UNITY/Lift_prog.thy	Mon Oct 18 15:20:21 1999 +0200
+++ b/src/HOL/UNITY/Lift_prog.thy	Mon Oct 18 16:16:03 1999 +0200
@@ -31,8 +31,8 @@
 		   lift_act i `` Acts F)"
 
   (*Argument C allows weak safety laws to be projected*)
-  drop_prog :: "[('a=>'b) set, 'a, ('a=>'b) program] => 'b program"
-    "drop_prog C i F ==
+  drop_prog :: "['a, ('a=>'b) set, ('a=>'b) program] => 'b program"
+    "drop_prog i C F ==
        mk_program (drop_set i (Init F),
 		   drop_act i `` Restrict C `` (Acts F))"