author | paulson |
Mon, 26 May 1997 12:38:29 +0200 | |
changeset 3342 | ec3b55fcb165 |
parent 1558 | 9c6ebfab4e05 |
child 3947 | eb707467f8c5 |
permissions | -rw-r--r-- |
1475 | 1 |
(* Title: HOL/Lfp.thy |
923 | 2 |
ID: $Id$ |
1475 | 3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
923 | 4 |
Copyright 1992 University of Cambridge |
5 |
||
6 |
The Knaster-Tarski Theorem |
|
7 |
*) |
|
8 |
||
1114 | 9 |
Lfp = mono + Prod + |
1558 | 10 |
|
11 |
constdefs |
|
12 |
lfp :: ['a set=>'a set] => 'a set |
|
13 |
"lfp(f) == Inter({u. f(u) <= u})" (*least fixed point*) |
|
14 |
||
923 | 15 |
end |