| author | wenzelm | 
| Wed, 22 Oct 1997 11:36:43 +0200 | |
| changeset 3970 | e1843233c694 | 
| parent 1474 | 3f7d67927fe2 | 
| child 17456 | bcf7544875b2 | 
| permissions | -rw-r--r-- | 
| 1474 | 1  | 
(* Title: HOL/lfp.thy  | 
| 0 | 2  | 
ID: $Id$  | 
| 1474 | 3  | 
Author: Lawrence C Paulson, Cambridge University Computer Laboratory  | 
| 0 | 4  | 
Copyright 1992 University of Cambridge  | 
5  | 
||
6  | 
The Knaster-Tarski Theorem  | 
|
7  | 
*)  | 
|
8  | 
||
9  | 
Lfp = Set +  | 
|
10  | 
consts lfp :: "['a set=>'a set] => 'a set"  | 
|
11  | 
rules  | 
|
12  | 
(*least fixed point*)  | 
|
13  | 
 lfp_def "lfp(f) == Inter({u. f(u) <= u})"
 | 
|
14  | 
end  |