Skip to content

Commit

Permalink
ScopedSnocList: Fix CI
Browse files Browse the repository at this point in the history
Co-authored-by: Viktor Yudov <[email protected]>
  • Loading branch information
GulinSS and spcfox committed Feb 7, 2025
1 parent 7fc2f3a commit b2542e3
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
4 changes: 2 additions & 2 deletions src/Compiler/CompileExpr.idr
Original file line number Diff line number Diff line change
Expand Up @@ -478,7 +478,7 @@ mutual
-- the RHS
then do log "compiler.newtype.world" 50 "Inlining case on \{show n} (no world)"

sc' : CExp (vars <>< args) <- toCExpTree n sc
sc' <- toCExpTree n sc
let sc'' : CExp (vars ++ cast args)
:= rewrite sym $ fishAsSnocAppend vars args in sc'

Expand All @@ -493,7 +493,7 @@ mutual
let (s, env) : (_, SubstCEnv (cast args) (vars :< MN "eff" 0))
= mkSubst 0 (CLocal fc First) pos args
sc' : CExp (vars <>< args) <- toCExpTree n sc
sc' <- toCExpTree n sc

let sc'' : CExp (vars ++ cast args)
:= rewrite sym $ fishAsSnocAppend vars args in sc'
Expand Down
2 changes: 1 addition & 1 deletion src/Core/Name/Scoped.idr
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ import Core.Name
import Core.Name.CompatibleVars

import Data.SnocList
import Data.SnocList.HasLength
import Libraries.Data.SnocList.HasLength
import Libraries.Data.SnocList.SizeOf
import Libraries.Data.List.SizeOf

Expand Down

0 comments on commit b2542e3

Please sign in to comment.