more direct notation;
authorwenzelm
Mon, 27 May 2013 22:30:07 +0200
changeset 52191 636b62eb7e88
parent 52190 c87b7f26e2c7
child 52192 fce4a365f280
more direct notation;
src/HOL/Library/Order_Union.thy
--- a/src/HOL/Library/Order_Union.thy	Mon May 27 22:26:08 2013 +0200
+++ b/src/HOL/Library/Order_Union.thy	Mon May 27 22:30:07 2013 +0200
@@ -14,8 +14,7 @@
 definition Osum :: "'a rel \<Rightarrow> 'a rel \<Rightarrow> 'a rel"  (infix "Osum" 60) where
   "r Osum r' = r \<union> r' \<union> {(a, a'). a \<in> Field r \<and> a' \<in> Field r'}"
 
-abbreviation Osum2 :: "'a rel \<Rightarrow> 'a rel \<Rightarrow> 'a rel" (infix "\<union>o" 60) where
-  "r \<union>o r' \<equiv> r Osum r'"
+notation Osum  (infix "\<union>o" 60)
 
 lemma Field_Osum: "Field (r \<union>o r') = Field r \<union> Field r'"
   unfolding Osum_def Field_def by blast