src/ZF/Fixedpt.thy
changeset 13356 c9cfe1638bf2
parent 13220 62c899c77151
child 14046 6616e6c53d48
--- a/src/ZF/Fixedpt.thy	Sun Jul 14 15:11:21 2002 +0200
+++ b/src/ZF/Fixedpt.thy	Sun Jul 14 15:14:43 2002 +0200
@@ -3,11 +3,11 @@
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1992  University of Cambridge
 
-Least and greatest fixed points; the Knaster-Tarski Theorem
-
 Proved in the lattice of subsets of D, namely Pow(D), with Inter as glb
 *)
 
+header{*Least and Greatest Fixed Points; the Knaster-Tarski Theorem*}
+
 theory Fixedpt = equalities:
 
 constdefs
@@ -23,7 +23,7 @@
      "gfp(D,h) == Union({X: Pow(D). X <= h(X)})"
 
 
-(*** Monotone operators ***)
+subsection{*Monotone Operators*}
 
 lemma bnd_monoI:
     "[| h(D)<=D;   
@@ -124,7 +124,7 @@
 apply (erule lfp_unfold)
 done
 
-(*** General induction rule for least fixedpoints ***)
+subsection{*General Induction Rule for Least Fixedpoints*}
 
 lemma Collect_is_pre_fixedpt:
     "[| bnd_mono(D,h);  !!x. x : h(Collect(lfp(D,h),P)) ==> P(x) |]
@@ -243,7 +243,7 @@
 done
 
 
-(*** Coinduction rules for greatest fixed points ***)
+subsection{*Coinduction Rules for Greatest Fixed Points*}
 
 (*weak version*)
 lemma weak_coinduct: "[| a: X;  X <= h(X);  X <= D |] ==> a : gfp(D,h)"