Skip to content

Commit f8f19ec

Browse files
Merge pull request #1286 from laMudri/product-changelog
2 parents 82a6826 + 6c22327 commit f8f19ec

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
@@ -433,6 +433,16 @@ Other minor additions
433433
recompute : .(Coprime n d) → Coprime n d
434434
```
435435

436+
* Added new functions to `Data.Product`:
437+
```agda
438+
dmap : (f : (a : A) → B a) → (∀ {a} (p : P a) → Q p (f a)) →
439+
(ap : Σ A P) → Σ (B (proj₁ ap)) (Q (proj₂ ap))
440+
dmap : ((a : A) → X a) → ((b : B) → Y b) →
441+
(ab : A × B) → X (proj₁ ab) × Y (proj₂ ab)
442+
_<*>_ : ((a : A) → X a) × ((b : B) → Y b) →
443+
((a , b) : A × B) → X a × Y b
444+
```
445+
436446
* Made first argument of `[,]-∘-distr` in `Data.Sum.Properties` explicit
437447

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

0 commit comments

Comments
 (0)