Skip to content

Commit ac42713

Browse files
committed
cleaning up proofs
1 parent 98478a4 commit ac42713

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
@@ -6601,7 +6601,7 @@ Definition join_product (x : T) : PU := fun i => f_ i x.
66016601
Lemma join_product_continuous : continuous join_product.
66026602
Proof.
66036603
suff : continuous (join_product : weakT -> PU).
6604-
by move=> cts x U => /cts; rewrite /= nbhs_simpl /= -weak_sep_nbhsE.
6604+
by move=> cts x U => /cts; rewrite nbhs_simpl /= -weak_sep_nbhsE.
66056605
move=> x; apply/cvg_sup; first exact/fmap_filter/(nbhs_filter (x : weakT)).
66066606
move=> i; move: x; apply/(@continuousP _ (weak_topologicalType _)) => A [B ? E].
66076607
rewrite -E (_ : @^~ i = prod_topo_apply i) //.
@@ -6622,9 +6622,8 @@ apply: (@filterS _ _ _ ((join_product @` setT) `&` B)).
66226622
have -> : prod_topo_apply i (join_product w) = f_ i w by [].
66236623
by move=> /exists2P/forallNP/(_ w)/not_andP [] // /contrapT.
66246624
apply: open_nbhs_nbhs; split; last by rewrite -jxy.
6625-
apply: openI; first exact: open_subspaceT.
6626-
apply: open_subspaceW; apply: open_comp.
6627-
by move=> + _; exact: prod_topo_apply_continuous.
6625+
apply: openI; first exact: open_subspaceT; apply: open_subspaceW.
6626+
apply: open_comp; first by move=> + _; exact: prod_topo_apply_continuous.
66286627
by exact/closed_openC/closed_closure.
66296628
Qed.
66306629

0 commit comments

Comments
 (0)