renamed because of duplicateion to avoid very long qualified names
authornipkow
Sun, 27 Oct 2019 14:54:07 +0100
changeset 70949 581083959358
parent 70948 5ed8c7e826a2
child 70950 7378fa1d0892
renamed because of duplicateion to avoid very long qualified names
src/HOL/Complete_Lattices.thy
--- a/src/HOL/Complete_Lattices.thy	Sat Oct 26 19:39:16 2019 +0200
+++ b/src/HOL/Complete_Lattices.thy	Sun Oct 27 14:54:07 2019 +0100
@@ -193,10 +193,10 @@
 lemma Sup_UNIV [simp]: "\<Squnion>UNIV = \<top>"
   by (auto intro!: antisym Sup_upper)
 
-lemma Inf_Sup: "\<Sqinter>A = \<Squnion>{b. \<forall>a \<in> A. b \<le> a}"
+lemma Inf_eq_Sup: "\<Sqinter>A = \<Squnion>{b. \<forall>a \<in> A. b \<le> a}"
   by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least)
 
-lemma Sup_Inf:  "\<Squnion>A = \<Sqinter>{b. \<forall>a \<in> A. a \<le> b}"
+lemma Sup_eq_Inf:  "\<Squnion>A = \<Sqinter>{b. \<forall>a \<in> A. a \<le> b}"
   by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least)
 
 lemma Inf_superset_mono: "B \<subseteq> A \<Longrightarrow> \<Sqinter>A \<le> \<Sqinter>B"