src/HOL/Conditionally_Complete_Lattices.thy
changeset 54261 89991ef58448
parent 54259 71c701dc5bf9
child 54262 326fd7103cb4
--- a/src/HOL/Conditionally_Complete_Lattices.thy	Tue Nov 05 09:44:59 2013 +0100
+++ b/src/HOL/Conditionally_Complete_Lattices.thy	Tue Nov 05 09:45:00 2013 +0100
@@ -90,6 +90,12 @@
 
 end
 
+lemma (in order_top) bdd_above_top[simp, intro!]: "bdd_above A"
+  by (rule bdd_aboveI[of _ top]) simp
+
+lemma (in order_bot) bdd_above_bot[simp, intro!]: "bdd_below A"
+  by (rule bdd_belowI[of _ bot]) simp
+
 context lattice
 begin
 
@@ -270,6 +276,12 @@
 lemma cSUP_upper2: "bdd_above (f ` A) \<Longrightarrow> x \<in> A \<Longrightarrow> u \<le> f x \<Longrightarrow> u \<le> SUPR A f"
   by (auto intro: cSUP_upper assms order_trans)
 
+lemma cSUP_const: "A \<noteq> {} \<Longrightarrow> (SUP x:A. c) = c"
+  by (intro antisym cSUP_least) (auto intro: cSUP_upper)
+
+lemma cINF_const: "A \<noteq> {} \<Longrightarrow> (INF x:A. c) = c"
+  by (intro antisym cINF_greatest) (auto intro: cINF_lower)
+
 lemma le_cINF_iff: "A \<noteq> {} \<Longrightarrow> bdd_below (f ` A) \<Longrightarrow> u \<le> INFI A f \<longleftrightarrow> (\<forall>x\<in>A. u \<le> f x)"
   by (metis cINF_greatest cINF_lower assms order_trans)