File tree Expand file tree Collapse file tree 2 files changed +25
-0
lines changed
Topology/MetricSpace/Pseudo Expand file tree Collapse file tree 2 files changed +25
-0
lines changed Original file line number Diff line number Diff line change @@ -1281,6 +1281,13 @@ theorem eq_of_le_of_forall_ge_of_dense [LinearOrder α] [DenselyOrdered α] {a
1281
1281
(h₂ : ∀ a₃ < a₁, a₃ ≤ a₂) : a₁ = a₂ :=
1282
1282
(le_of_forall_ge_of_dense h₂).antisymm h₁
1283
1283
1284
+ theorem forall_lt_le_iff [LinearOrder α] [DenselyOrdered α] {a b : α} : (∀ c < a, c ≤ b) ↔ a ≤ b :=
1285
+ ⟨le_of_forall_ge_of_dense, fun hab _c hca ↦ hca.le.trans hab⟩
1286
+
1287
+ theorem forall_gt_ge_iff [LinearOrder α] [DenselyOrdered α] {a b : α} :
1288
+ (∀ c, a < c → b ≤ c) ↔ b ≤ a :=
1289
+ forall_lt_le_iff (α := αᵒᵈ)
1290
+
1284
1291
theorem dense_or_discrete [LinearOrder α] (a₁ a₂ : α) :
1285
1292
(∃ a, a₁ < a ∧ a < a₂) ∨ (∀ a, a₁ < a → a₂ ≤ a) ∧ ∀ a < a₂, a ≤ a₁ :=
1286
1293
or_iff_not_imp_left.2 fun h ↦
Original file line number Diff line number Diff line change @@ -89,4 +89,22 @@ lemma exists_isCompact_closedBall [WeaklyLocallyCompactSpace α] (x : α) :
89
89
eventually_nhdsWithin_of_eventually_nhds (eventually_isCompact_closedBall x)
90
90
simpa only [and_comm] using (this.and self_mem_nhdsWithin).exists
91
91
92
+ theorem biInter_gt_closedBall (x : α) (r : ℝ) : ⋂ r' > r, closedBall x r' = closedBall x r := by
93
+ ext
94
+ simp [forall_gt_ge_iff]
95
+
96
+ theorem biInter_gt_ball (x : α) (r : ℝ) : ⋂ r' > r, ball x r' = closedBall x r := by
97
+ ext
98
+ simp [forall_lt_iff_le']
99
+
100
+ theorem biUnion_lt_ball (x : α) (r : ℝ) : ⋃ r' < r, ball x r' = ball x r := by
101
+ ext
102
+ rw [← not_iff_not]
103
+ simp [forall_lt_le_iff]
104
+
105
+ theorem biUnion_lt_closedBall (x : α) (r : ℝ) : ⋃ r' < r, closedBall x r' = ball x r := by
106
+ ext
107
+ rw [← not_iff_not]
108
+ simp [forall_lt_iff_le]
109
+
92
110
end Metric
You can’t perform that action at this time.
0 commit comments