src/ZF/UNITY/AllocImpl.thy
changeset 26289 9d2c375e242b
parent 24893 b8ef7afe3a6b
child 32960 69916a850301
--- a/src/ZF/UNITY/AllocImpl.thy	Sat Mar 15 22:07:28 2008 +0100
+++ b/src/ZF/UNITY/AllocImpl.thy	Sat Mar 15 22:07:29 2008 +0100
@@ -1,4 +1,4 @@
-(*Title: ZF/UNITY/AllocImpl
+(*  Title: ZF/UNITY/AllocImpl.thy
     ID:    $Id$
     Author:     Sidi O Ehmety, Cambridge University Computer Laboratory
     Copyright   2002  University of Cambridge
@@ -124,7 +124,8 @@
 
 (** Safety property: (28) **)
 lemma alloc_prog_Increasing_giv: "alloc_prog \<in> program guarantees Incr(lift(giv))"
-apply (auto intro!: increasing_imp_Increasing simp add: guar_def increasing_def alloc_prog_ok_iff alloc_prog_Allowed, safety+)
+apply (auto intro!: increasing_imp_Increasing simp add: guar_def
+  Increasing.increasing_def alloc_prog_ok_iff alloc_prog_Allowed, safety+)
 apply (auto dest: ActsD)
 apply (drule_tac f = "lift (giv) " in preserves_imp_eq)
 apply auto