Skip to content

Commit

Permalink
move and simplify equiv_ab_biprod_ind_homotopy
Browse files Browse the repository at this point in the history
Signed-off-by: Ali Caglayan <[email protected]>
  • Loading branch information
Alizter committed Sep 10, 2024
1 parent 96b6e0b commit acba3a7
Showing 1 changed file with 11 additions and 12 deletions.
23 changes: 11 additions & 12 deletions theories/Algebra/AbGroups/Biproduct.v
Original file line number Diff line number Diff line change
Expand Up @@ -52,6 +52,17 @@ Proof.
f_ap.
Defined.

(* Maps out of biproducts are determined on the two inclusions. *)
Definition equiv_ab_biprod_ind_homotopy `{Funext} {A B X : AbGroup} (phi psi : ab_biprod A B $-> X)
: (phi $o ab_biprod_inl == psi $o ab_biprod_inl)
* (phi $o ab_biprod_inr == psi $o ab_biprod_inr)
<~> phi == psi.
Proof.
apply equiv_iff_hprop.
- exact (uncurry ab_biprod_ind_homotopy).
- exact (fun h => (fun a => h _, fun b => h _)).
Defined.

(** Recursion principle *)
Proposition ab_biprod_rec {A B Y : AbGroup}
(f : A $-> Y) (g : B $-> Y)
Expand Down Expand Up @@ -223,18 +234,6 @@ Defined.

(** *** Lemmas for working with biproducts *)

(* Maps out of biproducts are determined on the two inclusions. *)
Lemma equiv_ab_biprod_ind_homotopy `{Funext} {A B X : AbGroup} (phi psi : ab_biprod A B $-> X)
: ((phi $o ab_biprod_inl == psi $o ab_biprod_inl) * (phi $o ab_biprod_inr == psi $o ab_biprod_inr))
<~> phi == psi.
Proof.
apply equiv_iff_hprop.
- intros [h k].
apply ab_biprod_ind_homotopy; assumption.
- intro h.
exact (fun a => h _, fun b => h _).
Defined.

(** The swap isomorphism of the biproduct of two groups. *)
Definition direct_sum_swap {A B : AbGroup}
: ab_biprod A B $<~> ab_biprod B A.
Expand Down

0 comments on commit acba3a7

Please sign in to comment.