| author | wenzelm |
| Thu, 06 Feb 1997 18:22:21 +0100 | |
| changeset 2588 | b472d703fa06 |
| parent 2394 | 91d8abf108be |
| child 2640 | ee4dfce170a0 |
| permissions | -rw-r--r-- |
(* Title: HOLCF/Up3.thy ID: $Id$ Author: Franz Regensburger Copyright 1993 Technische Universitaet Muenchen Class instance of ('a)u for class pcpo *) Up3 = Up2 + arities "u" :: (pcpo)pcpo (* Witness up2.ML *) consts up :: "'a -> ('a)u" fup :: "('a->'c)-> ('a)u -> 'c" rules inst_up_pcpo "(UU::('a)u) = UU_up" defs up_def "up == (LAM x.Iup(x))" fup_def "fup == (LAM f p.Ifup(f)(p))" translations "case l of up`x => t1" == "fup`(LAM x.t1)`l" end