@@ -17,7 +17,7 @@ two results for `ℤ` (and a ring `R`) and `ℚ` (and a field `R`).
17
17
18
18
variables {α R : Type *}
19
19
20
- open filter
20
+ open filter set
21
21
22
22
lemma tendsto_coe_nat_at_top_iff [ordered_semiring R] [nontrivial R] [archimedean R]
23
23
{f : α → ℕ} {l : filter α} :
@@ -45,6 +45,44 @@ lemma tendsto_coe_rat_at_top_iff [linear_ordered_field R] [archimedean R]
45
45
tendsto_at_top_embedding (assume a₁ a₂, rat.cast_le) $
46
46
assume r, let ⟨n, hn⟩ := exists_nat_ge r in ⟨(n:ℚ), by assumption_mod_cast⟩
47
47
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
+
48
86
variables [linear_ordered_semiring R] [archimedean R]
49
87
variables {l : filter α} {f : α → R} {r : R}
50
88
0 commit comments