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

Commit efe794c

Browse files
committed
chore(order/filter): turn tendsto_id' into an iff lemma (#14791)
1 parent 6cefaf4 commit efe794c

File tree

6 files changed

+11
-15
lines changed

6 files changed

+11
-15
lines changed

src/dynamics/omega_limit.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -68,7 +68,7 @@ begin
6868
end
6969

7070
lemma omega_limit_mono_left {f₁ f₂ : filter τ} (hf : f₁ ≤ f₂) : ω f₁ ϕ s ⊆ ω f₂ ϕ s :=
71-
omega_limit_subset_of_tendsto ϕ s (tendsto_id' hf)
71+
omega_limit_subset_of_tendsto ϕ s (tendsto_id'.2 hf)
7272

7373
lemma omega_limit_mono_right {s₁ s₂ : set α} (hs : s₁ ⊆ s₂) : ω f ϕ s₁ ⊆ ω f ϕ s₂ :=
7474
Inter₂_mono $ λ u hu, closure_mono (image2_subset subset.rfl hs)

src/measure_theory/measure/haar_lebesgue.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -445,7 +445,7 @@ begin
445445
have A : tendsto (λ (r : ℝ), ennreal.of_real (r ^ (finrank ℝ E)) * μ (closed_ball (0 : E) 1))
446446
(𝓝[<] 1) (𝓝 (ennreal.of_real (1 ^ (finrank ℝ E)) * μ (closed_ball (0 : E) 1))),
447447
{ refine ennreal.tendsto.mul _ (by simp) tendsto_const_nhds (by simp),
448-
exact ennreal.tendsto_of_real ((tendsto_id' nhds_within_le_nhds).pow _) },
448+
exact ennreal.tendsto_of_real ((tendsto_id'.2 nhds_within_le_nhds).pow _) },
449449
simp only [one_pow, one_mul, ennreal.of_real_one] at A,
450450
refine le_of_tendsto A _,
451451
refine mem_nhds_within_Iio_iff_exists_Ioo_subset.2 ⟨(0 : ℝ), by simp, λ r hr, _⟩,

src/order/filter/basic.lean

Lines changed: 3 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -2320,16 +2320,13 @@ theorem tendsto.congr {f₁ f₂ : α → β} {l₁ : filter α} {l₂ : filter
23202320
(h : ∀ x, f₁ x = f₂ x) : tendsto f₁ l₁ l₂ → tendsto f₂ l₁ l₂ :=
23212321
(tendsto_congr h).1
23222322

2323-
lemma tendsto_id' {x y : filter α} : x ≤ y → tendsto id x y :=
2324-
by simp only [tendsto, map_id, forall_true_iff] {contextual := tt}
2323+
lemma tendsto_id' {x y : filter α} : tendsto id x y ↔ x ≤ y := iff.rfl
23252324

2326-
lemma tendsto_id {x : filter α} : tendsto id x x := tendsto_id' $ le_refl x
2325+
lemma tendsto_id {x : filter α} : tendsto id x x := le_refl x
23272326

23282327
lemma tendsto.comp {f : α → β} {g : β → γ} {x : filter α} {y : filter β} {z : filter γ}
23292328
(hg : tendsto g y z) (hf : tendsto f x y) : tendsto (g ∘ f) x z :=
2330-
calc map (g ∘ f) x = map g (map f x) : by rw [map_map]
2331-
... ≤ map g y : map_mono hf
2332-
... ≤ z : hg
2329+
λ s hs, hf (hg hs)
23332330

23342331
lemma tendsto.mono_left {f : α → β} {x y : filter α} {z : filter β}
23352332
(hx : tendsto f x z) (h : y ≤ x) : tendsto f y z :=

src/topology/instances/ennreal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -614,7 +614,7 @@ have Inf ((λb, ↑r - b) '' range b) = ↑r - (⨆i, b i),
614614
from is_glb.Inf_eq $ is_lub_supr.is_glb_of_tendsto
615615
(assume x _ y _, tsub_le_tsub (le_refl (r : ℝ≥0∞)))
616616
(range_nonempty _)
617-
(ennreal.tendsto_coe_sub.comp (tendsto_id' inf_le_left)),
617+
(ennreal.tendsto_coe_sub.comp (tendsto_id'.2 inf_le_left)),
618618
by rw [eq, ←this]; simp [Inf_image, infi_range, -mem_range]; exact le_rfl
619619

620620
lemma exists_countable_dense_no_zero_top :

src/topology/order.lean

Lines changed: 4 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -725,12 +725,11 @@ continuous_iff_le_induced.2 $ bot_le
725725
@[continuity] lemma continuous_top {t : tspace α} : cont t ⊤ f :=
726726
continuous_iff_coinduced_le.2 $ le_top
727727

728+
lemma continuous_id_iff_le {t t' : tspace α} : cont t t' id ↔ t ≤ t' :=
729+
@continuous_def _ _ t t' id
730+
728731
lemma continuous_id_of_le {t t' : tspace α} (h : t ≤ t') : cont t t' id :=
729-
begin
730-
rw continuous_def,
731-
assume u hu,
732-
exact h u hu
733-
end
732+
continuous_id_iff_le.2 h
734733

735734
/- 𝓝 in the induced topology -/
736735

src/topology/separation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -587,7 +587,7 @@ lemma eq_of_tendsto_nhds [topological_space β] [t1_space β] {f : α → β} {a
587587
(h : tendsto f (𝓝 a) (𝓝 b)) : f a = b :=
588588
by_contra $ assume (hfa : f a ≠ b),
589589
have fact₁ : {f a}ᶜ ∈ 𝓝 b := compl_singleton_mem_nhds hfa.symm,
590-
have fact₂ : tendsto f (pure a) (𝓝 b) := h.comp (tendsto_id' $ pure_le_nhds a),
590+
have fact₂ : tendsto f (pure a) (𝓝 b) := h.comp (tendsto_id'.2 $ pure_le_nhds a),
591591
fact₂ fact₁ (eq.refl $ f a)
592592

593593
/-- To prove a function to a `t1_space` is continuous at some point `a`, it suffices to prove that

0 commit comments

Comments
 (0)