diff -r 46f59511b7bb -r d97fdabd9e2b src/Doc/Locales/Examples3.thy --- a/src/Doc/Locales/Examples3.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/Doc/Locales/Examples3.thy Fri Sep 20 19:51:08 2024 +0200 @@ -204,7 +204,7 @@ locale order_preserving = le: partial_order le + le': partial_order le' - for le (infixl "\" 50) and le' (infixl "\" 50) + + for le (infixl \\\ 50) and le' (infixl \\\ 50) + fixes \ assumes hom_le: "x \ y \ \ x \ \ y" @@ -222,7 +222,7 @@ available for the original instance it was declared for. We may introduce infix syntax for \le'.less\ with the following declaration:\ - notation (in order_preserving) le'.less (infixl "\" 50) + notation (in order_preserving) le'.less (infixl \\\ 50) text (in order_preserving) \Now the theorem is displayed nicely as @{thm [source] le'.less_le_trans}: @@ -279,7 +279,7 @@ join.\ locale lattice_hom = - le: lattice + le': lattice le' for le' (infixl "\" 50) + + le: lattice + le': lattice le' for le' (infixl \\\ 50) + fixes \ assumes hom_meet: "\ (x \ y) = le'.meet (\ x) (\ y)" and hom_join: "\ (x \ y) = le'.join (\ x) (\ y)" @@ -295,8 +295,8 @@ context lattice_hom begin - notation le'.meet (infixl "\''" 50) - notation le'.join (infixl "\''" 50) + notation le'.meet (infixl \\''\ 50) + notation le'.join (infixl \\''\ 50) end text \The next example makes radical use of the short hand