Skip to content

Commit 98843ee

Browse files
committed
[ fix ] whitespace violations
1 parent 7eaabc2 commit 98843ee

File tree

3 files changed

+4
-4
lines changed

3 files changed

+4
-4
lines changed

doc/README/Design/Hierarchies.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -265,7 +265,7 @@ record Semigroup : Set (suc (a ⊔ ℓ)) where
265265
-- IsA A
266266
-- / || \ / || \
267267
-- IsB IsC IsD B C D
268-
268+
269269
-- The procedure for re-exports in the bundles is as follows:
270270

271271
-- 1. `open IsA isA public using (IsC, M)` where `M` is everything
@@ -280,7 +280,7 @@ record Semigroup : Set (suc (a ⊔ ℓ)) where
280280

281281
-- 5. `open B b public using (O)` where `O` is everything exported
282282
-- by `B` but not exported by `IsA`.
283-
283+
284284
-- 6. Construct `d : D` via the `isC` obtained in step 1.
285285

286286
-- 7. `open D d public using (P)` where `P` is everything exported

src/Effect/Applicative.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -56,7 +56,7 @@ record RawApplicative (F : Set f → Set g) : Set (suc f ⊔ g) where
5656
-- Haskell-style alternative name for pure
5757
return : A F A
5858
return = pure
59-
59+
6060
-- backwards compatibility: unicode variants
6161
_⊛_ : F (A B) F A F B
6262
_⊛_ = _<*>_

src/Function/Bundles.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -380,7 +380,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
380380
-- For further background on (split) surjections, one may consult any
381381
-- general mathematical references which work without the principle
382382
-- of choice. For example:
383-
--
383+
--
384384
-- https://ncatlab.org/nlab/show/split+epimorphism.
385385
--
386386
-- The connection to set-theoretic notions with the same names is

0 commit comments

Comments
 (0)