src/HOL/Lattices.thy
changeset 67727 ce3e87a51488
parent 67399 eab6ce8368fa
child 69593 3dda49e08b9d
--- a/src/HOL/Lattices.thy	Sun Feb 25 20:05:05 2018 +0100
+++ b/src/HOL/Lattices.thy	Mon Feb 26 07:34:05 2018 +0100
@@ -757,6 +757,11 @@
 
 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)