| author | paulson |
| Sun, 23 Jun 2002 10:14:13 +0200 | |
| changeset 13240 | bb5f4faea1f3 |
| parent 12030 | 46d57d0290a2 |
| child 14981 | e73f8140af78 |
| permissions | -rw-r--r-- |
(* Title: HOLCF/Up3.thy ID: $Id$ Author: Franz Regensburger License: GPL (GNU GENERAL PUBLIC LICENSE) Class instance of ('a)u for class pcpo *) Up3 = Up2 + instance u :: (pcpo)pcpo (least_up,cpo_up) constdefs up :: "'a -> ('a)u" "up == (LAM x. Iup(x))" fup :: "('a->'c)-> ('a)u -> 'c" "fup == (LAM f p. Ifup(f)(p))" translations "case l of up$x => t1" == "fup$(LAM x. t1)$l" end