src/HOL/Product_Type.thy
changeset 18963 3adfc9dfb30a
parent 18757 f0d901bc0686
child 19008 14c1b2f5dda4
--- a/src/HOL/Product_Type.thy	Mon Feb 06 21:02:01 2006 +0100
+++ b/src/HOL/Product_Type.thy	Tue Feb 07 08:47:43 2006 +0100
@@ -787,12 +787,12 @@
 
 code_primconst fst
 ml {*
-fun fst (x, y) = x;
+fun `_` (x, y) = x;
 *}
 
 code_primconst snd
 ml {*
-fun snd (x, y) = y;
+fun `_` (x, y) = y;
 *}
 
 code_syntax_tyco