Skip to content

Commit

Permalink
better name for bpwedge point
Browse files Browse the repository at this point in the history
  • Loading branch information
zstone1 committed Nov 19, 2024
1 parent 6a67c0d commit a503a13
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 7 deletions.
2 changes: 1 addition & 1 deletion CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -116,7 +116,7 @@
+ new definitions `reparameterize`, `mk_path`, and `chain_path`.
+ new lemmas `path_eqP`, and `chain_path_cts_point`.
- in file `homotopy_theory/wedge_sigT.v`,
+ new definition `wedge2p`.
+ new definition `bpwedge_shared_pt`.
+ new notations `bpwedge`, and `bpwedge_lift`.

### Changed
Expand Down
13 changes: 7 additions & 6 deletions theories/homotopy_theory/wedge_sigT.v
Original file line number Diff line number Diff line change
Expand Up @@ -24,8 +24,9 @@ From mathcomp Require Import separation_axioms function_spaces.
(* 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. *)
(* bpwedge_shared_pt b == the shared point in the bpwedge. Either zero or one *)
(* depending on `b`. *)
(* bpwedge == wedge of two bipointed spaces gluing zero to one *)
(* wedge2p == the shared point in the bpwedge *)
(* bpwedge_lift == wedge_lift specialized to the bipointed wedge *)
(* ``` *)
(* *)
Expand Down Expand Up @@ -390,10 +391,10 @@ End pwedge.
Section bpwedge.
Context (X Y : bpTopologicalType).

Definition wedge2p b :=
Definition bpwedge_shared_pt b :=
if b return (if b then X else Y) then @one X else @zero Y.
Local Notation bpwedge := (@wedge bool _ wedge2p).
Local Notation bpwedge_lift := (@wedge_lift bool _ wedge2p).
Local Notation bpwedge := (@wedge bool _ bpwedge_shared_pt).
Local Notation bpwedge_lift := (@wedge_lift bool _ bpwedge_shared_pt).

Local Lemma wedge_neq : @bpwedge_lift true zero != @bpwedge_lift false one.
Proof.
Expand All @@ -407,5 +408,5 @@ HB.instance Definition _ := @isBiPointed.Build
bpwedge (@bpwedge_lift true zero) (@bpwedge_lift false one) wedge_neq.
End bpwedge.

Notation bpwedge X Y := (@wedge bool _ (wedge2p X Y)).
Notation bpwedge_lift X Y := (@wedge_lift bool _ (wedge2p X Y)).
Notation bpwedge X Y := (@wedge bool _ (bpwedge_shared_pt X Y)).
Notation bpwedge_lift X Y := (@wedge_lift bool _ (bpwedge_shared_pt X Y)).

0 comments on commit a503a13

Please sign in to comment.