src/ZF/Fixedpt.thy
author nipkow
Thu, 26 Nov 1998 12:18:08 +0100
changeset 5974 6acf3ff0f486
parent 3940 1d5bee4d047f
child 6093 87bf8c03b169
permissions -rw-r--r--
Added filter_prems_tac
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     1
(*  Title:      ZF/fixedpt.thy
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     2
    ID:         $Id$
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     3
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     4
    Copyright   1992  University of Cambridge
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     5
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     6
Least and greatest fixed points
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     7
*)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     8
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1478
diff changeset
     9
Fixedpt = domrange +
3923
c257b82a1200 global;
wenzelm
parents: 2469
diff changeset
    10
c257b82a1200 global;
wenzelm
parents: 2469
diff changeset
    11
global
c257b82a1200 global;
wenzelm
parents: 2469
diff changeset
    12
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    13
consts
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 753
diff changeset
    14
  bnd_mono    :: [i,i=>i]=>o
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 753
diff changeset
    15
  lfp, gfp    :: [i,i=>i]=>i
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    16
3940
wenzelm
parents: 3923
diff changeset
    17
local
3923
c257b82a1200 global;
wenzelm
parents: 2469
diff changeset
    18
753
ec86863e87c8 replaced "rules" by "defs"
lcp
parents: 124
diff changeset
    19
defs
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    20
  (*monotone operator from Pow(D) to itself*)
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    21
  bnd_mono_def 
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    22
      "bnd_mono(D,h) == h(D)<=D & (ALL W X. W<=X --> X<=D --> h(W) <= h(X))"
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    23
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    24
  lfp_def     "lfp(D,h) == Inter({X: Pow(D). h(X) <= X})"
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    25
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    26
  gfp_def     "gfp(D,h) == Union({X: Pow(D). X <= h(X)})"
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    27
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    28
end