Skip to content

Commit f702bee

Browse files
committed
add changelog entry
1 parent cc6addb commit f702bee

File tree

1 file changed

+7
-0
lines changed

1 file changed

+7
-0
lines changed

CHANGELOG.md

Lines changed: 7 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -736,6 +736,13 @@ Additions to existing modules
736736
toVec : (as : Vec≤ A n) → Vec A (Vec≤.length as)
737737
```
738738

739+
* Added new proofs to `Data.Vec.Relation.Binary.Equality.Cast`:
740+
```agda
741+
≈-cong′ : ∀ {f-len : ℕ → ℕ} (f : ∀ {n} → Vec A n → Vec B (f-len n))
742+
{m n} {xs : Vec A m} {ys : Vec A n} .{eq} →
743+
xs ≈[ eq ] ys → f xs ≈[ _ ] f ys
744+
```
745+
739746
* In `Data.Word64.Base`:
740747
```agda
741748
_≤_ : Rel Word64 zero

0 commit comments

Comments
 (0)