diff -r 6d4fb57eb66c -r a4b47c684445 src/Doc/Main/Main_Doc.thy --- a/src/Doc/Main/Main_Doc.thy Tue Jul 05 09:44:38 2022 +0200 +++ b/src/Doc/Main/Main_Doc.thy Sat Jun 25 13:21:27 2022 +0200 @@ -58,8 +58,6 @@ \<^const>\Orderings.max\ & \<^typeof>\Orderings.max\\\ @{const[source] top} & \<^typeof>\Orderings.top\\\ @{const[source] bot} & \<^typeof>\Orderings.bot\\\ -\<^const>\Orderings.mono\ & \<^typeof>\Orderings.mono\\\ -\<^const>\Orderings.strict_mono\ & \<^typeof>\Orderings.strict_mono\\\ \end{tabular} \subsubsection*{Syntax} @@ -152,6 +150,12 @@ \<^const>\Fun.surj\ & \<^typeof>\Fun.surj\\\ \<^const>\Fun.bij\ & \<^typeof>\Fun.bij\\\ \<^const>\Fun.bij_betw\ & @{term_type_only Fun.bij_betw "('a\'b)\'a set\'b set\bool"}\\ +\<^const>\Fun.monotone_on\ & \<^typeof>\Fun.monotone_on\\\ +\<^const>\Fun.monotone\ & \<^typeof>\Fun.monotone\\\ +\<^const>\Fun.mono_on\ & \<^typeof>\Fun.mono_on\\\ +\<^const>\Fun.mono\ & \<^typeof>\Fun.mono\\\ +\<^const>\Fun.strict_mono_on\ & \<^typeof>\Fun.strict_mono_on\\\ +\<^const>\Fun.strict_mono\ & \<^typeof>\Fun.strict_mono\\\ \<^const>\Fun.fun_upd\ & \<^typeof>\Fun.fun_upd\\\ \end{tabular}