Skip to content

Commit e5cde84

Browse files
authored
Update Construction.agda
1 parent 5a92d3c commit e5cde84

File tree

1 file changed

+5
-9
lines changed

1 file changed

+5
-9
lines changed

Cubical/Categories/RezkCompletion/Construction.agda

+5-9
Original file line numberDiff line numberDiff line change
@@ -376,7 +376,7 @@ module RezkByHIT (C : Category ℓ ℓ') where
376376
Rezk⋆Assoc : x y z w f g h
377377
Rezk⋆ x z w (Rezk⋆ x y z f g) h ≡ Rezk⋆ x y w f (Rezk⋆ y z w g h)
378378
Rezk⋆Assoc = elimProp₂ (λ x y isPropΠ5 λ z w _ _ _ isSetRezkHom x w _ _) λ x y
379-
elimProp₂ (λ z w isPropΠ3 λ _ _ _ isSetRezkHom (inc x) w _ _) λ z w C.⋆Assoc
379+
elimProp₂ (λ z w isPropΠ3 λ _ _ _ isSetRezkHom (inc x) w _ _) λ z w C.⋆Assoc
380380

381381
Rezk : Category (ℓ-max ℓ ℓ') ℓ'
382382
Rezk .ob = RezkOb
@@ -412,19 +412,15 @@ module RezkByHIT (C : Category ℓ ℓ') where
412412
inc-ua (⋆Iso f' (invIso e)) ∙ inc-ua e
413413
≡⟨ sym (inc-⋆ (⋆Iso f' (invIso e)) e) ⟩
414414
inc-ua (⋆Iso (⋆Iso f' (invIso e)) e)
415-
≡⟨ cong inc-ua (CatIso≡ _ _ (
416-
C.⋆Assoc _ _ _ ∙ congR C._⋆_ (e .snd .sec) ∙ C.⋆IdR _)
417-
) ⟩
415+
≡⟨ cong inc-ua (CatIso≡ _ _ (C.⋆Assoc _ _ _ ∙ congR C._⋆_ (e .snd .sec) ∙ C.⋆IdR _)) ⟩
418416
inc-ua f' ∎
419417

420418
R-ua₂ : {x y z : C.ob} (f : Σ C.Hom[ x , y ] (isIso C))
421419
PathP (λ i CatIso Rezk (inc-ua f i) (inc z) inc-ua f i ≡ inc z)
422420
(R-inc x z) (R-inc y z)
423421
R-ua₂ e = toPathP $ funExt λ f let f' = RezkIso→Iso f in
424422
subst2 _≡_ (inc-ua e) refl (inc-ua _)
425-
≡⟨ cong (subst2 _≡_ (inc-ua e) refl ∘ inc-ua) (
426-
CatIso≡ _ _ (congR C._⋆_ (transportRefl _))
427-
) ⟩
423+
≡⟨ cong (subst2 _≡_ (inc-ua e) refl ∘ inc-ua) (CatIso≡ _ _ (congR C._⋆_ (transportRefl _))) ⟩
428424
subst2 _≡_ (inc-ua e) refl (inc-ua (⋆Iso e f'))
429425
≡⟨ fromPathP (compPath-filler' (sym (inc-ua e)) (inc-ua (⋆Iso e f'))) ⟩
430426
sym (inc-ua e) ∙ inc-ua (⋆Iso e f')
@@ -460,8 +456,8 @@ module RezkByHIT (C : Category ℓ ℓ') where
460456
→RezkSurj = elimProp (λ x isPropPropTrunc) λ x ∣ x , idCatIso ∣₁
461457

462458
isWkEquiv→Rezk : isWeakEquivalence →Rezk
463-
isWkEquiv→Rezk .isWeakEquivalence.fullfaith = →RezkFF
464-
isWkEquiv→Rezk .isWeakEquivalence.esssurj = →RezkSurj
459+
isWkEquiv→Rezk .fullfaith = →RezkFF
460+
isWkEquiv→Rezk .esssurj = →RezkSurj
465461

466462
isRezkCompletion→Rezk : isRezkCompletion →Rezk
467463
isRezkCompletion→Rezk = makeIsRezkCompletion isUnivalentRezk isWkEquiv→Rezk

0 commit comments

Comments
 (0)