src/HOLCF/Porder0.thy
changeset 2278 d63ffafce255
parent 1479 21eb5e156d91
child 2291 fbd14a05fb88
--- a/src/HOLCF/Porder0.thy	Fri Nov 29 12:17:30 1996 +0100
+++ b/src/HOLCF/Porder0.thy	Fri Nov 29 12:22:22 1996 +0100
@@ -40,6 +40,12 @@
 inst_void_po    "((op <<)::[void,void]=>bool) = less_void"
 
 (* start 8bit 1 *)
+syntax
+	"Ý"	::	"['a,'a::po] => bool"	(infixl 55)
+
+translations
+  "x Ý y"	== "x << y"
+
 (* end 8bit 1 *)
 
 end