We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
1 parent 387a130 commit 09530bdCopy full SHA for 09530bd
CHANGELOG.md
@@ -540,6 +540,13 @@ Additions to existing modules
540
map-concat : map f (concat xss) ≡ concat (map (map f) xss)
541
```
542
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
+
550
* In `Data.Vec.Relation.Binary.Equality.DecPropositional`:
551
```agda
552
_≡?_ : DecidableEquality (Vec A n)
0 commit comments