Skip to content

Commit 09530bd

Browse files
committed
add changelog entry
1 parent 387a130 commit 09530bd

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

CHANGELOG.md

+7
Original file line numberDiff line numberDiff line change
@@ -540,6 +540,13 @@ Additions to existing modules
540540
map-concat : map f (concat xss) ≡ concat (map (map f) xss)
541541
```
542542

543+
* New lemma in `Data.Vec.Relation.Binary.Equality.Cast`:
544+
```agda
545+
≈-cong′ : ∀ {f-len : ℕ → ℕ} (f : ∀ {n} → Vec A n → Vec B (f-len n))
546+
{m n} {xs : Vec A m} {ys : Vec A n} .{eq} →
547+
xs ≈[ eq ] ys → f xs ≈[ _ ] f ys
548+
```
549+
543550
* In `Data.Vec.Relation.Binary.Equality.DecPropositional`:
544551
```agda
545552
_≡?_ : DecidableEquality (Vec A n)

0 commit comments

Comments
 (0)