src/ZF/Fixedpt.thy
changeset 6093 87bf8c03b169
parent 3940 1d5bee4d047f
child 13168 afcbca3498b0
equal deleted inserted replaced
6092:d9db67970c73 6093:87bf8c03b169
     6 Least and greatest fixed points
     6 Least and greatest fixed points
     7 *)
     7 *)
     8 
     8 
     9 Fixedpt = domrange +
     9 Fixedpt = domrange +
    10 
    10 
    11 global
       
    12 
       
    13 consts
    11 consts
    14   bnd_mono    :: [i,i=>i]=>o
    12   bnd_mono    :: [i,i=>i]=>o
    15   lfp, gfp    :: [i,i=>i]=>i
    13   lfp, gfp    :: [i,i=>i]=>i
    16 
       
    17 local
       
    18 
    14 
    19 defs
    15 defs
    20   (*monotone operator from Pow(D) to itself*)
    16   (*monotone operator from Pow(D) to itself*)
    21   bnd_mono_def 
    17   bnd_mono_def 
    22       "bnd_mono(D,h) == h(D)<=D & (ALL W X. W<=X --> X<=D --> h(W) <= h(X))"
    18       "bnd_mono(D,h) == h(D)<=D & (ALL W X. W<=X --> X<=D --> h(W) <= h(X))"