| author | berghofe | 
| Wed, 11 Jan 2006 18:21:23 +0100 | |
| changeset 18658 | 317a6f0ef8b9 | 
| parent 17456 | bcf7544875b2 | 
| child 20140 | 98acc6d0fab6 | 
| permissions | -rw-r--r-- | 
(* Title: CCL/Gfp.thy ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1992 University of Cambridge *) header {* Greatest fixed points *} theory Gfp imports Lfp begin constdefs gfp :: "['a set=>'a set] => 'a set" (*greatest fixed point*) "gfp(f) == Union({u. u <= f(u)})" ML {* use_legacy_bindings (the_context ()) *} end