Skip to content

Commit f81fd0f

Browse files
committed
cleaning up proofs
1 parent 022b5e4 commit f81fd0f

File tree

1 file changed

+3
-4
lines changed

1 file changed

+3
-4
lines changed

theories/topology.v

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -6600,7 +6600,7 @@ Definition join_product (x : T) : PU := fun i => f_ i x.
66006600
Lemma join_product_continuous : continuous join_product.
66016601
Proof.
66026602
suff : 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.
66046604
move=> x; apply/cvg_sup; first exact/fmap_filter/(nbhs_filter (x : weakT)).
66056605
move=> i; move: x; apply/(@continuousP _ (weak_topologicalType _)) => A [B ? E].
66066606
rewrite -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.
66236623
apply: 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.
66276626
by exact/closed_openC/closed_closure.
66286627
Qed.
66296628

0 commit comments

Comments
 (0)