Skip to content

Commit

Permalink
definition of cohomology groups
Browse files Browse the repository at this point in the history
Signed-off-by: Ali Caglayan <[email protected]>

<!-- ps-id: c12c59da-ff46-41d1-a362-09c83052f54c -->
  • Loading branch information
Alizter committed Feb 25, 2024
1 parent 3866f7f commit 568f170
Showing 1 changed file with 20 additions and 0 deletions.
20 changes: 20 additions & 0 deletions theories/Homotopy/Cohomology.v
Original file line number Diff line number Diff line change
@@ -0,0 +1,20 @@
Require Import Basics Types Pointed.Core.
Require Import Truncations.Core.
Require Import Homotopy.EMSpace.
Require Import Homotopy.HSpace.Core Homotopy.HSpace.Pointwise Homotopy.HSpace.HGroup Homotopy.HSpace.Coherent.
Require Import Algebra.AbGroups.AbelianGroup.

Local Open Scope pointed_scope.

(** * Cohomology groups *)

(** Reduced cohomology groups are defined as the homotopy classes of pointed maps from the space to an Eilenberg-MacLane space. The group structure comes from the H-space structure on [K(G, n)]. *)
Definition Cohomology `{Univalence} (n : nat) (X : pType) (G : AbGroup) : AbGroup.
Proof.
snrapply Build_AbGroup'.
1: exact (Tr 0 (X ->** K(G, n))).
1-3: shelve.
nrapply isabgroup_ishabgroup_tr.
nrapply ishabgroup_hspace_pmap.
apply iscohhabgroup_em.
Defined.

0 comments on commit 568f170

Please sign in to comment.