Skip to content

Commit

Permalink
ScopedSnocList: WIP: a (b +%+ c) => a (c ++ b) but actually a speci…
Browse files Browse the repository at this point in the history
…al case for `elemInsertedMiddle`
  • Loading branch information
GulinSS committed Sep 23, 2024
1 parent 60e78dd commit f50ee80
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Core/Case/CaseBuilder.idr
Original file line number Diff line number Diff line change
Expand Up @@ -688,7 +688,7 @@ zeroedScore nps = Scored nps (replicate (S $ length ps) 0)
||| Proof that a value `v` inserted in the middle of a list with
||| prefix `ps` and suffix `qs` can equivalently be snoced with
||| `ps` or consed with `qs` before appending `qs` to `ps`.
elemInsertedMiddle : (v : a) -> (ps,qs : SnocList a) -> (ps +%+ (qs :< v)) = ((ps `snoc` v) +%+ qs)
elemInsertedMiddle : (v : a) -> (ps,qs : SnocList a) -> ((qs :< v) ++ ps) = (qs ++ (ps `snoc` v))
elemInsertedMiddle v [<] qs = Refl
elemInsertedMiddle v (xs :< x) qs = rewrite elemInsertedMiddle v xs qs in Refl

Expand Down

0 comments on commit f50ee80

Please sign in to comment.