author | lcp |
Fri, 13 Jan 1995 02:02:00 +0100 | |
changeset 863 | 67692db44c70 |
parent 752 | b89462f9d5f1 |
child 1168 | 74be52691d62 |
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" (* definitions *) (* The least element in type 'a->'b *) UU_cfun_def "UU_cfun == fabs(% x.UU)" end