src/HOLCF/Pcpo.thy
author paulson
Wed, 25 Sep 1996 15:03:13 +0200
changeset 2025 9acc10ac1e1d
parent 1479 21eb5e156d91
child 2278 d63ffafce255
permissions -rw-r--r--
Prevention of Overflow exception (for SML/NJ) in gensym

Pcpo = Porder +

classes pcpo < po
arities void :: pcpo

consts  
        UU :: "'a::pcpo"        

rules

        minimal "UU << x"       
        cpo     "is_chain(S) ==> ? x. range(S) <<| (x::'a::pcpo)" 

inst_void_pcpo  "(UU::void) = UU_void"

(* start 8bit 1 *)
(* end 8bit 1 *)
end