src/HOLCF/Sprod1.thy
changeset 243 c22b85994e17
child 1150 66512c9e6bd6
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOLCF/Sprod1.thy	Wed Jan 19 17:35:01 1994 +0100
@@ -0,0 +1,22 @@
+(*  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"	
+
+rules
+
+  less_sprod_def "less_sprod(p1,p2) == @z.\
+\	 ( p1=Ispair(UU,UU) --> z = True)\
+\	&(~p1=Ispair(UU,UU) --> z = (   Isfst(p1) << Isfst(p2) &\
+\					Issnd(p1) << Issnd(p2)))"
+
+end
+