src/HOL/Sum.thy
changeset 9311 ab5b24cbaa16
parent 7293 959e060f4a2f
--- a/src/HOL/Sum.thy	Thu Jul 13 23:09:03 2000 +0200
+++ b/src/HOL/Sum.thy	Thu Jul 13 23:09:25 2000 +0200
@@ -31,7 +31,7 @@
   Inr            :: "'b => 'a + 'b"
 
   (*disjoint sum for sets; the operator + is overloaded with wrong type!*)
-  Plus          :: "['a set, 'b set] => ('a + 'b) set"        (infixr 65)
+  Plus          :: "['a set, 'b set] => ('a + 'b) set"        (infixr "<+>" 65)
   Part          :: ['a set, 'b => 'a] => 'a set
 
 local
@@ -40,7 +40,7 @@
   Inl_def       "Inl == (%a. Abs_Sum(Inl_Rep(a)))"
   Inr_def       "Inr == (%b. Abs_Sum(Inr_Rep(b)))"
 
-  sum_def       "A Plus B == (Inl``A) Un (Inr``B)"
+  sum_def       "A <+> B == (Inl``A) Un (Inr``B)"
 
   (*for selecting out the components of a mutually recursive definition*)
   Part_def      "Part A h == A Int {x. ? z. x = h(z)}"