Skip to content

Commit 860e516

Browse files
author
Madeleine Sydney Ślaga
committed
Resolve naming conflicts
1 parent cfa1208 commit 860e516

File tree

5 files changed

+25
-27
lines changed

5 files changed

+25
-27
lines changed

Cubical/Data/Containers/ContainerExtensionProofs.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -61,11 +61,11 @@ module _ {C : Category ℓ ℓ'} where
6161
(funExt₂ λ X (s , h) sym (funExt⁻ (nat h) (s , C .id)) ∙
6262
cong (λ Z mors X (s , Z)) (C .⋆IdL h))
6363

64-
ret : X→Y fib (⟦ X→Y ⟧-mor) ≡ X→Y
65-
ret (u ◁ f) i = u ◁ λ s C .⋆IdR (f s) i
64+
ret' : X→Y fib (⟦ X→Y ⟧-mor) ≡ X→Y
65+
ret' (u ◁ f) i = u ◁ λ s C .⋆IdR (f s) i
6666

6767
unique : (y : fiber (⟦_⟧-mor) (natTrans mors nat)) (fib (natTrans mors nat) , fib-pf) ≡ y
68-
unique (m , m-eq) = Σ≡Prop (λ _ isSetNatTrans _ _) (cong fib (sym m-eq) ∙ ret m)
68+
unique (m , m-eq) = Σ≡Prop (λ _ isSetNatTrans _ _) (cong fib (sym m-eq) ∙ ret' m)
6969

7070
-- Proof 2 that the functor ⟦_⟧ is full and faithful
7171
-- Uses the Yoneda lemma

Cubical/HITs/Pushout/PushoutProduct.agda

Lines changed: 2 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -57,8 +57,6 @@ module _
5757
fam : A Type _
5858
fam a = Σ[ k ∈ ((b : B) P (a , b) .fst) ] ((y : Y) k (g y) ≡ sec (inr (a , y)))
5959

60-
open Iso
61-
6260
fiberEquiv : (a : A)
6361
fam a ≃ fiber (λ(s : (b : B) P (a , b) .fst) s ∘ g) (λ y sec (inr (a , y)))
6462
fiberEquiv a = isoToEquiv
@@ -76,8 +74,8 @@ module _
7674

7775
map-iso = elim.isIsoPrecompose f _ (λ a fam a , is-m-trunc-fam a) connf
7876

79-
k = map-iso .inv sec-fam
80-
ϕ = map-iso .sec sec-fam
77+
k = map-iso .Iso.inv sec-fam
78+
ϕ = map-iso .Iso.sec sec-fam
8179

8280
ext : (x : A × B) P x .fst
8381
ext (a , b) = k a .fst b

Cubical/HITs/SequentialColimit/Properties.agda

Lines changed: 10 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -190,31 +190,31 @@ module _
190190
(Y : SeqColim X TypeOfHLevel ℓ' d) where
191191

192192
module _
193-
(sec : (x : X .obj n) Y (incl (X .map x)) .fst) where
193+
(sec' : (x : X .obj n) Y (incl (X .map x)) .fst) where
194194

195195
lift-iso = elim.isIsoPrecompose _ d (Y ∘ incl) conn
196196

197197
liftSec' : (x : X .obj (1 + n)) Y (incl x) .fst
198-
liftSec' = lift-iso .inv sec
198+
liftSec' = lift-iso .inv sec'
199199

200-
liftSecPath' : (x : X .obj n) sec x ≡ liftSec' (X .map x)
201-
liftSecPath' x i = lift-iso .sec sec (~ i) x
200+
liftSecPath' : (x : X .obj n) sec' x ≡ liftSec' (X .map x)
201+
liftSecPath' x i = lift-iso .sec sec' (~ i) x
202202

203203
module _
204-
(sec : (x : X .obj n) Y (incl x) .fst) where
204+
(sec' : (x : X .obj n) Y (incl x) .fst) where
205205

206206
liftSec : (x : X .obj (1 + n)) Y (incl x) .fst
207-
liftSec = liftSec' (transpSec n (λ x Y x .fst) sec)
207+
liftSec = liftSec' (transpSec n (λ x Y x .fst) sec')
208208

209209
liftSecPath :
210210
(x : X .obj n)
211-
PathP (λ i Y (push x i) .fst) (sec x) (liftSec (X .map x))
211+
PathP (λ i Y (push x i) .fst) (sec' x) (liftSec (X .map x))
212212
liftSecPath x i =
213213
hcomp (λ j λ
214-
{ (i = i0) sec x
214+
{ (i = i0) sec' x
215215
; (i = i1) liftSecPath'
216-
(transpSec n (λ x Y x .fst) sec) x j })
217-
(transport-filler (λ i Y (push x i) .fst) (sec x) i)
216+
(transpSec n (λ x Y x .fst) sec') x j })
217+
(transport-filler (λ i Y (push x i) .fst) (sec' x) i)
218218

219219
module _
220220
(d : ℕ)(n : ℕ)

Cubical/Homotopy/Group/Base.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -324,13 +324,13 @@ isEquiv-Ω→SphereMap zero {A = A} =
324324
, λ i j snd f (~ i ∨ j)))
325325
λ _ refl))
326326
isEquiv-Ω→SphereMap (suc zero) {A = A} =
327-
isoToIsEquiv (iso _ invFun sec λ p sym (rUnit p))
327+
isoToIsEquiv (iso _ invFun sec' λ p sym (rUnit p))
328328
where
329329
invFun : S₊∙ 1 →∙ A typ (Ω A)
330330
invFun (f , p) = sym p ∙∙ cong f loop ∙∙ p
331331

332-
sec : section (Ω→SphereMap 1) invFun
333-
sec (f , p) =
332+
sec' : section (Ω→SphereMap 1) invFun
333+
sec' (f , p) =
334334
ΣPathP ((funExt (λ { base sym p
335335
; (loop i) j doubleCompPath-filler
336336
(sym p) (cong f loop) p (~ j) i}))

Cubical/Homotopy/Group/Join.agda

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -221,13 +221,13 @@ private
221221
λ g cong ∣_∣₂
222222
(cong (fun (Iso-JoinMap-SphereMap n m)) (sym (·Π≡+* f g))
223223
∙ ∘∙-assoc _ _ _
224-
∙ cong (∙Π f g ∘∙_) ret
224+
∙ cong (∙Π f g ∘∙_) ret'
225225
∙ ∘∙-idˡ (∙Π f g)
226226
∙ cong₂ ∙Π
227-
((sym (∘∙-idˡ f) ∙ cong (f ∘∙_) (sym ret)) ∙ sym (∘∙-assoc _ _ _))
228-
(sym (∘∙-idˡ g) ∙ cong (g ∘∙_) (sym ret) ∙ sym (∘∙-assoc _ _ _))))
227+
((sym (∘∙-idˡ f) ∙ cong (f ∘∙_) (sym ret')) ∙ sym (∘∙-assoc _ _ _))
228+
(sym (∘∙-idˡ g) ∙ cong (g ∘∙_) (sym ret') ∙ sym (∘∙-assoc _ _ _))))
229229
where
230-
ret = ≃∙→ret/sec∙ {B = _ , ptSn (suc (n + m))}
230+
ret' = ≃∙→ret/sec∙ {B = _ , ptSn (suc (n + m))}
231231
(joinSphereEquiv∙ n m) .snd
232232

233233
-π*≡-π' : {ℓ} {A : Pointed ℓ} {n m : ℕ}
@@ -241,11 +241,11 @@ private
241241
(cong (_∘∙ (≃∙map (invEquiv∙ (joinSphereEquiv∙ n m))))
242242
(sym (-Π≡-* f))
243243
∙ ∘∙-assoc _ _ _
244-
∙ cong (-Π f ∘∙_) ret
244+
∙ cong (-Π f ∘∙_) ret'
245245
∙ ∘∙-idˡ (-Π f)
246-
∙ cong -Π (sym (∘∙-assoc _ _ _ ∙ cong (f ∘∙_) ret ∙ ∘∙-idˡ f))))
246+
∙ cong -Π (sym (∘∙-assoc _ _ _ ∙ cong (f ∘∙_) ret' ∙ ∘∙-idˡ f))))
247247
where
248-
ret = ≃∙→ret/sec∙ {B = _ , ptSn (suc (n + m))}
248+
ret' = ≃∙→ret/sec∙ {B = _ , ptSn (suc (n + m))}
249249
(joinSphereEquiv∙ n m) .snd
250250

251251
-- Homotopy groups in terms of joins

0 commit comments

Comments
 (0)