Skip to content

Commit

Permalink
fixed up CHANGELOG
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna committed Mar 17, 2024
1 parent 9b4ee0e commit 078d4f6
Showing 1 changed file with 5 additions and 18 deletions.
23 changes: 5 additions & 18 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -64,7 +64,7 @@ New modules
```agda
Algebra.Module.Construct.Idealization
```

* The unique morphism from the initial, resp. terminal, algebra:
```agda
Algebra.Morphism.Construct.Initial
Expand Down Expand Up @@ -171,7 +171,7 @@ Additions to existing modules
quasigroup : Quasigroup _ _
isLoop : IsLoop _∙_ _\\_ _//_ ε
loop : Loop _ _
\\-leftDividesˡ : LeftDividesˡ _∙_ _\\_
\\-leftDividesʳ : LeftDividesʳ _∙_ _\\_
\\-leftDivides : LeftDivides _∙_ _\\_
Expand All @@ -190,7 +190,7 @@ Additions to existing modules
identityʳ-unique : x ∙ y ≈ x → y ≈ ε
identity-unique : Identity x _∙_ → x ≈ ε
```

* In `Algebra.Properties.Monoid.Mult`:
```agda
×-homo-0 : ∀ x → 0 × x ≈ 0#
Expand All @@ -213,7 +213,7 @@ Additions to existing modules
_\\_ : Op₂ A
x \\ y = (x ⁻¹) ∙ y
```

* In `Data.Container.Indexed.Core`:
```agda
Subtrees o c = (r : Response c) → X (next c r)
Expand Down Expand Up @@ -315,7 +315,7 @@ Additions to existing modules
pred-injective : .{{NonZero m}} → .{{NonZero n}} → pred m ≡ pred n → m ≡ n
pred-cancel-≡ : pred m ≡ pred n → ((m ≡ 0 × n ≡ 1) ⊎ (m ≡ 1 × n ≡ 0)) ⊎ m ≡ n
```

* Added new proofs to `Data.Nat.Primality`:
```agda
rough∧square>⇒prime : .{{NonTrivial n}} → m Rough n → m * m > n → Prime n
Expand Down Expand Up @@ -378,16 +378,3 @@ Additions to existing modules
```agda
⌊⌋-map′ : (a? : Dec A) → ⌊ map′ t f a? ⌋ ≡ ⌊ a? ⌋
```

* Added module `Data.Vec.Functional.Relation.Binary.Permutation`:
```agda
_↭_ : IRel (Vector A) _
```

* Added new file `Data.Vec.Functional.Relation.Binary.Permutation.Properties`:
```agda
↭-refl : Reflexive (Vector A) _↭_
↭-reflexive : xs ≡ ys → xs ↭ ys
↭-sym : Symmetric (Vector A) _↭_
↭-trans : Transitive (Vector A) _↭_
```

0 comments on commit 078d4f6

Please sign in to comment.