We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent cc6addb commit f702beeCopy full SHA for f702bee
CHANGELOG.md
@@ -736,6 +736,13 @@ Additions to existing modules
736
toVec : (as : Vec≤ A n) → Vec A (Vec≤.length as)
737
```
738
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
+
746
* In `Data.Word64.Base`:
747
```agda
748
_≤_ : Rel Word64 zero
0 commit comments