1
1
mirror of https://github.com/idris-lang/Idris2.git synced 2025-01-08 08:52:22 +03:00
Idris2/tests/idris2/basic042/LiteralsString.idr

22 lines
408 B
Idris
Raw Normal View History

import Data.Maybe
%default total
FromString Int where
fromString x = cast x
test1 : Int
test1 = "42"
test2 : Int
test2 = "abc"
convert : String -> Maybe Bool
convert "True" = Just True
convert "False" = Just False
convert _ = Nothing
fromString : (str : String) -> {auto prf : IsJust (convert str)} -> Bool
fromString str {prf} with (convert str)
fromString str {prf = ItIsJust} | (Just ret) = ret