Skip to content

Commit f4316e1

Browse files
authoredMar 24, 2024··
Include CHANGELOG in fix-whitespace and whitespace fixes (#2325)
1 parent 36ea6ac commit f4316e1

File tree

7 files changed

+23
-24
lines changed

7 files changed

+23
-24
lines changed
 

‎CHANGELOG/v2.0.md

+10-10
Original file line numberDiff line numberDiff line change
@@ -38,7 +38,7 @@ Bug-fixes
3838
Consequently this field has been removed from the record, and the record
3939
`IsRingWithoutAnnihilatingZero` in `Algebra.Structures.Biased` has been
4040
deprecated as it is now identical to is `IsRing`.
41-
41+
4242
* In `Algebra.Definitions.RawSemiring` the record `Prime` did not
4343
enforce that the number was not divisible by `1#`. To fix this
4444
`p∤1 : p ∤ 1#` has been added as a field.
@@ -212,7 +212,7 @@ Non-backwards compatible changes
212212

213213
* Added new aliases `Is(Meet/Join)(Bounded)Semilattice` for `Is(Bounded)Semilattice`
214214
which can be used to indicate meet/join-ness of the original structures, and
215-
the field names in `IsSemilattice` and `Semilattice` have been renamed from
215+
the field names in `IsSemilattice` and `Semilattice` have been renamed from
216216
`∧-cong` to `∙-cong`to indicate their undirected nature.
217217

218218
* Finally, the following auxiliary files have been moved:
@@ -763,10 +763,10 @@ Non-backwards compatible changes
763763
- The records in `Function.Structures` and `Function.Bundles` export proofs
764764
of these under the names `strictlySurjective`, `strictlyInverseˡ` and
765765
`strictlyInverseʳ`,
766-
- Conversion functions for the definitions have been added in both directions
767-
to `Function.Consequences(.Propositional/Setoid)`.
768-
- Conversion functions for structures have been added in
769-
`Function.Structures.Biased`.
766+
- Conversion functions for the definitions have been added in both directions
767+
to `Function.Consequences(.Propositional/Setoid)`.
768+
- Conversion functions for structures have been added in
769+
`Function.Structures.Biased`.
770770
771771
### New `Function.Strict`
772772
@@ -852,9 +852,9 @@ Non-backwards compatible changes
852852

853853
4. The modules `Relation.Nullary.(Product/Sum/Implication)` have been deprecated
854854
and their contents moved to `Relation.Nullary.(Negation/Reflects/Decidable)`.
855-
855+
856856
5. The proof `T?` has been moved from `Data.Bool.Properties` to `Relation.Nullary.Decidable.Core`
857-
(but is still re-exported by the former).
857+
(but is still re-exported by the former).
858858

859859
as well as the following breaking changes:
860860

@@ -1214,7 +1214,7 @@ Other major improvements
12141214

12151215
* We have then moved raw bundles defined in `Data.X.Properties` to `Data.X.Base` for
12161216
`X` = `Nat`/`Nat.Binary`/`Integer`/`Rational`/`Rational.Unnormalised`.
1217-
1217+
12181218
### Upgrades to `README` sub-library
12191219

12201220
* The `README` sub-library has been moved to `doc/README` and a new `doc/standard-library-doc.agda-lib` has been added.
@@ -1223,7 +1223,7 @@ Other major improvements
12231223
using an out-of-the-box standard Agda installation without altering the main
12241224
`standard-library.agda-lib` file.
12251225

1226-
* The second is that the `README` files are now their own first-class library
1226+
* The second is that the `README` files are now their own first-class library
12271227
and can be imported like an other library.
12281228

12291229
Deprecated modules

‎HACKING.md

+1-1
Original file line numberDiff line numberDiff line change
@@ -31,7 +31,7 @@ Note on contributions to related/'coupled' modules
3131
==================================================
3232

3333
Before making changes to a `Data` module please have a look at related modules
34-
and see if they have any content along similar lines. If so, then please
34+
and see if they have any content along similar lines. If so, then please
3535
follow those conventions (e.g. naming, argument order).
3636
For example, if working on `Data.Rational`, please check `Data.Rational.Unnormalised`
3737
or if working on `Data.Vec` please check `Data.List` and vice versa.

‎fix-whitespace.yaml

+1-2
Original file line numberDiff line numberDiff line change
@@ -7,5 +7,4 @@ included-files:
77
- "*.md"
88

99
excluded-files:
10-
- "README/Text/Tabular.agda"
11-
- CHANGELOG.md
10+
- "README/Text/Tabular.agda"

‎src/Algebra/Module/Bundles/Raw.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -200,7 +200,7 @@ record RawBimodule (R : Set r) (S : Set s) m ℓm : Set (r ⊔ s ⊔ suc (m ⊔
200200
; 0ᴹ = 0ᴹ
201201
; -ᴹ_ = -ᴹ_
202202
}
203-
203+
204204
rawRightModule : RawRightModule S m ℓm
205205
rawRightModule = record
206206
{ _≈ᴹ_ = _≈ᴹ_

‎src/Algebra/Morphism/Construct/Initial.agda

+2-2
Original file line numberDiff line numberDiff line change
@@ -39,7 +39,7 @@ zero ()
3939
-- Basic properties
4040

4141
cong : (≈ : Rel A ℓm) Rel.Homomorphic₂ ℤero.Carrier A ℤero._≈_ ≈ zero
42-
cong _ {x = ()}
42+
cong _ {x = ()}
4343

4444
injective : (≈ : Rel A ℓm) Injective ℤero._≈_ ≈ zero
4545
injective _ {x = ()}
@@ -52,7 +52,7 @@ isMagmaHomomorphism : (M : RawMagma m ℓm) →
5252
isMagmaHomomorphism M = record
5353
{ isRelHomomorphism = record { cong = cong (RawMagma._≈_ M) }
5454
; homo = λ()
55-
}
55+
}
5656

5757
isMagmaMonomorphism : (M : RawMagma m ℓm)
5858
IsMagmaMonomorphism rawMagma M zero

‎src/Data/List/Relation/Ternary/Appending/Setoid/Properties.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -23,7 +23,7 @@ open import Relation.Binary.PropositionalEquality.Core using (refl)
2323
open import Relation.Binary.Construct.Composition using (_;_)
2424

2525
open Setoid S renaming (Carrier to A)
26-
open import Relation.Binary.Properties.Setoid S using (≈;≈⇒≈; ≈⇒≈;≈)
26+
open import Relation.Binary.Properties.Setoid S using (≈;≈⇒≈; ≈⇒≈;≈)
2727
open import Data.List.Relation.Ternary.Appending.Setoid S
2828

2929
private

‎src/Data/Nat/Primality/Factorisation.agda

+7-7
Original file line numberDiff line numberDiff line change
@@ -34,7 +34,7 @@ open import Relation.Binary.PropositionalEquality using (_≡_; refl; sym; trans
3434
private
3535
variable
3636
n :
37-
37+
3838
------------------------------------------------------------------------
3939
-- Core definition
4040

@@ -107,18 +107,18 @@ factorise n₀@(2+ _) = build [ <-recBuilder ⊗ <-recBuilder ] P facRec (n₀ ,
107107
pred (m * m) <⟨ s<s⁻¹ (m∸n≢0⇒n<m λ eq′ 0≢1+n (trans (sym eq′) eq)) ⟩
108108
n ∎
109109
where open ≤-Reasoning
110-
110+
111111
q = quotient m∣n
112-
112+
113113
instance _ = n>1⇒nonTrivial (quotient>1 m∣n m<n)
114-
114+
115115
factorisation[q] : PrimeFactorisation q
116116
factorisation[q] = recQuotient (quotient-< m∣n) (suc q ∸ m * m) (rough∧∣⇒rough rough (quotient-∣ m∣n)) refl
117-
117+
118118
ps = factors factorisation[q]
119-
119+
120120
primes = factorsPrime factorisation[q]
121-
121+
122122
m*Πps≡n : m * product ps ≡ n
123123
m*Πps≡n = begin
124124
m * product ps ≡⟨ cong (m *_) (isFactorisation factorisation[q]) ⟨

0 commit comments

Comments
 (0)
Please sign in to comment.