mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 09:12:34 +03:00
12 lines
180 B
Idris
12 lines
180 B
Idris
import Data.Singleton
|
|
|
|
%default total
|
|
|
|
-- data constructors
|
|
f : Singleton (MkPair True) -> Bool
|
|
f (Val _) = True
|
|
|
|
-- type constructors
|
|
g : Singleton Maybe -> Bool
|
|
g (Val _) = True
|