diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Lattice/Lattice.thy --- a/src/HOL/Lattice/Lattice.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Lattice/Lattice.thy Fri Sep 20 19:51:08 2024 +0200 @@ -24,10 +24,10 @@ \ definition - meet :: "'a::lattice \ 'a \ 'a" (infixl "\" 70) where + meet :: "'a::lattice \ 'a \ 'a" (infixl \\\ 70) where "x \ y = (THE inf. is_inf x y inf)" definition - join :: "'a::lattice \ 'a \ 'a" (infixl "\" 65) where + join :: "'a::lattice \ 'a \ 'a" (infixl \\\ 65) where "x \ y = (THE sup. is_sup x y sup)" text \