Skip to content

Commit 6c22327

Browse files
committed
[ changelog ] document new functions in Data.Product
1 parent 409af12 commit 6c22327

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

CHANGELOG.md

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -426,6 +426,16 @@ Other minor additions
426426
recompute : .(Coprime n d) → Coprime n d
427427
```
428428

429+
* Added new functions to `Data.Product`:
430+
```agda
431+
dmap : (f : (a : A) → B a) → (∀ {a} (p : P a) → Q p (f a)) →
432+
(ap : Σ A P) → Σ (B (proj₁ ap)) (Q (proj₂ ap))
433+
dmap : ((a : A) → X a) → ((b : B) → Y b) →
434+
(ab : A × B) → X (proj₁ ab) × Y (proj₂ ab)
435+
_<*>_ : ((a : A) → X a) × ((b : B) → Y b) →
436+
((a , b) : A × B) → X a × Y b
437+
```
438+
429439
* Made first argument of `[,]-∘-distr` in `Data.Sum.Properties` explicit
430440

431441
* Added new proofs to `Data.Sum.Properties`:

0 commit comments

Comments
 (0)