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

Commit adae1ad

Browse files
committed
feat(order/filter/archimedean): in an archimedean linear ordered ring, at_top and at_bot are countably generated (#7751)
1 parent 6d85ff2 commit adae1ad

File tree

1 file changed

+39
-1
lines changed

1 file changed

+39
-1
lines changed

src/order/filter/archimedean.lean

Lines changed: 39 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,7 @@ two results for `ℤ` (and a ring `R`) and `ℚ` (and a field `R`).
1717

1818
variables {α R : Type*}
1919

20-
open filter
20+
open filter set
2121

2222
lemma tendsto_coe_nat_at_top_iff [ordered_semiring R] [nontrivial R] [archimedean R]
2323
{f : α → ℕ} {l : filter α} :
@@ -45,6 +45,44 @@ lemma tendsto_coe_rat_at_top_iff [linear_ordered_field R] [archimedean R]
4545
tendsto_at_top_embedding (assume a₁ a₂, rat.cast_le) $
4646
assume r, let ⟨n, hn⟩ := exists_nat_ge r in ⟨(n:ℚ), by assumption_mod_cast⟩
4747

48+
lemma at_top_countable_basis_of_archimedean [linear_ordered_semiring R] [archimedean R] :
49+
(at_top : filter R).has_countable_basis (λ i, i ∈ range (coe : ℕ → R)) Ici :=
50+
{ countable := countable_range coe,
51+
mem_iff' := λ t,
52+
begin
53+
rw at_top_basis.mem_iff' t,
54+
simp only [exists_prop, mem_range, exists_exists_eq_and, exists_true_left],
55+
split,
56+
{ rintro ⟨i, hi⟩,
57+
rcases exists_nat_ge i with ⟨n, hn⟩,
58+
exact ⟨n, trans (Ici_subset_Ici.mpr hn) hi⟩ },
59+
{ rintro ⟨n, hn⟩,
60+
exact ⟨n, hn⟩ }
61+
end }
62+
63+
lemma at_bot_countable_basis_of_archimedean [linear_ordered_ring R] [archimedean R] :
64+
(at_bot : filter R).has_countable_basis (λ i, i ∈ range (coe : ℤ → R)) Iic :=
65+
{ countable := countable_range coe,
66+
mem_iff' := λ t,
67+
begin
68+
rw at_bot_basis.mem_iff' t,
69+
simp only [exists_prop, mem_range, exists_exists_eq_and, exists_true_left],
70+
split,
71+
{ rintro ⟨i, hi⟩,
72+
rcases exists_int_lt i with ⟨n, hn⟩,
73+
exact ⟨n, trans (Iic_subset_Iic.mpr hn.le) hi⟩ },
74+
{ rintro ⟨n, hn⟩,
75+
exact ⟨n, hn⟩ }
76+
end }
77+
78+
lemma at_top_countably_generated_of_archimedean [linear_ordered_semiring R] [archimedean R] :
79+
(at_top : filter R).is_countably_generated :=
80+
at_top_countable_basis_of_archimedean.is_countably_generated
81+
82+
lemma at_bot_countably_generated [linear_ordered_ring R] [archimedean R] :
83+
(at_bot : filter R).is_countably_generated :=
84+
at_bot_countable_basis_of_archimedean.is_countably_generated
85+
4886
variables [linear_ordered_semiring R] [archimedean R]
4987
variables {l : filter α} {f : α → R} {r : R}
5088

0 commit comments

Comments
 (0)