mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 08:11:45 +03:00
22 lines
408 B
Idris
22 lines
408 B
Idris
|
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
|