src/HOLCF/Cprod3.thy
changeset 625 119391dd1d59
parent 442 13ac1fd0a14d
child 752 b89462f9d5f1
--- a/src/HOLCF/Cprod3.thy	Tue Oct 04 13:02:16 1994 +0100
+++ b/src/HOLCF/Cprod3.thy	Thu Oct 06 18:40:18 1994 +0100
@@ -20,6 +20,8 @@
 	csnd         :: "('a*'b)->'b"
 	csplit       :: "('a->'b->'c)->('a*'b)->'c"
 
+translations "x#y" => "cpair[x][y]"
+
 rules 
 
 inst_cprod_pcpo	"(UU::'a*'b) = <UU,UU>"
@@ -31,13 +33,6 @@
 
 end
 
-ML
-
-(* ----------------------------------------------------------------------*)
-(* parse translations for the above mixfix                               *)
-(* ----------------------------------------------------------------------*)
-
-val parse_translation = [("@cpair",mk_cinfixtr "@cpair")];