Skip to content

Commit 15e555e

Browse files
hrmacbethADedecker
andcommitted
feat: characterize "eventually" in a subtype (#7568)
Co-authored-by: Anatole Dedecker <anatolededecker@gmail.com> Co-authored-by: ADedecker <anatolededecker@gmail.com>
1 parent d3a6c9f commit 15e555e

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

Mathlib/Topology/ContinuousOn.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -505,6 +505,14 @@ theorem preimage_coe_mem_nhds_subtype {s t : Set α} {a : s} : (↑) ⁻¹' t
505505
rw [← map_nhds_subtype_val, mem_map]
506506
#align preimage_coe_mem_nhds_subtype preimage_coe_mem_nhds_subtype
507507

508+
theorem eventually_nhds_subtype_if (s : Set α) (a : s) (P : α → Prop) :
509+
(∀ᶠ x : s in 𝓝 a, P x) ↔ ∀ᶠ x in 𝓝[s] a, P x :=
510+
preimage_coe_mem_nhds_subtype
511+
512+
theorem frequently_nhds_subtype_iff (s : Set α) (a : s) (P : α → Prop) :
513+
(∃ᶠ x : s in 𝓝 a, P x) ↔ ∃ᶠ x in 𝓝[s] a, P x :=
514+
eventually_nhds_subtype_if s a (¬ P ·) |>.not
515+
508516
theorem tendsto_nhdsWithin_iff_subtype {s : Set α} {a : α} (h : a ∈ s) (f : α → β) (l : Filter β) :
509517
Tendsto f (𝓝[s] a) l ↔ Tendsto (s.restrict f) (𝓝 ⟨a, h⟩) l := by
510518
rw [nhdsWithin_eq_map_subtype_coe h, tendsto_map'_iff]; rfl

0 commit comments

Comments
 (0)