Skip to content

Commit 8c21248

Browse files
committed
Normalize whitespace everywhere
1 parent 6d67409 commit 8c21248

File tree

28 files changed

+151
-152
lines changed

28 files changed

+151
-152
lines changed

.github/workflows/nix-ci.yml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -63,4 +63,4 @@ jobs:
6363
- name: drop into the devshell and run cabal
6464
# for some reason this doesn't work without update
6565
# even though it doesn't actually download anything
66-
run: nix develop -Lv -c bash -c "cabal update; cabal v1-build"
66+
run: nix develop -Lv -c bash -c "cabal update; cabal v1-build"

.readthedocs.yaml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,4 +11,4 @@ sphinx:
1111
# Explicitly set the version of Python and its requirements
1212
python:
1313
install:
14-
- requirements: docs/requirements.txt
14+
- requirements: docs/requirements.txt

docs/source/features.md

Lines changed: 10 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -32,7 +32,7 @@ Standard data type declarations have a simple equivalent in Agda.
3232
Agda:
3333
```agda
3434
data Nat : Type where
35-
Zero : Nat
35+
Zero : Nat
3636
Suc : Nat Nat
3737

3838
{-# COMPILE AGDA2HS Nat #-}
@@ -52,7 +52,7 @@ Agda:
5252
data Tree (a : Type) : Type where
5353
Leaf : a Tree a
5454
Branch : a Tree a Tree a Tree a
55-
55+
5656
{-# COMPILE AGDA2HS Tree #-}
5757
```
5858

@@ -197,7 +197,7 @@ negate True = False
197197
negate False = True
198198

199199
negate' :: Bool -> Bool
200-
negate' x = case x of
200+
negate' x = case x of
201201
True -> False
202202
False -> True
203203

@@ -260,7 +260,7 @@ createRange low high = if low <= high then Just (MkRange low high) else Nothing
260260
{-# COMPILE AGDA2HS createRange #-}
261261
262262
createRangeCase : Int → Int → Maybe Range
263-
createRangeCase low high =
263+
createRangeCase low high =
264264
case low <= high of λ where
265265
True → Just (MkRange low high)
266266
False → Nothing
@@ -393,7 +393,7 @@ open Equal public
393393
{-# COMPILE AGDA2HS Equal newtype #-}
394394
395395
constructEqual : ⦃ iEqA : Eq a ⦄ → @0 ⦃ IsLawfulEq a ⦄ → (c : a) → (d : a) → Maybe (Equal a)
396-
constructEqual a b =
396+
constructEqual a b =
397397
if a == b then
398398
(λ ⦃ h ⦄ → Just (MkEqual (a , b) (equality a b h)))
399399
else Nothing
@@ -475,10 +475,10 @@ record Class2 (a : Type) : Type where
475475
Haskell:
476476
```hs
477477
class Class1 a where
478-
field1 :: a
478+
field1 :: a
479479

480480
class Class1 a => Class2 a where
481-
field2 :: a
481+
field2 :: a
482482
```
483483

484484
### Default Typeclass Field Implementations
@@ -507,7 +507,7 @@ open Ord ⦃ ... ⦄
507507

508508
{-# COMPILE AGDA2HS Ord class Ord₁ Ord₂ #-}
509509

510-
instance
510+
instance
511511
Ord-Bool : OrdBool
512512
Ord-Bool .Ord._<_ False b = b
513513
Ord-Bool .Ord._<_ True _ = False
@@ -701,7 +701,7 @@ add1 = 1 +_
701701

702702
Haskell:
703703
```hs
704-
add1 :: Nat -> Nat
704+
add1 :: Nat -> Nat
705705
add1 = (1 +)
706706
```
707707

@@ -729,7 +729,7 @@ even (Suc n) = odd n
729729

730730
odd :: Nat -> Bool
731731
odd Zero = False
732-
odd (Suc n) = even n
732+
odd (Suc n) = even n
733733
```
734734

735735
### Mutually Recursive Datatype and Function

docs/source/tutorials.md

Lines changed: 69 additions & 69 deletions
Large diffs are not rendered by default.

lib/base/Haskell/Law/Applicative/List.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ private
2626
rewrite sym $ concatMap-++-distr (map (u ∘_) v) (((pure _∘_) <*> us) <*> v) (λ f map f w)
2727
| sym $ map-<*>-recomp v w u
2828
| compositionList us v w
29-
= refl
29+
= refl
3030

3131
interchangeList : {a b : Type} (u : List (a b)) (y : a)
3232
(u <*> (pure y)) ≡ (pure (_$ y) <*> u)

lib/base/Haskell/Law/Int.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,4 +6,4 @@ open import Haskell.Prim.Int using ( int64 )
66
open import Haskell.Law.Def
77

88
int64-injective : Injective int64
9-
int64-injective refl = refl
9+
int64-injective refl = refl

lib/base/Haskell/Law/List.agda

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ open import Haskell.Prim.Applicative
1212
--------------------------------------------------
1313
-- _∷_
1414

15-
module _ {x y : a} {xs ys : List a} where
15+
module _ {x y : a} {xs ys : List a} where
1616
∷-injective-left : x ∷ xs ≡ y ∷ ys x ≡ y
1717
∷-injective-left refl = refl
1818

@@ -40,14 +40,14 @@ map-∘ g f (x ∷ xs) = cong (_ ∷_) (map-∘ g f xs)
4040

4141
map-concatMap : (f : a b) (xs : List a) (map f xs) ≡ concatMap (λ g f g ∷ []) xs
4242
map-concatMap f [] = refl
43-
map-concatMap f (x ∷ xs)
43+
map-concatMap f (x ∷ xs)
4444
rewrite map-concatMap f xs
4545
= refl
4646

47-
map-<*>-recomp : {a b c : Type} (xs : List (a b)) (ys : List a) (u : (b c))
47+
map-<*>-recomp : {a b c : Type} (xs : List (a b)) (ys : List a) (u : (b c))
4848
((map (u ∘_) xs) <*> ys) ≡ map u (xs <*> ys)
4949
map-<*>-recomp [] _ _ = refl
50-
map-<*>-recomp (x ∷ xs) ys u
50+
map-<*>-recomp (x ∷ xs) ys u
5151
rewrite map-∘ u x ys
5252
| map-++ u (map x ys) (xs <*> ys)
5353
| map-<*>-recomp xs ys u
@@ -102,7 +102,7 @@ lengthNat-++ (x ∷ xs) = cong suc (lengthNat-++ xs)
102102
++-cancel-right [] [] eq = refl
103103
++-cancel-right (x ∷ xs) [] eq = ++-identity-left-unique (x ∷ xs) (sym eq)
104104
++-cancel-right [] (y ∷ ys) eq = sym $ ++-identity-left-unique (y ∷ ys) eq
105-
++-cancel-right (x ∷ xs) (y ∷ ys) eq
105+
++-cancel-right (x ∷ xs) (y ∷ ys) eq
106106
rewrite ∷-injective-left eq = cong (y ∷_) $ ++-cancel-right xs ys (∷-injective-right eq)
107107

108108
++-conical-left : (xs ys : List a) xs ++ ys ≡ [] xs ≡ []
@@ -114,7 +114,7 @@ lengthNat-++ (x ∷ xs) = cong suc (lengthNat-++ xs)
114114
∷-not-identity : x (xs ys : List a) (x ∷ xs) ++ ys ≡ ys
115115
∷-not-identity x xs ys eq = []≠∷ x xs (sym $ ++-identity-left-unique (x ∷ xs) (sym eq))
116116

117-
concatMap-++-distr : (xs ys : List a) (f : a List b)
117+
concatMap-++-distr : (xs ys : List a) (f : a List b)
118118
((concatMap f xs) ++ (concatMap f ys)) ≡ (concatMap f (xs ++ ys))
119119
concatMap-++-distr [] ys f = refl
120120
concatMap-++-distr (x ∷ xs) ys f
@@ -129,7 +129,7 @@ foldr-universal : ∀ (h : List a → b) f e → (h [] ≡ e) →
129129
( x xs h (x ∷ xs) ≡ f x (h xs))
130130
xs h xs ≡ foldr f e xs
131131
foldr-universal h f e base step [] = base
132-
foldr-universal h f e base step (x ∷ xs) rewrite step x xs = cong (f x) (foldr-universal h f e base step xs)
132+
foldr-universal h f e base step (x ∷ xs) rewrite step x xs = cong (f x) (foldr-universal h f e base step xs)
133133

134134
foldr-cong : {f g : a b b} {d e : b}
135135
( x y f x y ≡ g x y) d ≡ e

lib/base/Haskell/Law/Monoid/Maybe.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,6 +16,6 @@ instance
1616
iLawfulMonoidMaybe .leftIdentity = λ { Nothing refl; (Just _) refl }
1717

1818
iLawfulMonoidMaybe .concatenation [] = refl
19-
iLawfulMonoidMaybe .concatenation (x ∷ xs)
19+
iLawfulMonoidMaybe .concatenation (x ∷ xs)
2020
rewrite (concatenation xs)
2121
= refl

lib/base/Haskell/Law/Num/Integer.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -290,7 +290,7 @@ instance
290290
iLawfulNumInteger .IsLawfulNum.+-idˡ x = addInteger-idˡ x
291291
iLawfulNumInteger .IsLawfulNum.+-idʳ x = addInteger-idʳ x
292292
iLawfulNumInteger .IsLawfulNum.neg-inv x = n-n≡0-Integer x
293-
iLawfulNumInteger .IsLawfulNum.*-assoc = mulInteger-assoc
293+
iLawfulNumInteger .IsLawfulNum.*-assoc = mulInteger-assoc
294294
iLawfulNumInteger .IsLawfulNum.*-idˡ x = mulInteger-idˡ x
295295
iLawfulNumInteger .IsLawfulNum.*-idʳ x = mulInteger-idʳ x
296296
iLawfulNumInteger .IsLawfulNum.distributeˡ = mulInteger-distributeˡ-addInteger

lib/base/Haskell/Law/Num/Word.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -61,7 +61,7 @@ addWord-comm : Commutative addWord
6161
addWord-comm = map-comm addWord addNat w2n n2w (embedding +-wordsAsNats) addNat-comm
6262

6363
addWord-assoc : Associative addWord
64-
addWord-assoc = map-assoc addWord addNat w2n n2w (embedding +-wordsAsNats) addNat-assoc
64+
addWord-assoc = map-assoc addWord addNat w2n n2w (embedding +-wordsAsNats) addNat-assoc
6565

6666
mulWord-comm : Commutative mulWord
6767
mulWord-comm = map-comm mulWord mulNat w2n n2w (embedding *-wordsAsNats) mulNat-comm

0 commit comments

Comments
 (0)