Skip to content

Commit 1fd8717

Browse files
committed
This was incorrectly marked as forward-ported in #2110. You can see that by looking at [the status page](https://leanprover-community.github.io/mathlib-port-status/file/topology/constructions?range=bcfa726826abd57587355b4b5b7e78ad6527b7e4..dde670c9a3f503647fd5bfdf1037bad526d3397a) and noting that no commits in mathlib4 contain the diff from the highlighted commits on the left.
1 parent 5d07683 commit 1fd8717

File tree

1 file changed

+9
-0
lines changed

1 file changed

+9
-0
lines changed

Mathlib/Topology/Constructions.lean

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1254,6 +1254,15 @@ theorem continuous_update [DecidableEq ι] (i : ι) :
12541254
continuous_fst.update i continuous_snd
12551255
#align continuous_update continuous_update
12561256

1257+
/-- `Pi.mulSingle i x` is continuous in `x`. -/
1258+
-- porting note: todo: restore @[continuity]
1259+
@[to_additive "`Pi.single i x` is continuous in `x`."]
1260+
theorem continuous_mulSingle [∀ i, One (π i)] [DecidableEq ι] (i : ι) :
1261+
Continuous fun x => (Pi.mulSingle i x : ∀ i, π i) :=
1262+
continuous_const.update _ continuous_id
1263+
#align continuous_mul_single continuous_mulSingle
1264+
#align continuous_single continuous_single
1265+
12571266
theorem Filter.Tendsto.fin_insertNth {n} {π : Fin (n + 1) → Type _} [∀ i, TopologicalSpace (π i)]
12581267
(i : Fin (n + 1)) {f : β → π i} {l : Filter β} {x : π i} (hf : Tendsto f l (𝓝 x))
12591268
{g : β → ∀ j : Fin n, π (i.succAbove j)} {y : ∀ j, π (i.succAbove j)} (hg : Tendsto g l (𝓝 y)) :

0 commit comments

Comments
 (0)