File tree Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Original file line number Diff line number Diff line change @@ -1254,6 +1254,15 @@ theorem continuous_update [DecidableEq ι] (i : ι) :
1254
1254
continuous_fst.update i continuous_snd
1255
1255
#align continuous_update continuous_update
1256
1256
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
+
1257
1266
theorem Filter.Tendsto.fin_insertNth {n} {π : Fin (n + 1 ) → Type _} [∀ i, TopologicalSpace (π i)]
1258
1267
(i : Fin (n + 1 )) {f : β → π i} {l : Filter β} {x : π i} (hf : Tendsto f l (𝓝 x))
1259
1268
{g : β → ∀ j : Fin n, π (i.succAbove j)} {y : ∀ j, π (i.succAbove j)} (hg : Tendsto g l (𝓝 y)) :
You can’t perform that action at this time.
0 commit comments