src/HOL/Lattices.thy
changeset 76055 8d56461f85ec
parent 76054 a4b47c684445
child 79099 05a753360b25
--- a/src/HOL/Lattices.thy	Sat Jun 25 13:21:27 2022 +0200
+++ b/src/HOL/Lattices.thy	Sat Jun 25 13:34:41 2022 +0200
@@ -606,11 +606,6 @@
 
 end
 
-lemma max_of_antimono: "antimono f \<Longrightarrow> max (f x) (f y) = f (min x y)"
-  and min_of_antimono: "antimono f \<Longrightarrow> min (f x) (f y) = f (max x y)"
-  for f::"'a::linorder \<Rightarrow> 'b::linorder"
-  by (auto simp: antimono_def Orderings.max_def min_def intro!: antisym)
-
 lemma inf_min: "inf = (min :: 'a::{semilattice_inf,linorder} \<Rightarrow> 'a \<Rightarrow> 'a)"
   by (auto intro: antisym simp add: min_def fun_eq_iff)