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

Commit 5193194

Browse files
committed
feat(order/filter): reorder filter theory; add filter_upwards tactic
1 parent 0487a32 commit 5193194

File tree

3 files changed

+236
-208
lines changed

3 files changed

+236
-208
lines changed

analysis/topology/topological_space.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -384,7 +384,7 @@ is_closed_iff_nhds.mp hs _ $ neq_bot_of_le_neq_bot (@map_ne_bot _ _ _ f h) $
384384
/- locally finite family [General Topology (Bourbaki, 1995)] -/
385385
section locally_finite
386386

387-
/-- A family of sets in `set α` is locally finite if at every point `x:α`,
387+
/-- A family of sets in `set α` is locally finite if at every point `x:α`,
388388
there is a neighborhood of `x` which meets only finitely many sets in the family -/
389389
def locally_finite (f : β → set α) :=
390390
∀x:α, ∃t∈(nhds x).sets, finite {i | f i ∩ t ≠ ∅ }
@@ -412,7 +412,7 @@ is_open_iff_nhds.mpr $ assume a, assume h : a ∉ (⋃i, f i),
412412
begin
413413
rw [le_principal_iff],
414414
apply @filter.inter_mem_sets _ (nhds a) _ _ h_sets,
415-
apply @filter.Inter_mem_sets _ _ (nhds a) _ _ h_fin,
415+
apply @filter.Inter_mem_sets _ (nhds a) _ _ _ h_fin,
416416
exact assume i h, this i
417417
end
418418
... ≤ principal (- ⋃i, f i) :

analysis/topology/uniform_space.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -100,7 +100,7 @@ lemma uniform_space.core_eq : ∀{u₁ u₂ : uniform_space.core α}, u₁.unifo
100100
metric space. It consists of a filter on `α × α` called the "uniformity", which
101101
satisfies properties analogous to the reflexivity, symmetry, and triangle properties
102102
of a metric.
103-
103+
104104
A metric space has a natural uniformity, and a uniform space has a natural topology.
105105
A topological group also has a natural uniformity, even when it is not metrizable. -/
106106
class uniform_space (α : Type u) extends topological_space α, uniform_space.core α :=
@@ -999,8 +999,7 @@ let ⟨s, hs, ss_t⟩ := comp_mem_uniformity_sets ht in
999999
ss_t ⟨b₂, show ((b₁, a₂).1, b₂) ∈ s, from hb, ba₂⟩⟩⟩
10001000

10011001
lemma vmap_quotient_eq_uniformity : vmap (λ (p : α × α), (⟦p.fst⟧, ⟦p.snd⟧)) uniformity = uniformity :=
1002-
le_antisymm vmap_quotient_le_uniformity
1003-
(assume s ⟨t, ht, hs⟩, uniformity.upwards_sets ht hs)
1002+
le_antisymm vmap_quotient_le_uniformity le_vmap_map
10041003

10051004
lemma complete_space_separation [h : complete_space α] :
10061005
complete_space (quotient (separation_setoid α)) :=

0 commit comments

Comments
 (0)