Skip to content
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
4 changes: 4 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -69,6 +69,8 @@
- in `measurable_realfun.v`:
+ lemmas `measurable_funN`
+ lemmas `nondecreasing_measurable`, `nonincreasing_measurable`
- in `subspace_topology.v`:
+ definition `from_subspace`

### Changed

Expand All @@ -83,6 +85,8 @@

- in `lebesgue_integral_monotone_convergence.v`:
+ lemma `ge0_le_integral` (remove superfluous hypothesis)
- in `subspace_topology.v`:
+ notation `{within _, continuous _}` (now uses `from_subspace`)

### Renamed

Expand Down
Original file line number Diff line number Diff line change
Expand Up @@ -758,7 +758,7 @@ exists (\bigcup_(i in range f) dK i); split.
+ move=> i _; split; first by apply: compact_closed; have [] := dkP i.
apply: (continuous_subspaceW (dKsub i)).
apply: (@subspace_eq_continuous _ _ _ (fun=> i)).
by move=> ? /set_mem ->.
by rewrite /from_subspace => ? /set_mem ->.
by apply: continuous_subspaceT => ?; exact: cvg_cst.
Qed.

Expand Down
34 changes: 23 additions & 11 deletions theories/topology_theory/subspace_topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,16 +9,24 @@ From mathcomp Require Import product_topology.
(* # Subspaces of topological spaces *)
(* *)
(* ``` *)
(* subspace A == for (A : set T), this is a copy of T with a *)
(* topology that ignores points outside A *)
(* incl_subspace x == with x of type subspace A with (A : set T), *)
(* inclusion of subspace A into T *)
(* nbhs_subspace x == filter associated with x : subspace A *)
(* subspace_ent A == subspace entourages *)
(* subspace_ball A == balls of the pseudometric subspace structure *)
(* continuousFunType A B == type of continuous function from set A to set B *)
(* with domain subspace A *)
(* The HB structure is ContinuousFun. *)
(* subspace A == for (A : set T), this is a copy of T with a *)
(* topology that ignores points outside A *)
(* incl_subspace x == with x of type subspace A with (A : set T), *)
(* inclusion of subspace A into T *)
(* nbhs_subspace x == filter associated with x : subspace A *)
(* from_subspace A f == function of type `subspace A -> U` given a *)
(* function f of type `A -> U` *)
(* The purpose of this definition is to preserve *)
(* the pretty-printing of the notation *)
(* {within _, continuous _} below. Its use is *)
(* however likely to be later superseded by a *)
(* better (compositional) mechanism. *)
(* {within A, continuous f} := continuous (from_subspace A f)) *)
(* subspace_ent A == subspace entourages *)
(* subspace_ball A == balls of the pseudometric subspace structure *)
(* continuousFunType A B == type of continuous functions from set A to *)
(* set B with domain subspace A *)
(* The HB structure is ContinuousFun. *)
(* ``` *)
(******************************************************************************)

Expand Down Expand Up @@ -303,8 +311,12 @@ Global Instance subspace_proper_filter {T : topologicalType}
(A : set T) (x : subspace A) :
ProperFilter (nbhs_subspace x) := nbhs_subspace_filter x.

Definition from_subspace {T U : Type} (A : set T) (f : T -> U) : subspace A -> U :=
f.
Arguments from_subspace {T U} A f.

Notation "{ 'within' A , 'continuous' f }" :=
(continuous (f : subspace A -> _)) : classical_set_scope.
(continuous (from_subspace A f)) : classical_set_scope.

Arguments nbhs_subspaceP {T} A x.

Expand Down