Skip to content

Commit

Permalink
functions on wedges
Browse files Browse the repository at this point in the history
  • Loading branch information
zstone1 committed Nov 15, 2024
1 parent d227e94 commit fd062aa
Show file tree
Hide file tree
Showing 2 changed files with 22 additions and 7 deletions.
7 changes: 7 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -102,6 +102,13 @@
+ new lemmas `continuous_curry_fun`, `continuous_curry_cvg`,
`eval_continuous`, and `compose_continuous`

- in file `wedge_sigT.v`,
+ new definitions `wedge_fun`, and `wedge_prod`.
+ new lemmas `wedge_fun_continuous`, `wedge_lift_funE`,
`wedge_fun_comp`, `wedge_prod_pointE`, `wedge_prod_inj`,
`wedge_prod_continuous`, `wedge_prod_open`, `wedge_hausdorff`, and
`wedge_fun_joint_continuous`.

### Changed

- in file `normedtype.v`,
Expand Down
22 changes: 15 additions & 7 deletions theories/homotopy_theory/wedge_sigT.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,6 +19,14 @@ Require Import EqdepFacts.
(* wedge_lift i == the lifting of elements of (X i) into the wedge *)
(* pwedge p0 == the wedge of ptopologicalTypes at their designated *)
(* point *)
(* wedge_fun f == lifts a family of functions on each component into *)
(* a function on the wedge, when they all agree at the *)
(* wedge point *)
(* wedge_prod == the mapping from the wedge as a quotient of sums to *)
(* the wedge as a subspace of the product topology. *)
(* It's an embedding when the index is finite. *)
(* *)
(* *)
(* ``` *)
(* The type `wedge p0` is endowed with the structures of: *)
(* - topology via `quotient_topology` *)
Expand Down Expand Up @@ -347,26 +355,26 @@ case : (wedge_nbhs_specP u) => //.
move: Ukp0; rewrite (@kE t i0 x).
rewrite -[k x ]uncurryK /curry=> /kcts; case; case=> P Q /= [Pt Qp0 pqU].
by exists (P,Q) => //.
have UPQ : nbhs (wedgei (p0 i0)) (
\bigcup_x (@wedgei x) @` (snd (projT1 (pq_ x)))).
have UPQ : nbhs (wedge_lift (p0 i0)) (
\bigcup_x (@wedge_lift x) @` (snd (projT1 (pq_ x)))).
rewrite wedge_point_nbhs => r _.
by case: (projT2 (pq_ r)) => /filterS + ? ?; apply => z /= ?; by exists r.
have /finite_fsetP [fI fIE] := Ifin.
have UPt : nbhs t (\bigcap_(r in [set` fI]) (fst (projT1 (pq_ r)))).
by apply: filter_bigI => x ?; case: (projT2 (pq_ x)).
near_simpl => /=; near=> t1 t2 => /=.
have [] // := near UPQ t2 => x _ [w /=] ? <-.
rewrite wedge_fun_wedgei //.
rewrite wedge_lift_funE //.
case: (projT2 (pq_ x)) => ? Npt /(_ (t1, w)) => /=; apply; split => //.
by have := near UPt t1; apply; rewrite // -fIE.
move: u => _ x u uNp0 /=; rewrite wedge_fun_wedgei //=.
move: u => _ x u uNp0 /=; rewrite wedge_lift_funE //=.
rewrite -[k x]uncurryK /curry => /kcts; rewrite nbhs_simpl /=.
case; case => /= P Q [Pt Qu] PQU.
have wQu : nbhs (wedgei u) ((@wedgei x) @` Q).
rewrite -wedgei_nbhs //=; move/filterS: Qu; apply.
have wQu : nbhs (wedge_lift u) ((@wedge_lift x) @` Q).
rewrite -wedge_lift_nbhs //=; move/filterS: Qu; apply.
by move=> z; exists z.
near_simpl; near=> t1 t2 => /=.
have [] // := near wQu t2 => l ? <-; rewrite wedge_fun_wedgei //.
have [] // := near wQu t2 => l ? <-; rewrite wedge_lift_funE //.
apply: (PQU (t1,l)); split => //.
exact: (near Pt t1).
Unshelve. all: by end_near. Qed.
Expand Down

0 comments on commit fd062aa

Please sign in to comment.