Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit c034b4c

Browse files
committed
chore(order/bounds): +2 lemmas, fix a name (#2877)
1 parent 9d76ac2 commit c034b4c

File tree

1 file changed

+5
-1
lines changed

1 file changed

+5
-1
lines changed

src/order/bounds.lean

Lines changed: 5 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -53,6 +53,10 @@ def is_lub (s : set α) : α → Prop := is_least (upper_bounds s)
5353
/-- `a` is a greatest lower bound of a set `s`; for a partial order, it is unique if exists. -/
5454
def is_glb (s : set α) : α → Prop := is_greatest (lower_bounds s)
5555

56+
lemma mem_upper_bounds : a ∈ upper_bounds s ↔ ∀ x ∈ s, x ≤ a := iff.rfl
57+
58+
lemma mem_lower_bounds : a ∈ lower_bounds s ↔ ∀ x ∈ s, a ≤ x := iff.rfl
59+
5660
/-!
5761
### Monotonicity
5862
-/
@@ -627,7 +631,7 @@ lemma is_lub_image_le (Ha : is_lub s a) {b : β} (Hb : is_lub (f '' s) b) :
627631
b ≤ f a :=
628632
Hb.2 (Hf.mem_upper_bounds_image Ha.1)
629633

630-
lemma le_is_glb_image_le (Ha : is_glb s a) {b : β} (Hb : is_glb (f '' s) b) :
634+
lemma le_is_glb_image (Ha : is_glb s a) {b : β} (Hb : is_glb (f '' s) b) :
631635
f a ≤ b :=
632636
Hb.2 (Hf.mem_lower_bounds_image Ha.1)
633637

0 commit comments

Comments
 (0)