src/HOL/Product_Type.thy
changeset 35427 ad039d29e01c
parent 35365 2fcd08c62495
child 35822 67e4de90d2c2
child 35828 46cfc4b8112e
--- a/src/HOL/Product_Type.thy	Tue Mar 02 23:56:13 2010 +0100
+++ b/src/HOL/Product_Type.thy	Tue Mar 02 23:59:54 2010 +0100
@@ -142,10 +142,10 @@
     by rule+
 qed
 
-syntax (xsymbols)
-  "*"      :: "[type, type] => type"         ("(_ \<times>/ _)" [21, 20] 20)
-syntax (HTML output)
-  "*"      :: "[type, type] => type"         ("(_ \<times>/ _)" [21, 20] 20)
+type_notation (xsymbols)
+  "*"  ("(_ \<times>/ _)" [21, 20] 20)
+type_notation (HTML output)
+  "*"  ("(_ \<times>/ _)" [21, 20] 20)
 
 consts
   Pair     :: "'a \<Rightarrow> 'b \<Rightarrow> 'a \<times> 'b"