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

Commit 2a86b06

Browse files
ChrisHughes24digama0
authored andcommitted
fix(order/filter): tendsto_at_top only requires preorder not partial_order
1 parent 9e6572f commit 2a86b06

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

order/filter.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1755,7 +1755,7 @@ calc map f (⨅a, principal {a' | a ≤ a'}) = (⨅a, map f $ principal {a' | a
17551755
mem_principal_sets, and_self, sup_le_iff, forall_true_iff] {contextual := tt}⟩) ⟨default α⟩
17561756
... = (⨅a, principal $ f '' {a' | a ≤ a'}) : by simp only [map_principal, eq_self_iff_true]
17571757

1758-
lemma tendsto_at_top {α β} [partial_order β] (m : α → β) (f : filter α) :
1758+
lemma tendsto_at_top {α β} [preorder β] (m : α → β) (f : filter α) :
17591759
tendsto m f at_top ↔ (∀b, {a | b ≤ m a} ∈ f.sets) :=
17601760
by simp only [at_top, tendsto_infi, tendsto_principal]; refl
17611761

0 commit comments

Comments
 (0)