Skip to content

Commit 8582957

Browse files
authored
Fix typo and whitespace violation (#2104)
1 parent 2c5e590 commit 8582957

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

src/Data/Container/FreeMonad.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -47,7 +47,7 @@ infix 1 _⋆_
4747
------------------------------------------------------------------------
4848
-- Type definition
4949

50-
-- The free moand can be defined as the least fixpoint `μ (C ⋆C X)`
50+
-- The free monad can be defined as the least fixpoint `μ (C ⋆C X)`
5151

5252
_⋆C_ : {x s p} Container s p Set x Container (s ⊔ x) p
5353
C ⋆C X = const X ⊎ C

src/Data/Vec/Base.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -272,7 +272,7 @@ drop m xs = proj₁ (proj₂ (splitAt m xs))
272272
group : n k (xs : Vec A (n * k))
273273
λ (xss : Vec (Vec A k) n) xs ≡ concat xss
274274
group zero k [] = ([] , refl)
275-
group (suc n) k xs =
275+
group (suc n) k xs =
276276
let ys , zs , eq-split = splitAt k xs in
277277
let zss , eq-group = group n k zs in
278278
(ys ∷ zss) , trans eq-split (cong (ys ++_) eq-group)

0 commit comments

Comments
 (0)