Skip to content

Commit

Permalink
fixing name clash
Browse files Browse the repository at this point in the history
  • Loading branch information
marcinjangrzybowski committed Aug 28, 2024
1 parent fc1b7c3 commit 4871437
Show file tree
Hide file tree
Showing 4 changed files with 8 additions and 8 deletions.
4 changes: 2 additions & 2 deletions Cubical/Data/List/Properties.agda
Original file line number Diff line number Diff line change
Expand Up @@ -341,8 +341,8 @@ lookupAlways a [] _ = a
lookupAlways _ (x ∷ _) zero = x
lookupAlways a (x ∷ xs) (suc k) = lookupAlways a xs k

lookup : List A Maybe A
lookup = lookupAlways nothing ∘S map just
lookupMb : List A Maybe A
lookupMb = lookupAlways nothing ∘S map just

rot : List A List A
rot [] = []
Expand Down
4 changes: 2 additions & 2 deletions Cubical/Tactics/PathSolver/MonoidalSolver/PathEval.agda
Original file line number Diff line number Diff line change
Expand Up @@ -294,7 +294,7 @@ fill-flatten' = hTop ∘S atVarOrConOrDefMmp
fill-offsetPa' : List (R.Arg R.Term) List (R.Arg R.Term)
fill-offsetPa' n xs =
let hd = fromJust-def (varg (R.lit (R.string "fatal in PathEval - offsetPa'")))
(lookup xs zero)
(lookupMb xs zero)
hs* = mapArg (dropFillWraps headFW) hd
hd' = mapArg
(replaceVarWithCon (λ { zero just (quote i0) ; _ nothing })) hs*
Expand All @@ -310,7 +310,7 @@ fill-flatten' = hTop ∘S atVarOrConOrDefMmp

hTop : List R.Term List R.Term
hTop = L.map (Mb.fromJust-def ( (R.lit (R.string "imposible in fill-flatten'")) )
∘S map-Maybe (unArg) ∘S flip lookup zero) ∘S h ∘S [_] ∘S L.map varg
∘S map-Maybe (unArg) ∘S flip lookupMb zero) ∘S h ∘S [_] ∘S L.map varg

df :
R.Name
Expand Down
6 changes: 3 additions & 3 deletions Cubical/Tactics/PathSolver/NSolver/NSolver.agda
Original file line number Diff line number Diff line change
Expand Up @@ -309,9 +309,9 @@ module _ (ty : R.Type) where
fcs0₀ Mb.rec (R.typeError [ "imposible" ]ₑ)
(λ y mapM (λ k (getVert 100 (replaceAt k true v0)) (fst y)
<|> fail ("fcs1 fail" ∷nl [ k ]ₑ)) (range dim))
(lookup fcs0 0)
(lookupMb fcs0 0)
fcs0₁ Mb.rec (R.typeError [ "imposible" ]ₑ)
(getVert 100 (replaceAt (predℕ dim) true v0) ∘S fst) (lookup fcs0 1)
(getVert 100 (replaceAt (predℕ dim) true v0) ∘S fst) (lookupMb fcs0 1)

fcs1 mapM (idfun _)
(zipWith (markVertSnd 100 dim) (fcs0₁ ∷ fcs0₀) ((snd ∘S snd) <$> xs))
Expand Down Expand Up @@ -480,7 +480,7 @@ solvePathsSolver goal = R.withReduceDefs (false , doNotReduceInPathSolver) do
R.debugPrint "solvePaths" 0 $ [ "solvePaths - matchNCube done" ]ₑ
let dim = length fcs

(t0 , _) Mb.rec (R.typeError [ "imposible in solvePaths''" ]ₑ) pure (lookup fcs zero)
(t0 , _) Mb.rec (R.typeError [ "imposible in solvePaths''" ]ₑ) pure (lookupMb fcs zero)

cuFcs ((zipWithIndex <$> quoteBd bdTM
-- <|> R.typeError [ "quoteBd - failed" ]ₑ
Expand Down
2 changes: 1 addition & 1 deletion Cubical/Tactics/Reflection/Utilities.agda
Original file line number Diff line number Diff line change
Expand Up @@ -387,7 +387,7 @@ replaceVarWithTerm f =


substTms : List Term Term Term
substTms xs = dropVars.rv (length xs) zero ∘S replaceVarWithTerm (lookup (map (liftVarsFrom (length xs) 0) xs))
substTms xs = dropVars.rv (length xs) zero ∘S replaceVarWithTerm (lookupMb (map (liftVarsFrom (length xs) 0) xs))

replaceAtTrm : Term Term Term
replaceAtTrm k t =
Expand Down

0 comments on commit 4871437

Please sign in to comment.