src/HOLCF/Cprod2.thy
author wenzelm
Wed, 14 Nov 2001 23:16:05 +0100
changeset 12186 9b7026a0b0ed
parent 12030 46d57d0290a2
child 14981 e73f8140af78
permissions -rw-r--r--
added Induct/Binary_Trees.thy, Induct/Datatypes.thy; removed ex/Data.ML ex/Data.thy ex/Enum.ML ex/Enum.thy;

(*  Title:      HOLCF/Cprod2.thy
    ID:         $Id$
    Author:     Franz Regensburger
    License:    GPL (GNU GENERAL PUBLIC LICENSE)

Class Instance *::(pcpo,pcpo)po

*)

Cprod2 = Cprod1 + 

default pcpo

instance "*"::(cpo,cpo)po 
	(refl_less_cprod,antisym_less_cprod,trans_less_cprod)
end