You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Copy file name to clipboardExpand all lines: theories/Homotopy/Hopf.v
+36-12Lines changed: 36 additions & 12 deletions
Original file line number
Diff line number
Diff line change
@@ -23,7 +23,7 @@ Proof.
23
23
srapply Build_pFam.
24
24
- apply (Susp_rec (Y:=Type) X X).
25
25
(** In order to use the flattening lemma for colimits to show that the total space is a join, we need for this equivalence to be a composition with the inverted identity equivalence so that the fiber is definitionally equivalent to the flattening lemma sigma type. This doesn't change anything elsewhere, but saves us having to rewrite an IsEquiv witness. *)
26
-
exact (fun x => path_universe ((x *.) o equiv_idmap^-1)).
26
+
exact (fun x => path_universe ((x *.) o equiv_idmap)).
27
27
- simpl. exact pt.
28
28
Defined.
29
29
@@ -106,14 +106,18 @@ Proof.
106
106
rapply freudenthal_hspace.
107
107
Defined.
108
108
109
-
(** *** Total space of the Hopf fibration*)
109
+
(** *** Total space of the Hopf construction*)
110
110
111
-
(** The total space of the Hopf fibration on [Susp X] is the join of [X] with itself. Note that we need both left and right multiplication to be equivalences. This is true when [X] is a 0-connected H-space for example. *)
111
+
(** The total space of the Hopf construction on [Susp X] is the join of [X] with itself. Note that we need both left and right multiplication to be equivalences. This is true when [X] is a 0-connected H-space for example. *)
112
112
(* TODO: Show that this is a pointed equivalence. We cannot yet do this as we cannot compute with the flattening lemma due to the massive size of the proof. *)
Copy file name to clipboardExpand all lines: theories/Types/Unit.v
-12Lines changed: 0 additions & 12 deletions
Original file line number
Diff line number
Diff line change
@@ -117,15 +117,3 @@ Definition contr_equiv_unit (A : Type) (f : A <~> Unit) : Contr A
117
117
118
118
(** The constant map to [Unit]. We define this so we can get rid of an unneeded universe variable that Coq generates when [const tt] is used in a context that doesn't have [Universe Minimization ToSet] as this file does. If we ever set that globally, then we could get rid of this and remove some imports of this file. *)
119
119
Definition const_tt (A : Type) := @const A Unit tt.
120
-
121
-
(** Families over Unit type are equivalent to the type at the base point. *)
0 commit comments