Skip to content

Commit aec06ab

Browse files
committed
chore(Topology): continuity -> fun_prop (#23136)
1 parent 88f302b commit aec06ab

File tree

7 files changed

+11
-19
lines changed

7 files changed

+11
-19
lines changed

Mathlib/Dynamics/Flow.lean

Lines changed: 2 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -153,14 +153,9 @@ def reverse : Flow τ α where
153153
map_add' _ _ _ := by dsimp; rw [neg_add, map_add]
154154
map_zero' _ := by dsimp; rw [neg_zero, map_zero_apply]
155155

156-
-- Porting note: add @continuity to Flow.toFun so that these works:
157-
-- Porting note: Homeomorphism.continuous_toFun : Continuous toFun := by continuity
158-
-- Porting note: Homeomorphism.continuous_invFun : Continuous invFun := by continuity
159-
@[continuity]
156+
@[continuity, fun_prop]
160157
theorem continuous_toFun (t : τ) : Continuous (ϕ.toFun t) := by
161-
rw [← curry_uncurry ϕ.toFun]
162-
apply continuous_curry
163-
exact ϕ.cont'
158+
fun_prop
164159

165160
/-- The map `ϕ t` as a homeomorphism. -/
166161
def toHomeomorph (t : τ) : (α ≃ₜ α) where

Mathlib/Topology/Algebra/Monoid.lean

Lines changed: 2 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -298,11 +298,8 @@ theorem isClosed_setOf_map_one [One M₁] [One M₂] : IsClosed { f : M₁ → M
298298
theorem isClosed_setOf_map_mul [Mul M₁] [Mul M₂] [ContinuousMul M₂] :
299299
IsClosed { f : M₁ → M₂ | ∀ x y, f (x * y) = f x * f y } := by
300300
simp only [setOf_forall]
301-
exact
302-
isClosed_iInter fun x =>
303-
isClosed_iInter fun y =>
304-
isClosed_eq (continuous_apply _)
305-
(by continuity)
301+
exact isClosed_iInter fun x ↦ isClosed_iInter fun y ↦
302+
isClosed_eq (continuous_apply _) (by fun_prop)
306303

307304
section Semigroup
308305

Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -188,7 +188,7 @@ theorem sublattice_closure_eq_top (L : Set C(X, ℝ)) (nA : L.Nonempty)
188188
have U_nhd_y : ∀ x y, U x y ∈ 𝓝 y := by
189189
intro x y
190190
refine IsOpen.mem_nhds ?_ ?_
191-
· apply isOpen_lt <;> continuity
191+
· apply isOpen_lt <;> fun_prop
192192
· rw [Set.mem_setOf_eq, w₂]
193193
exact sub_lt_self _ pos
194194
-- Fixing `x` for a moment, we have a family of functions `fun y ↦ g x y`
@@ -377,7 +377,7 @@ theorem Subalgebra.SeparatesPoints.rclike_to_real {A : StarSubalgebra 𝕜 C(X,
377377
simp only [coe_smul, coe_one, smul_apply, one_apply, Algebra.id.smul_eq_mul, mul_one,
378378
const_apply]
379379
-- Consider now the function `fun x ↦ |f x - f x₂| ^ 2`
380-
refine ⟨_, ⟨⟨(‖F ·‖ ^ 2), by continuity⟩, ?_, rfl⟩, ?_⟩
380+
refine ⟨_, ⟨⟨(‖F ·‖ ^ 2), by fun_prop⟩, ?_, rfl⟩, ?_⟩
381381
· -- This is also an element of the subalgebra, and takes only real values
382382
rw [SetLike.mem_coe, Subalgebra.mem_comap]
383383
convert (A.restrictScalars ℝ).mul_mem hFA (star_mem hFA : star F ∈ A)

Mathlib/Topology/ExtremallyDisconnected.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -300,6 +300,6 @@ instance instExtremallyDisconnected {ι : Type*} {π : ι → Type*} [∀ i, Top
300300
· rwa [← ij, sigma_mk_preimage_image_eq_self]
301301
· rw [sigma_mk_preimage_image' ij]
302302
exact isOpen_empty
303-
· continuity
303+
· fun_prop
304304

305305
end

Mathlib/Topology/Homotopy/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -212,7 +212,7 @@ def trans {f₀ f₁ f₂ : C(X, Y)} (F : Homotopy f₀ f₁) (G : Homotopy f₁
212212
toFun x := if (x.1 : ℝ) ≤ 1 / 2 then F.extend (2 * x.1) x.2 else G.extend (2 * x.1 - 1) x.2
213213
continuous_toFun := by
214214
refine
215-
continuous_if_le (continuous_induced_dom.comp continuous_fst) continuous_const
215+
continuous_if_le (by fun_prop) continuous_const
216216
(F.continuous.comp (by continuity)).continuousOn
217217
(G.continuous.comp (by continuity)).continuousOn ?_
218218
rintro x hx

Mathlib/Topology/Homotopy/HomotopyGroup.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -268,7 +268,7 @@ theorem homotopicTo (i : N) {p q : Ω^ N X x} :
268268
· rintro y ⟨i, iH⟩
269269
rw [homotopyTo_apply, H.eq_fst, p.2]
270270
all_goals apply Cube.insertAt_boundary; right; exact ⟨i, iH⟩
271-
· continuity
271+
· fun_prop
272272
iterate 2 intro; ext; erw [homotopyTo_apply, toLoop_apply]; swap
273273
· apply H.apply_zero
274274
· apply H.apply_one
@@ -282,7 +282,7 @@ theorem homotopicTo (i : N) {p q : Ω^ N X x} :
282282
@[simps!] def homotopyFrom (i : N) {p q : Ω^ N X x} (H : (toLoop i p).Homotopy (toLoop i q)) :
283283
C(I × I^N, X) :=
284284
(ContinuousMap.comp ⟨_, ContinuousMap.continuous_uncurry⟩
285-
(ContinuousMap.comp ⟨Subtype.val, by continuity⟩ H.toContinuousMap).curry).uncurry.comp <|
285+
(ContinuousMap.comp ⟨Subtype.val, by fun_prop⟩ H.toContinuousMap).curry).uncurry.comp <|
286286
(ContinuousMap.id I).prodMap (Cube.splitAt i)
287287

288288
theorem homotopicFrom (i : N) {p q : Ω^ N X x} :

Mathlib/Topology/MetricSpace/Perfect.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -122,7 +122,7 @@ theorem Perfect.exists_nat_bool_injection
122122
· rintro y ⟨x, rfl⟩
123123
exact map_mem ⟨_, hdom⟩ 0
124124
· apply hdiam.map_continuous.comp
125-
continuity
125+
fun_prop
126126
intro x y hxy
127127
simpa only [← Subtype.val_inj] using hdisj'.map_injective hxy
128128

0 commit comments

Comments
 (0)