src/HOLCF/Porder0.thy
changeset 2291 fbd14a05fb88
parent 2278 d63ffafce255
child 2394 91d8abf108be
equal deleted inserted replaced
2290:e5c08f8b483b 2291:fbd14a05fb88
    38 (* instance of << for the prototype void *)
    38 (* instance of << for the prototype void *)
    39 
    39 
    40 inst_void_po    "((op <<)::[void,void]=>bool) = less_void"
    40 inst_void_po    "((op <<)::[void,void]=>bool) = less_void"
    41 
    41 
    42 (* start 8bit 1 *)
    42 (* start 8bit 1 *)
    43 syntax
       
    44 	"Ý"	::	"['a,'a::po] => bool"	(infixl 55)
       
    45 
       
    46 translations
       
    47   "x Ý y"	== "x << y"
       
    48 
       
    49 (* end 8bit 1 *)
    43 (* end 8bit 1 *)
    50 
    44 
    51 end 
    45 end 
    52 
    46 
    53 
    47