diff -r 286c1741285c -r e89cfc004f18 src/Doc/Locales/Examples3.thy --- a/src/Doc/Locales/Examples3.thy Wed Nov 18 17:37:00 2015 +0000 +++ b/src/Doc/Locales/Examples3.thy Wed Nov 18 21:18:33 2015 +0100 @@ -223,15 +223,13 @@ \hspace*{1em}@{thm [source] le'.less_le_trans}: @{thm [display, indent=4] le'.less_le_trans} - While there is infix syntax for the strict operation associated to + While there is infix syntax for the strict operation associated with @{term "op \"}, there is none for the strict version of @{term - "op \"}. The abbreviation @{text less} with its infix syntax is only + "op \"}. The syntax @{text "\"} for @{text less} is only available for the original instance it was declared for. We may - introduce the abbreviation @{text less'} with infix syntax~@{text \} - with the following declaration:\ + introduce infix syntax for @{text le'.less} with the following declaration:\ - abbreviation (in order_preserving) - less' (infixl "\" 50) where "less' \ partial_order.less le'" + 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}: @@ -306,8 +304,8 @@ context lattice_hom begin - abbreviation meet' (infixl "\''" 50) where "meet' \ le'.meet" - abbreviation join' (infixl "\''" 50) where "join' \ le'.join" + notation le'.meet (infixl "\''" 50) + notation le'.join (infixl "\''" 50) end text \The next example makes radical use of the short hand