Skip to content

Commit

Permalink
chore(order/filter/basic): add @[simp] to principal_empty/univ (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Jul 27, 2020
1 parent d06f62d commit d6e399f
Show file tree
Hide file tree
Showing 4 changed files with 6 additions and 7 deletions.
1 change: 0 additions & 1 deletion src/order/filter/at_top_bot.lean
Original file line number Diff line number Diff line change
Expand Up @@ -630,7 +630,6 @@ end

end is_countably_generated


end filter

open filter finset
Expand Down
6 changes: 3 additions & 3 deletions src/order/filter/bases.lean
Original file line number Diff line number Diff line change
Expand Up @@ -507,7 +507,7 @@ begin
end

lemma countable_binfi_eq_infi_seq' [complete_lattice α] {B : set ι} (Bcbl : countable B) (f : ι → α)
{i₀ : ι} (h : f i₀ = ⊤) :
{i₀ : ι} (h : f i₀ = ⊤) :
∃ (x : ℕ → ι), (⨅ t ∈ B, f t) = ⨅ i, f (x i) :=
begin
cases B.eq_empty_or_nonempty with hB Bnonempty,
Expand Down Expand Up @@ -554,7 +554,7 @@ lemma has_countable_basis {l : filter α} (h : is_countably_generated l) :
countable_set_of_finite_subset h.countable_generating_set⟩

lemma exists_countable_infi_principal {f : filter α} (h : f.is_countably_generated) :
∃ s : set (set α), countable s ∧ f = ⨅ t ∈ s, 𝓟 t :=
∃ s : set (set α), countable s ∧ f = ⨅ t ∈ s, 𝓟 t :=
begin
let B := h.countable_filter_basis,
use [B.sets, B.countable],
Expand All @@ -564,7 +564,7 @@ begin
end

lemma exists_seq {f : filter α} (cblb : f.is_countably_generated) :
∃ x : ℕ → set α, f = ⨅ i, 𝓟 (x i) :=
∃ x : ℕ → set α, f = ⨅ i, 𝓟 (x i) :=
begin
rcases cblb.exists_countable_infi_principal with ⟨B, Bcbl, rfl⟩,
exact countable_binfi_principal_eq_seq_infi Bcbl,
Expand Down
4 changes: 2 additions & 2 deletions src/order/filter/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -467,10 +467,10 @@ by simp only [le_antisymm_iff, le_principal_iff, mem_principal_sets]; refl

@[simp] lemma join_principal_eq_Sup {s : set (filter α)} : join (𝓟 s) = Sup s := rfl

lemma principal_univ : 𝓟 (univ : set α) = ⊤ :=
@[simp] lemma principal_univ : 𝓟 (univ : set α) = ⊤ :=
top_unique $ by simp only [le_principal_iff, mem_top_sets, eq_self_iff_true]

lemma principal_empty : 𝓟 (∅ : set α) = ⊥ :=
@[simp] lemma principal_empty : 𝓟 (∅ : set α) = ⊥ :=
bot_unique $ assume s _, empty_subset _

/-! ### Lattice equations -/
Expand Down
2 changes: 1 addition & 1 deletion src/topology/subset_properties.lean
Original file line number Diff line number Diff line change
Expand Up @@ -363,7 +363,7 @@ lemma compact_univ [h : compact_space α] : is_compact (univ : set α) := h.comp

lemma cluster_point_of_compact [compact_space α]
(f : filter α) [ne_bot f] : ∃ x, cluster_pt x f :=
by simpa using compact_univ (by simpa using f.univ_sets)
by simpa using compact_univ (show f ≤ 𝓟 univ, by simp)

theorem compact_space_of_finite_subfamily_closed {α : Type u} [topological_space α]
(h : Π {ι : Type u} (Z : ι → (set α)), (∀ i, is_closed (Z i)) →
Expand Down

0 comments on commit d6e399f

Please sign in to comment.