Skip to content

Commit

Permalink
Constant: more style cleanups to SurjectiveFactor
Browse files Browse the repository at this point in the history
  • Loading branch information
jdchristensen committed Feb 18, 2025
1 parent b39ace6 commit eb17f67
Showing 1 changed file with 6 additions and 9 deletions.
15 changes: 6 additions & 9 deletions theories/Constant.v
Original file line number Diff line number Diff line change
Expand Up @@ -192,24 +192,21 @@ Section SurjectiveFactor.
Proof.
rapply (merely_rec_hset (f o pr1)).
intros [x p] [y q]; cbn.
exact (resp _ _ (p @ q^)).
exact (resp x y (p @ q^)).
Defined.

(** When [g] is surjective, those propositional truncations are contractible, giving us a way to get an element of [C]. *)
Definition surjective_factor {Esurj : IsSurjection g} : B -> C.
Definition surjective_factor `{IsSurjection g} : B -> C.
Proof.
intro b.
apply (surjective_factor_aux b).
rapply center.
exact (surjective_factor_aux b (center _)).
Defined.

Definition surjective_factor_pr {Esurj : IsSurjection g}
Definition surjective_factor_factors `{IsSurjection g}
: surjective_factor o g == f.
Proof.
intros a.
unfold surjective_factor.
nrapply (ap (y:=tr (a; idpath)) (surjective_factor_aux (g a))).
1: apply path_ishprop.
intros a; unfold surjective_factor.
exact (ap (surjective_factor_aux (g a)) (contr (tr (a; idpath)))).
Defined.

End SurjectiveFactor.

0 comments on commit eb17f67

Please sign in to comment.