diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Complete_Partial_Order.thy --- a/src/HOL/Complete_Partial_Order.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Complete_Partial_Order.thy Fri Jan 04 23:22:53 2019 +0100 @@ -11,7 +11,7 @@ subsection \Monotone functions\ -text \Dictionary-passing version of @{const Orderings.mono}.\ +text \Dictionary-passing version of \<^const>\Orderings.mono\.\ definition monotone :: "('a \ 'a \ bool) \ ('b \ 'b \ bool) \ ('a \ 'b) \ bool" where "monotone orda ordb f \ (\x y. orda x y \ ordb (f x) (f y))"