src/HOLCF/Sprod1.thy
author clasohm
Tue, 24 Oct 1995 13:40:06 +0100
changeset 1289 2edd7a39d92a
parent 1168 74be52691d62
child 1479 21eb5e156d91
permissions -rw-r--r--
added "execute"

(*  Title: 	HOLCF/sprod1.thy
    ID:         $Id$
    Author: 	Franz Regensburger
    Copyright   1993  Technische Universitaet Muenchen

Partial ordering for the strict product
*)

Sprod1 = Sprod0 +

consts
  less_sprod	:: "[('a ** 'b),('a ** 'b)] => bool"	

defs
  less_sprod_def "less_sprod p1 p2 == 
	if p1 = Ispair UU UU
		then True
		else Isfst p1 << Isfst p2 & Issnd p1 << Issnd p2"

end