src/HOL/Lattice/Lattice.thy
changeset 61983 8fb53badad99
parent 58879 143c85e3cdb5
child 61986 2461779da2b8
--- a/src/HOL/Lattice/Lattice.thy	Wed Dec 30 18:03:23 2015 +0100
+++ b/src/HOL/Lattice/Lattice.thy	Wed Dec 30 18:07:10 2015 +0100
@@ -24,15 +24,11 @@
 *}
 
 definition
-  meet :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "&&" 70) where
-  "x && y = (THE inf. is_inf x y inf)"
+  meet :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "\<sqinter>" 70) where
+  "x \<sqinter> y = (THE inf. is_inf x y inf)"
 definition
-  join :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "||" 65) where
-  "x || y = (THE sup. is_sup x y sup)"
-
-notation (xsymbols)
-  meet  (infixl "\<sqinter>" 70) and
-  join  (infixl "\<squnion>" 65)
+  join :: "'a::lattice \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "\<squnion>" 65) where
+  "x \<squnion> y = (THE sup. is_sup x y sup)"
 
 text {*
   Due to unique existence of bounds, the lattice operations may be