Skip to content

Commit

Permalink
linting pass
Browse files Browse the repository at this point in the history
fixing lines

Update theories/topology.v

using a better lemma to eliminate Eqdep_dec.eq_rect_eq_dec

Co-authored-by: Cyril Cohen <[email protected]>

doc, lint, compress
  • Loading branch information
zstone1 committed Jan 20, 2022
1 parent 3f7d5f0 commit 958cc30
Showing 1 changed file with 44 additions and 0 deletions.
44 changes: 44 additions & 0 deletions theories/topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -208,7 +208,14 @@ Require Import boolp reals classical_sets posnum.
(* cluster F == set of cluster points of F. *)
(* compact == set of compact sets w.r.t. the filter- *)
(* based definition of compactness. *)
<<<<<<< HEAD
(* hausdorff_space T <-> T is a Hausdorff space (T_2). *)
=======
(* hausdorff T <-> T is a Hausdorff space (T_2). *)
(* evaluator_dep x f == application of f to x, f being a *)
(* product topology of a family K *)
(* (K : X -> topologicalType) *)
>>>>>>> 83b8836... doc, lint, compress
(* cover_compact == set of compact sets w.r.t. the open *)
(* cover-based definition of compactness. *)
(* connected A <-> the only non empty subset of A which *)
Expand Down Expand Up @@ -2873,6 +2880,43 @@ Qed.

End Tychonoff.

Section DependentEvaluators.
Context {X : choiceType} {K : X -> topologicalType}.

Definition evaluator_dep x (f : product_topologicalType K) := f x.

Lemma evaluator_depE x f : evaluator_dep x f = f x.
Proof. by []. Qed.

Lemma evaluator_dep_continuous x : continuous (evaluator_dep x).
Proof.
move=> f; have /cvg_sup/(_ x)/cvg_image : f --> f by apply: cvg_id.
move=> h; apply: (cvg_trans _ (h _)) => {h}; last first.
pose xval x (y : K x) i : K i :=
match eqVneq x i return K i with
| EqNotNeq r => @eq_rect X x K y i r
| NeqNotEq _ => point
end.
rewrite eqEsubset; split => y //= _; exists (xval x y) => //; rewrite /xval.
by case (eqVneq x x) => [e|/eqP//]; rewrite eq_axiomK.
by move=> Q /= [W nbdW <-]; apply: filterS nbdW; exact: preimage_image.
Qed.

Lemma hausdorff_product :
(forall x, hausdorff (K x)) -> hausdorff (@product_topologicalType X K).
Proof.
move=> hsdfK p q /= clstr; apply: functional_extensionality_dep => x.
apply: hsdfK; move: clstr; rewrite ?cluster_cvgE /= => -[G PG [GtoQ psubG]].
exists (evaluator_dep x @ G); [exact: fmap_proper_filter|split].
rewrite -(evaluator_depE x).
apply: cvg_trans; last exact: (@evaluator_dep_continuous x q).
by apply: cvg_app; exact: GtoQ.
move/(cvg_app (evaluator_dep x)): psubG => /cvg_trans; apply.
exact: evaluator_dep_continuous.
Qed.

End DependentEvaluators.

Definition finI (I : choiceType) T (D : set I) (f : I -> set T) :=
forall D' : {fset I}, {subset D' <= D} ->
\bigcap_(i in [set i | i \in D']) f i !=set0.
Expand Down

0 comments on commit 958cc30

Please sign in to comment.