File tree Expand file tree Collapse file tree 1 file changed +1
-7
lines changed
Expand file tree Collapse file tree 1 file changed +1
-7
lines changed Original file line number Diff line number Diff line change @@ -10,7 +10,6 @@ open HomReasoning
1010open Equiv
1111
1212open import Level
13- open import Function.Base using (_$_)
1413open import Relation.Binary.Core using (Rel)
1514
1615open import Categories.Morphism.Reasoning 𝒞
@@ -42,7 +41,7 @@ Slice A = record
4241 ; _≈_ = λ where
4342 (slicearr {f} _) (slicearr {g} _) → f ≈ g
4443 ; id = slicearr identityʳ
45- ; _∘_ = _∘′_
44+ ; _∘_ = λ (slicearr △) (slicearr △′) → slicearr (glueTrianglesʳ △ △′)
4645 ; assoc = assoc
4746 ; sym-assoc = sym-assoc
4847 ; identityˡ = identityˡ
@@ -55,8 +54,3 @@ Slice A = record
5554 }
5655 ; ∘-resp-≈ = ∘-resp-≈
5756 }
58- where _∘′_ : Slice⇒ Y Z → Slice⇒ X Y → Slice⇒ X Z
59- _∘′_ {Y = sliceobj y} {Z = sliceobj z} {X = sliceobj x} (slicearr {g} △) (slicearr {f} △′) = slicearr $ begin
60- z ∘ g ∘ f ≈⟨ pullˡ △ ⟩
61- y ∘ f ≈⟨ △′ ⟩
62- x ∎
You can’t perform that action at this time.
0 commit comments