src/ZF/UNITY/ClientImpl.thy
changeset 26289 9d2c375e242b
parent 24893 b8ef7afe3a6b
child 32960 69916a850301
--- a/src/ZF/UNITY/ClientImpl.thy	Sat Mar 15 22:07:28 2008 +0100
+++ b/src/ZF/UNITY/ClientImpl.thy	Sat Mar 15 22:07:29 2008 +0100
@@ -121,7 +121,7 @@
 "client_prog: program guarantees Incr(lift(ask)) Int Incr(lift(rel))"
 apply (unfold guar_def)
 apply (auto intro!: increasing_imp_Increasing 
-            simp add: client_prog_ok_iff increasing_def preserves_imp_prefix)
+            simp add: client_prog_ok_iff Increasing.increasing_def preserves_imp_prefix)
 apply (safety, force, force)+
 done