mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 08:11:45 +03:00
22bfa90971
If the "can't convert" error arises from a mismatch between a type constructor and a primitive value, it is not recoverable.
14 lines
250 B
Idris
14 lines
250 B
Idris
module Sing
|
|
|
|
%default total
|
|
|
|
data Fing : Type -> Type where
|
|
StringFing : String -> Fing String
|
|
BoolFing : Bool -> Fing Bool
|
|
|
|
stringFing : Fing String -> String
|
|
stringFing (StringFing s) = s
|
|
|
|
boolFing : Fing Bool -> Bool
|
|
boolFing (BoolFing b) = b
|