Skip to content

Commit

Permalink
Fix the indentation of a few lines in CHANGELOG
Browse files Browse the repository at this point in the history
  • Loading branch information
shhyou committed Jan 3, 2025
1 parent d85cd7e commit 602b623
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -53,7 +53,7 @@ Deprecated names
∣-respˡ ↦ ∣-respˡ-≈
∣-respʳ ↦ ∣-respʳ-≈
∣-resp ↦ ∣-resp-≈
```
```

* In `Algebra.Solver.CommutativeMonoid`:
```agda
Expand Down Expand Up @@ -293,12 +293,12 @@ Additions to existing modules
```agda
Env : ℕ → Set _
Env = Vec Carrier
```
```

* In `Algebra.Structures.RingWithoutOne`:
```agda
isNearSemiring : IsNearSemiring _ _
```
```

* In `Data.List.Membership.Propositional.Properties`:
```agda
Expand Down Expand Up @@ -544,7 +544,7 @@ Additions to existing modules
```agda
value-injective : value v ≡ value w → v ≡ w
_≟_ : DecidableEquality A → DecidableEquality [ x ∈ A ∣ P x ]
```
```

* New lemma in `Data.Vec.Properties`:
```agda
Expand All @@ -570,7 +570,7 @@ Additions to existing modules
×-distribˡ-⊎ : (A × (B ⊎ C)) ↔ (A × B ⊎ A × C)
×-distribʳ-⊎ : ((A ⊎ B) × C) ↔ (A × C ⊎ B × C)
∃-≡ : ∀ (P : A → Set b) {x} → P x ↔ (∃[ y ] y ≡ x × P y)
```
```

* In `Relation.Binary.Bundles`:
```agda
Expand Down

0 comments on commit 602b623

Please sign in to comment.