File tree Expand file tree Collapse file tree 1 file changed +5
-5
lines changed
Expand file tree Collapse file tree 1 file changed +5
-5
lines changed Original file line number Diff line number Diff line change @@ -53,7 +53,7 @@ Deprecated names
5353 ∣-respˡ ↦ ∣-respˡ-≈
5454 ∣-respʳ ↦ ∣-respʳ-≈
5555 ∣-resp ↦ ∣-resp-≈
56- ```
56+ ```
5757
5858* In ` Algebra.Solver.CommutativeMonoid ` :
5959 ``` agda
@@ -293,12 +293,12 @@ Additions to existing modules
293293 ``` agda
294294 Env : ℕ → Set _
295295 Env = Vec Carrier
296- ```
296+ ```
297297
298298* In ` Algebra.Structures.RingWithoutOne ` :
299299 ``` agda
300300 isNearSemiring : IsNearSemiring _ _
301- ```
301+ ```
302302
303303* In ` Data.List.Membership.Propositional.Properties ` :
304304 ``` agda
@@ -544,7 +544,7 @@ Additions to existing modules
544544 ``` agda
545545 value-injective : value v ≡ value w → v ≡ w
546546 _≟_ : DecidableEquality A → DecidableEquality [ x ∈ A ∣ P x ]
547- ```
547+ ```
548548
549549* New lemma in ` Data.Vec.Properties ` :
550550 ``` agda
@@ -570,7 +570,7 @@ Additions to existing modules
570570 ×-distribˡ-⊎ : (A × (B ⊎ C)) ↔ (A × B ⊎ A × C)
571571 ×-distribʳ-⊎ : ((A ⊎ B) × C) ↔ (A × C ⊎ B × C)
572572 ∃-≡ : ∀ (P : A → Set b) {x} → P x ↔ (∃[ y ] y ≡ x × P y)
573- ```
573+ ```
574574
575575* In ` Relation.Binary.Bundles ` :
576576 ``` agda
You can’t perform that action at this time.
0 commit comments