Skip to content

Commit 5ad8432

Browse files
committed
adding local notations for proof legibility
1 parent c8f09f0 commit 5ad8432

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

theories/topology.v

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -6698,8 +6698,14 @@ Hypothesis ctsf : forall i, continuous (f_ i).
66986698

66996699
Let weakT := @sup_topologicalType T I
67006700
(fun i => Topological.class (weak_topologicalType (f_ i))).
6701+
67016702
Let PU := product_topologicalType U_.
67026703

6704+
Local Notation sup_open := (@open weakT).
6705+
Local Notation "'weak_open' i" :=
6706+
(@open (weak_topologicalType (f_ i))) (at level 0).
6707+
Local Notation natural_open := (@open T).
6708+
67036709
Lemma weak_sep_cvg (F : set (set T)) (x : T) :
67046710
Filter F -> (F --> (x : T)) <-> (F --> (x : weakT)).
67056711
Proof.
@@ -6745,6 +6751,8 @@ apply: open_comp => // + _; rewrite /cvg_to => x U.
67456751
by rewrite nbhs_simpl /= -weak_sep_nbhsE; move: x U; exact: ctsf.
67466752
Qed.
67476753

6754+
Local Notation prod_open := (@open (subspace_topologicalType (range join_product))).
6755+
67486756
Lemma join_product_open (A : set T) : open A ->
67496757
open ((join_product @` A) : set (subspace (range join_product))).
67506758
Proof.

0 commit comments

Comments
 (0)