Skip to content

Commit 81230ec

Browse files
fix whitespace
1 parent 1af553e commit 81230ec

File tree

3 files changed

+6
-6
lines changed

3 files changed

+6
-6
lines changed

CHANGELOG.md

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -42,7 +42,7 @@ Un-deprecated modules
4242
* The modules `Function.Endomorphism.Propositional` and
4343
`Function.Endomorphism.Setoid` previously used the old `Function`
4444
hierarchy but have now been ported to using the new one.
45-
45+
4646
Deprecated names
4747
----------------
4848

@@ -186,7 +186,7 @@ Additions to existing modules
186186
IsSemigroupMonomorphism : (A → B) → Set _
187187
IsSemigroupIsomorphism : (A → B) → Set _
188188
```
189-
189+
190190
* In `Algebra.Properties.Group`:
191191
```agda
192192
isQuasigroup : IsQuasigroup _∙_ _\\_ _//_

src/Function/Endomorphism/Propositional.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -97,7 +97,7 @@ private
9797
{ isRelHomomorphism = record { cong = cong (f ^_) }
9898
; homo = ^-homo f
9999
}
100-
100+
101101
^-isMonoidMorphism : f IsMonoidHomomorphism +-0-rawMonoid ∘-id-rawMonoid (f ^_)
102102
^-isMonoidMorphism f = record
103103
{ isMagmaHomomorphism = ^-isSemigroupMorphism f

src/Function/Endomorphism/Setoid.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -43,7 +43,7 @@ infixr 8 _^_
4343
private
4444
id : Endo
4545
id = identity S
46-
46+
4747
_^_ : Endo Endo
4848
f ^ zero = id
4949
f ^ suc n = f ∘ (f ^ n)
@@ -62,7 +62,7 @@ f ^ suc n = f ∘ (f ^ n)
6262
∘-isMagma : IsMagma _≈_ _∘_
6363
∘-isMagma = record
6464
{ isEquivalence = isEquivalence
65-
; ∙-cong = λ {_} {_} {_} {v} x≈y u≈v S.trans u≈v (cong v x≈y)
65+
; ∙-cong = λ {_} {_} {_} {v} x≈y u≈v S.trans u≈v (cong v x≈y)
6666
}
6767
where
6868
module S = Setoid S
@@ -94,7 +94,7 @@ private
9494

9595
∘-id-rawMonoid : RawMonoid (c ⊔ e) (c ⊔ e)
9696
∘-id-rawMonoid = Monoid.rawMonoid ∘-id-monoid
97-
97+
9898
------------------------------------------------------------------------
9999
-- Homomorphism
100100

0 commit comments

Comments
 (0)