| author | sandnerr |
| Mon, 09 Dec 1996 19:11:11 +0100 | |
| changeset 2354 | b4a1e3306aa0 |
| parent 1479 | 21eb5e156d91 |
| child 2640 | ee4dfce170a0 |
| permissions | -rw-r--r-- |
(* Title: HOLCF/cfun2.thy ID: $Id$ Author: Franz Regensburger Copyright 1993 Technische Universitaet Muenchen Class Instance ->::(pcpo,pcpo)po *) Cfun2 = Cfun1 + (* Witness for the above arity axiom is cfun1.ML *) arities "->" :: (pcpo,pcpo)po consts UU_cfun :: "'a->'b" rules (* instance of << for type ['a -> 'b] *) inst_cfun_po "((op <<)::['a->'b,'a->'b]=>bool) = less_cfun" defs (* The least element in type 'a->'b *) UU_cfun_def "UU_cfun == fabs(% x.UU)" end