src/HOL/HOLCF/Sprod.thy
changeset 61998 b66d2ca1f907
parent 61378 3e04c9ca001a
child 62175 8ffc4d0e652d
--- a/src/HOL/HOLCF/Sprod.thy	Wed Dec 30 21:10:19 2015 +0100
+++ b/src/HOL/HOLCF/Sprod.thy	Wed Dec 30 21:23:38 2015 +0100
@@ -15,14 +15,14 @@
 
 definition "sprod = {p::'a \<times> 'b. p = \<bottom> \<or> (fst p \<noteq> \<bottom> \<and> snd p \<noteq> \<bottom>)}"
 
-pcpodef ('a, 'b) sprod (infixr "**" 20) = "sprod :: ('a \<times> 'b) set"
+pcpodef ('a, 'b) sprod  ("(_ \<otimes>/ _)" [21,20] 20) = "sprod :: ('a \<times> 'b) set"
   unfolding sprod_def by simp_all
 
 instance sprod :: ("{chfin,pcpo}", "{chfin,pcpo}") chfin
 by (rule typedef_chfin [OF type_definition_sprod below_sprod_def])
 
-type_notation (xsymbols)
-  sprod  ("(_ \<otimes>/ _)" [21,20] 20)
+type_notation (ASCII)
+  sprod  (infixr "**" 20)
 
 
 subsection {* Definitions of constants *}