Skip to content

Commit

Permalink
feat(order/upper_lower): Iic is not bounded below (#16425)
Browse files Browse the repository at this point in the history
Nonempty lower sets are not bounded below in a `no_min_order`, and dual.
  • Loading branch information
YaelDillies committed Sep 8, 2022
1 parent d2d6652 commit ba346d8
Showing 1 changed file with 30 additions and 0 deletions.
30 changes: 30 additions & 0 deletions src/order/upper_lower.lean
Original file line number Diff line number Diff line change
Expand Up @@ -185,6 +185,36 @@ lemma is_lower_set.not_bot_mem (hs : is_lower_set s) : ⊥ ∉ s ↔ s = ∅ :=
hs.bot_mem.not.trans not_nonempty_iff_eq_empty

end order_bot

section no_max_order
variables [no_max_order α] (a)

lemma is_upper_set.not_bdd_above (hs : is_upper_set s) : s.nonempty → ¬ bdd_above s :=
begin
rintro ⟨a, ha⟩ ⟨b, hb⟩,
obtain ⟨c, hc⟩ := exists_gt b,
exact hc.not_le (hb $ hs ((hb ha).trans hc.le) ha),
end

lemma not_bdd_above_Ici : ¬ bdd_above (Ici a) := (is_upper_set_Ici _).not_bdd_above nonempty_Ici
lemma not_bdd_above_Ioi : ¬ bdd_above (Ioi a) := (is_upper_set_Ioi _).not_bdd_above nonempty_Ioi

end no_max_order

section no_min_order
variables [no_min_order α] (a)

lemma is_lower_set.not_bdd_below (hs : is_lower_set s) : s.nonempty → ¬ bdd_below s :=
begin
rintro ⟨a, ha⟩ ⟨b, hb⟩,
obtain ⟨c, hc⟩ := exists_lt b,
exact hc.not_le (hb $ hs (hc.le.trans $ hb ha) ha),
end

lemma not_bdd_below_Iic : ¬ bdd_below (Iic a) := (is_lower_set_Iic _).not_bdd_below nonempty_Iic
lemma not_bdd_below_Iio : ¬ bdd_below (Iio a) := (is_lower_set_Iio _).not_bdd_below nonempty_Iio

end no_min_order
end preorder

/-! ### Bundled upper/lower sets -/
Expand Down

0 comments on commit ba346d8

Please sign in to comment.