src/HOL/Complete_Lattices.thy
changeset 57448 159e45728ceb
parent 57197 4cf607675df8
child 58889 5b7a9633cfa8
--- a/src/HOL/Complete_Lattices.thy	Mon Jun 30 15:45:21 2014 +0200
+++ b/src/HOL/Complete_Lattices.thy	Mon Jun 30 15:45:25 2014 +0200
@@ -415,6 +415,15 @@
   then show ?thesis by simp
 qed
 
+lemma INF_inf_const1:
+  "I \<noteq> {} \<Longrightarrow> (INF i:I. inf x (f i)) = inf x (INF i:I. f i)"
+  by (intro antisym INF_greatest inf_mono order_refl INF_lower)
+     (auto intro: INF_lower2 le_infI2 intro!: INF_mono)
+
+lemma INF_inf_const2:
+  "I \<noteq> {} \<Longrightarrow> (INF i:I. inf (f i) x) = inf (INF i:I. f i) x"
+  using INF_inf_const1[of I x f] by (simp add: inf_commute)
+
 lemma INF_constant:
   "(\<Sqinter>y\<in>A. c) = (if A = {} then \<top> else c)"
   by simp