[ lint ] remove trailing whitespace

This commit is contained in:
Guillaume Allais 2021-01-16 14:26:55 +00:00
parent 25def217fb
commit fb77a3e043
4 changed files with 5 additions and 4 deletions

View File

@ -23,4 +23,5 @@ doSort (S k) = do let xs = sort $ randishInts 12000 $ natToInteger k
main : IO ()
main = do max <- getLine
doSort (integerToNat (cast max))
doSort (integerToNat (cast max))

View File

@ -19,7 +19,7 @@ doSort (S k) = do Right dict<-readFile "words"
-- sort reversed list and get last word
putStrLn $ show $ mylast $ sort xs
doSort k
main : IO ()
main = do max <- getLine
doSort (integerToNat (cast max))

View File

@ -3,7 +3,7 @@ import Data.Strings
import Data.List
main : IO ()
main = do
main = do
putStrLn "input file: "
file<-getLine
Right tocheck<-readFile file

View File

@ -620,7 +620,7 @@ docsOrSignature fc n
let ns@(_ :: _) = concatMap (\n => lookupName n (docstrings syn))
(map fst all)
| [] => typeSummary defs
getDocsFor fc n
getDocsFor fc n
where
typeSummary : Defs -> Core (List String)
typeSummary defs = do Just def <- lookupCtxtExact n (gamma defs)