Skip to content

Commit

Permalink
Removing extra trailing whitespace.
Browse files Browse the repository at this point in the history
  • Loading branch information
Matthew-Mosior committed Jul 26, 2024
1 parent 704e80c commit 8e24f12
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/Idris/Package/Init.idr
Original file line number Diff line number Diff line change
Expand Up @@ -72,7 +72,7 @@ interactive : IO (Either () PkgDesc)
interactive = do
pname <- prompt "Package name: "
-- check to ensure that pname is a valid Idris2 identifier.
case checkPackageName $ fastUnpack pname of
case checkPackageName $ fastUnpack pname of
False => do () <- putStrLn "Package name is not a valid Idris Identifier."
pure $ Left ()
True => do pauthors <- prompt "Package authors: "
Expand All @@ -94,13 +94,13 @@ interactive = do
mstring str = case trim str of
"" => Nothing
str => Just str

isIdentStart : Char -> Bool
isIdentStart '_' = True
isIdentStart x = isUpper x ||
isAlpha x ||
x > chr 160

isIdentTrailing : List Char -> Bool
isIdentTrailing [] = True
isIdentTrailing (x::xs) = case isAlphaNum x ||
Expand Down

0 comments on commit 8e24f12

Please sign in to comment.