Skip to content

Commit 2bfa3eb

Browse files
committed
Merge branch 'nightly-testing' of github.com:leanprover-community/mathlib4 into nightly-testing
2 parents d05784f + 4d73e85 commit 2bfa3eb

File tree

1 file changed

+18
-0
lines changed

1 file changed

+18
-0
lines changed

Mathlib/Topology/Constructions.lean

Lines changed: 18 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -564,6 +564,18 @@ theorem Filter.Eventually.prod_nhds {p : X → Prop} {q : Y → Prop} {x : X} {y
564564
(hx : ∀ᶠ x in 𝓝 x, p x) (hy : ∀ᶠ y in 𝓝 y, q y) : ∀ᶠ z : X × Y in 𝓝 (x, y), p z.1 ∧ q z.2 :=
565565
prod_mem_nhds hx hy
566566

567+
theorem Filter.EventuallyEq.prodMap_nhds {α β : Type*} {f₁ f₂ : X → α} {g₁ g₂ : Y → β}
568+
{x : X} {y : Y} (hf : f₁ =ᶠ[𝓝 x] f₂) (hg : g₁ =ᶠ[𝓝 y] g₂) :
569+
Prod.map f₁ g₁ =ᶠ[𝓝 (x, y)] Prod.map f₂ g₂ := by
570+
rw [nhds_prod_eq]
571+
exact hf.prod_map hg
572+
573+
theorem Filter.EventuallyLE.prodMap_nhds {α β : Type*} [LE α] [LE β] {f₁ f₂ : X → α} {g₁ g₂ : Y → β}
574+
{x : X} {y : Y} (hf : f₁ ≤ᶠ[𝓝 x] f₂) (hg : g₁ ≤ᶠ[𝓝 y] g₂) :
575+
Prod.map f₁ g₁ ≤ᶠ[𝓝 (x, y)] Prod.map f₂ g₂ := by
576+
rw [nhds_prod_eq]
577+
exact hf.prod_map hg
578+
567579
theorem nhds_swap (x : X) (y : Y) : 𝓝 (x, y) = (𝓝 (y, x)).map Prod.swap := by
568580
rw [nhds_prod_eq, Filter.prod_comm, nhds_prod_eq]; rfl
569581

@@ -572,6 +584,12 @@ theorem Filter.Tendsto.prod_mk_nhds {γ} {x : X} {y : Y} {f : Filter γ} {mx :
572584
Tendsto (fun c => (mx c, my c)) f (𝓝 (x, y)) := by
573585
rw [nhds_prod_eq]; exact Filter.Tendsto.prod_mk hx hy
574586

587+
theorem Filter.Tendsto.prodMap_nhds {x : X} {y : Y} {z : Z} {w : W} {f : X → Y} {g : Z → W}
588+
(hf : Tendsto f (𝓝 x) (𝓝 y)) (hg : Tendsto g (𝓝 z) (𝓝 w)) :
589+
Tendsto (Prod.map f g) (𝓝 (x, z)) (𝓝 (y, w)) := by
590+
rw [nhds_prod_eq, nhds_prod_eq]
591+
exact hf.prod_map hg
592+
575593
theorem Filter.Eventually.curry_nhds {p : X × Y → Prop} {x : X} {y : Y}
576594
(h : ∀ᶠ x in 𝓝 (x, y), p x) : ∀ᶠ x' in 𝓝 x, ∀ᶠ y' in 𝓝 y, p (x', y') := by
577595
rw [nhds_prod_eq] at h

0 commit comments

Comments
 (0)