Skip to content

Commit e6f51de

Browse files
committed
Add new functions to CHANGELOG
1 parent e468b94 commit e6f51de

File tree

1 file changed

+14
-0
lines changed

1 file changed

+14
-0
lines changed

CHANGELOG.md

Lines changed: 14 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -48,6 +48,11 @@ New modules
4848
Additions to existing modules
4949
-----------------------------
5050

51+
* In `Data.Product.Function.Dependent.Propositional`:
52+
```agda
53+
cong′ : ∀ {k} → (∀ {x} → A x ∼[ k ] B x) → Σ I A ∼[ k ] Σ I B
54+
```
55+
5156
* In `Data.List.Properties`:
5257
```agda
5358
product≢0 : All NonZero ns → NonZero (product ns)
@@ -93,6 +98,15 @@ Additions to existing modules
9398
_≡?_ : DecidableEquality (Vec A n)
9499
```
95100

101+
* In `Function.Related.TypeIsomorphisms`:
102+
```agda
103+
Σ-distribˡ-⊎ : {P : A → Set a} {Q : A → Set b} → (∃ λ a → P a ⊎ Q a) ↔ (∃ P ⊎ ∃ Q)
104+
Σ-distribʳ-⊎ : {P : Set a} {Q : Set b} {R : P ⊎ Q → Set c} → (Σ (P ⊎ Q) R) ↔ (Σ P (R ∘ inj₁) ⊎ Σ Q (R ∘ inj₂))
105+
×-distribˡ-⊎′ : (A × (B ⊎ C)) ↔ (A × B ⊎ A × C)
106+
×-distribʳ-⊎′ : ((A ⊎ B) × C) ↔ (A × C ⊎ B × C)
107+
∃-≡ : ∀ (P : A → Set b) {x} → P x ↔ (∃[ y ] y ≡ x × P y)
108+
```
109+
96110
* In `Relation.Nullary.Decidable`:
97111
```agda
98112
does-⇔ : A ⇔ B → (a? : Dec A) → (b? : Dec B) → does a? ≡ does b?

0 commit comments

Comments
 (0)