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

Commit fe0f2a3

Browse files
Patrick Massotjohoelzl
authored andcommitted
fix(analysis/topology/topological_structures): remove unnecessary hypothesis
1 parent a7d8c5f commit fe0f2a3

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

analysis/topology/topological_structures.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -342,8 +342,8 @@ lemma tendsto_orderable {f : β → α} {a : α} {x : filter β} :
342342
tendsto f x (nhds a) ↔ (∀a'<a, {b | a' < f b} ∈ x.sets) ∧ (∀a'>a, {b | a' > f b} ∈ x.sets) :=
343343
by simp [@nhds_eq_orderable α _ _, tendsto_inf, tendsto_infi, tendsto_principal]
344344

345-
/-- Also known as squeez or sandwich theorem. -/
346-
lemma tendsto_of_tendsto_of_tendsto_of_le_of_le {f g h : β → α} {b : filter β} {a : α} (hb : b ≠ ⊥)
345+
/-- Also known as squeeze or sandwich theorem. -/
346+
lemma tendsto_of_tendsto_of_tendsto_of_le_of_le {f g h : β → α} {b : filter β} {a : α}
347347
(hg : tendsto g b (nhds a)) (hh : tendsto h b (nhds a))
348348
(hgf : {b | g b ≤ f b} ∈ b.sets) (hfh : {b | f b ≤ h b} ∈ b.sets) :
349349
tendsto f b (nhds a) :=

0 commit comments

Comments
 (0)