src/HOL/HOLCF/Ssum.thy
changeset 81095 49c04500c5f9
parent 80914 d97fdabd9e2b
child 81583 b6df83045178
--- a/src/HOL/HOLCF/Ssum.thy	Tue Oct 01 22:12:11 2024 +0200
+++ b/src/HOL/HOLCF/Ssum.thy	Tue Oct 01 23:36:10 2024 +0200
@@ -19,7 +19,7 @@
     (fst p = TT \<and> fst (snd p) \<noteq> \<bottom> \<and> snd (snd p) = \<bottom>) \<or>
     (fst p = FF \<and> fst (snd p) = \<bottom> \<and> snd (snd p) \<noteq> \<bottom>)}"
 
-pcpodef ('a, 'b) ssum  (\<open>(_ \<oplus>/ _)\<close> [21, 20] 20) = "ssum :: (tr \<times> 'a \<times> 'b) set"
+pcpodef ('a, 'b) ssum  (\<open>(\<open>notation=\<open>infix strict sum\<close>\<close>_ \<oplus>/ _)\<close> [21, 20] 20) = "ssum :: (tr \<times> 'a \<times> 'b) set"
   by (simp_all add: ssum_def)
 
 instance ssum :: ("{chfin,pcpo}", "{chfin,pcpo}") chfin