src/HOLCF/Sprod1.thy
changeset 3323 194ae2e0c193
parent 2640 ee4dfce170a0
child 12030 46d57d0290a2
--- a/src/HOLCF/Sprod1.thy	Fri May 23 18:55:28 1997 +0200
+++ b/src/HOLCF/Sprod1.thy	Sun May 25 11:07:52 1997 +0200
@@ -8,7 +8,9 @@
 
 Sprod1 = Sprod0 +
 
+instance "**"::(sq_ord,sq_ord)sq_ord 
+
 defs
-  less_sprod_def "less p1 p2 == Isfst p1 << Isfst p2 & Issnd p1 << Issnd p2"
+  less_sprod_def "p1 << p2 == Isfst p1 << Isfst p2 & Issnd p1 << Issnd p2"
 
 end