diff -r a4b47c684445 -r 8d56461f85ec src/HOL/Orderings.thy --- a/src/HOL/Orderings.thy Sat Jun 25 13:21:27 2022 +0200 +++ b/src/HOL/Orderings.thy Sat Jun 25 13:34:41 2022 +0200 @@ -1058,36 +1058,6 @@ *) -subsection \Monotonicity\ - -context order -begin - -definition antimono :: "('a \ 'b::order) \ bool" where - "antimono f \ (\x y. x \ y \ f x \ f y)" - -lemma antimonoI [intro?]: - fixes f :: "'a \ 'b::order" - shows "(\x y. x \ y \ f x \ f y) \ antimono f" - unfolding antimono_def by iprover - -lemma antimonoD [dest?]: - fixes f :: "'a \ 'b::order" - shows "antimono f \ x \ y \ f x \ f y" - unfolding antimono_def by iprover - -lemma antimonoE: - fixes f :: "'a \ 'b::order" - assumes "antimono f" - assumes "x \ y" - obtains "f x \ f y" -proof - from assms show "f x \ f y" by (simp add: antimono_def) -qed - -end - - subsection \min and max -- fundamental\ definition (in ord) min :: "'a \ 'a \ 'a" where