src/CCL/Gfp.ML
changeset 1459 d12da312eff4
parent 757 2ca12511676d
child 2035 e329b36d9136
--- a/src/CCL/Gfp.ML	Mon Jan 29 13:56:41 1996 +0100
+++ b/src/CCL/Gfp.ML	Mon Jan 29 13:58:15 1996 +0100
@@ -1,9 +1,9 @@
-(*  Title: 	CCL/gfp
+(*  Title:      CCL/gfp
     ID:         $Id$
 
 Modified version of
-    Title: 	HOL/gfp
-    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
+    Title:      HOL/gfp
+    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1993  University of Cambridge
 
 For gfp.thy.  The Knaster-Tarski Theorem for greatest fixed points.
@@ -28,12 +28,12 @@
 
 val [mono] = goal Gfp.thy "mono(f) ==> gfp(f) <= f(gfp(f))";
 by (EVERY1 [rtac gfp_least, rtac subset_trans, atac,
-	    rtac (mono RS monoD), rtac gfp_upperbound, atac]);
+            rtac (mono RS monoD), rtac gfp_upperbound, atac]);
 qed "gfp_lemma2";
 
 val [mono] = goal Gfp.thy "mono(f) ==> f(gfp(f)) <= gfp(f)";
 by (EVERY1 [rtac gfp_upperbound, rtac (mono RS monoD), 
-	    rtac gfp_lemma2, rtac mono]);
+            rtac gfp_lemma2, rtac mono]);
 qed "gfp_lemma3";
 
 val [mono] = goal Gfp.thy "mono(f) ==> gfp(f) = f(gfp(f))";