File tree Expand file tree Collapse file tree 1 file changed +3
-4
lines changed Expand file tree Collapse file tree 1 file changed +3
-4
lines changed Original file line number Diff line number Diff line change @@ -6600,7 +6600,7 @@ Definition join_product (x : T) : PU := fun i => f_ i x.
66006600Lemma join_product_continuous : continuous join_product.
66016601Proof .
66026602suff : continuous (join_product : weakT -> PU).
6603- by move=> cts x U => /cts; rewrite /= nbhs_simpl /= -weak_sep_nbhsE.
6603+ by move=> cts x U => /cts; rewrite nbhs_simpl /= -weak_sep_nbhsE.
66046604move=> x; apply/cvg_sup; first exact/fmap_filter/(nbhs_filter (x : weakT)).
66056605move=> i; move: x; apply/(@continuousP _ (weak_topologicalType _)) => A [B ? E].
66066606rewrite -E (_ : @^~ i = prod_topo_apply i) //.
@@ -6621,9 +6621,8 @@ apply: (@filterS _ _ _ ((join_product @` setT) `&` B)).
66216621 have -> : prod_topo_apply i (join_product w) = f_ i w by [].
66226622 by move=> /exists2P/forallNP/(_ w)/not_andP [] // /contrapT.
66236623apply: open_nbhs_nbhs; split; last by rewrite -jxy.
6624- apply: openI; first exact: open_subspaceT.
6625- apply: open_subspaceW; apply: open_comp.
6626- by move=> + _; exact: prod_topo_apply_continuous.
6624+ apply: openI; first exact: open_subspaceT; apply: open_subspaceW.
6625+ apply: open_comp; first by move=> + _; exact: prod_topo_apply_continuous.
66276626by exact/closed_openC/closed_closure.
66286627Qed .
66296628
You can’t perform that action at this time.
0 commit comments