equal
deleted
inserted
replaced
191 by (auto intro!: antisym Inf_lower) |
191 by (auto intro!: antisym Inf_lower) |
192 |
192 |
193 lemma Sup_UNIV [simp]: "\<Squnion>UNIV = \<top>" |
193 lemma Sup_UNIV [simp]: "\<Squnion>UNIV = \<top>" |
194 by (auto intro!: antisym Sup_upper) |
194 by (auto intro!: antisym Sup_upper) |
195 |
195 |
196 lemma Inf_Sup: "\<Sqinter>A = \<Squnion>{b. \<forall>a \<in> A. b \<le> a}" |
196 lemma Inf_eq_Sup: "\<Sqinter>A = \<Squnion>{b. \<forall>a \<in> A. b \<le> a}" |
197 by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least) |
197 by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least) |
198 |
198 |
199 lemma Sup_Inf: "\<Squnion>A = \<Sqinter>{b. \<forall>a \<in> A. a \<le> b}" |
199 lemma Sup_eq_Inf: "\<Squnion>A = \<Sqinter>{b. \<forall>a \<in> A. a \<le> b}" |
200 by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least) |
200 by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least) |
201 |
201 |
202 lemma Inf_superset_mono: "B \<subseteq> A \<Longrightarrow> \<Sqinter>A \<le> \<Sqinter>B" |
202 lemma Inf_superset_mono: "B \<subseteq> A \<Longrightarrow> \<Sqinter>A \<le> \<Sqinter>B" |
203 by (auto intro: Inf_greatest Inf_lower) |
203 by (auto intro: Inf_greatest Inf_lower) |
204 |
204 |