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

Commit

Permalink
feat(order/upper_lower/locally_finite): Upper closure preserves finit…
Browse files Browse the repository at this point in the history
…eness (#18678)

`locally_finite_order` and `upper_set` don't naturally impot one another, so I'm dumping those two lemmas in a new file.
  • Loading branch information
YaelDillies committed Mar 28, 2023
1 parent 6876fa1 commit 3e17545
Showing 1 changed file with 26 additions and 0 deletions.
26 changes: 26 additions & 0 deletions src/order/upper_lower/locally_finite.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,26 @@
/-
Copyright (c) 2023 Yaël Dillies, Sara Rousta. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import order.locally_finite
import order.upper_lower.basic

/-!
# Upper and lower sets in a locally finite order
In this file we characterise the interaction of `upper_set`/`lower_set` and `locally_finite_order`.
-/

namespace set
variables {α : Type*} [preorder α] {s : set α}

protected lemma finite.upper_closure [locally_finite_order_top α] (hs : s.finite) :
(upper_closure s : set α).finite :=
by { rw coe_upper_closure, exact hs.bUnion (λ _ _, finite_Ici _) }

protected lemma finite.lower_closure [locally_finite_order_bot α] (hs : s.finite) :
(lower_closure s : set α).finite :=
by { rw coe_lower_closure, exact hs.bUnion (λ _ _, finite_Iic _) }

end set

0 comments on commit 3e17545

Please sign in to comment.