Skip to content

Commit 0dd231d

Browse files
authored
Get rid of redundant dependencies in System.Console.ANSI (#1994)
1 parent a5b3564 commit 0dd231d

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

src/Data/Nat/Show.agda

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,7 @@ open import Data.Maybe.Base as Maybe using (Maybe; nothing; _<∣>_; when)
1717
import Data.Maybe.Effectful as Maybe
1818
open import Data.Nat
1919
open import Data.Product using (proj₁)
20-
open import Data.String as String using (String)
20+
open import Data.String.Base using (toList; fromList; String)
2121
open import Function.Base
2222
open import Relation.Nullary.Decidable using (True)
2323

@@ -28,7 +28,7 @@ readMaybe : ∀ base {base≤16 : True (base ≤? 16)} → String → Maybe ℕ
2828
readMaybe _ "" = nothing
2929
readMaybe base = Maybe.map convert
3030
∘′ TraversableA.mapA Maybe.applicative readDigit
31-
∘′ String.toList
31+
∘′ toList
3232

3333
where
3434

@@ -62,7 +62,7 @@ toDecimalChars : ℕ → List Char
6262
toDecimalChars = List.map toDigitChar ∘′ toNatDigits 10
6363

6464
show : String
65-
show = String.fromList ∘ toDecimalChars
65+
show = fromList ∘ toDecimalChars
6666

6767
-- Arbitrary base betwen 2 & 16.
6868
-- Warning: when compiled the time complexity of `showInBase b n` is
@@ -81,5 +81,5 @@ showInBase : (base : ℕ)
8181
{base≥2 : True (2 ≤? base)}
8282
{base≤16 : True (base ≤? 16)}
8383
String
84-
showInBase base {base≥2} {base≤16} = String.fromList
84+
showInBase base {base≥2} {base≤16} = fromList
8585
∘ charsInBase base {base≥2} {base≤16}

0 commit comments

Comments
 (0)