File tree Expand file tree Collapse file tree 1 file changed +14
-0
lines changed Expand file tree Collapse file tree 1 file changed +14
-0
lines changed Original file line number Diff line number Diff line change @@ -48,6 +48,11 @@ New modules
48
48
Additions to existing modules
49
49
-----------------------------
50
50
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
+
51
56
* In ` Data.List.Properties ` :
52
57
``` agda
53
58
product≢0 : All NonZero ns → NonZero (product ns)
@@ -93,6 +98,15 @@ Additions to existing modules
93
98
_≡?_ : DecidableEquality (Vec A n)
94
99
```
95
100
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
+
96
110
* In ` Relation.Nullary.Decidable ` :
97
111
``` agda
98
112
does-⇔ : A ⇔ B → (a? : Dec A) → (b? : Dec B) → does a? ≡ does b?
You can’t perform that action at this time.
0 commit comments