diff -r 5ed8c7e826a2 -r 581083959358 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]: "\UNIV = \" by (auto intro!: antisym Sup_upper) -lemma Inf_Sup: "\A = \{b. \a \ A. b \ a}" +lemma Inf_eq_Sup: "\A = \{b. \a \ A. b \ a}" by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least) -lemma Sup_Inf: "\A = \{b. \a \ A. a \ b}" +lemma Sup_eq_Inf: "\A = \{b. \a \ A. a \ b}" by (auto intro: antisym Inf_lower Inf_greatest Sup_upper Sup_least) lemma Inf_superset_mono: "B \ A \ \A \ \B"