Skip to content

Commit fc473ec

Browse files
jamesmckinnagallais
authored andcommitted
cosmetic: two whitespace violations
1 parent cd70bc2 commit fc473ec

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/Data/List/Properties.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -872,7 +872,7 @@ module _ {R : Rel A p} (R? : B.Decidable R) where
872872
length-derun : xs length (derun R? xs) ≤ length xs
873873
length-derun [] = ≤-refl
874874
length-derun (x ∷ []) = ≤-refl
875-
length-derun (x ∷ y ∷ xs) with ih length-derun (y ∷ xs) | does (R? x y)
875+
length-derun (x ∷ y ∷ xs) with ih length-derun (y ∷ xs) | does (R? x y)
876876
... | true = m≤n⇒m≤1+n ih
877877
... | false = s≤s ih
878878

src/Data/Nat/Combinatorics.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ open import Data.Nat.Base
1212
open import Data.Nat.DivMod
1313
open import Data.Nat.Divisibility
1414
open import Data.Nat.Properties
15-
open import Relation.Binary.Definitions
15+
open import Relation.Binary.Definitions
1616
open import Relation.Binary.PropositionalEquality
1717
using (_≡_; refl; sym; cong; subst)
1818

@@ -118,7 +118,7 @@ module _ {n k} (k<n : k < n) where
118118

119119
[n-k]! = [n-k] !
120120
[n-k-1]! = [n-k-1] !
121-
121+
122122
[n-k]≡1+[n-k-1] : [n-k] ≡ suc [n-k-1]
123123
[n-k]≡1+[n-k-1] = +-∸-assoc 1 k<n
124124

0 commit comments

Comments
 (0)