{-# OPTIONS_GHC -Wunused-imports #-}
module Agda.TypeChecking.Empty
( isEmptyType
, isEmptyTel
, ensureEmptyType
, checkEmptyTel
) where
import Control.Monad.Except ( MonadError(..) )
import Data.Semigroup
import Agda.Syntax.Common
import Agda.Syntax.Internal
import Agda.Syntax.Internal.MetaVars
import Agda.Syntax.Position
import Agda.TypeChecking.Monad
import Agda.TypeChecking.Coverage
import Agda.TypeChecking.Coverage.Match ( fromSplitPatterns )
import Agda.TypeChecking.Records
import Agda.TypeChecking.Reduce ( instantiateFull )
import Agda.TypeChecking.Substitute
import Agda.TypeChecking.Telescope
import Agda.Utils.Either
import Agda.Utils.List
import Agda.Utils.Monad
import Agda.Utils.Impossible
data ErrorNonEmpty
= Fail
| FailBecause TCErr
| DontKnow Blocker
instance Semigroup ErrorNonEmpty where
DontKnow Blocker
u1 <> :: ErrorNonEmpty -> ErrorNonEmpty -> ErrorNonEmpty
<> DontKnow Blocker
u2 = Blocker -> ErrorNonEmpty
DontKnow (Blocker -> ErrorNonEmpty) -> Blocker -> ErrorNonEmpty
forall a b. (a -> b) -> a -> b
$ Blocker -> Blocker -> Blocker
unblockOnBoth Blocker
u1 Blocker
u2
e :: ErrorNonEmpty
e@DontKnow{} <> ErrorNonEmpty
_ = ErrorNonEmpty
e
ErrorNonEmpty
_ <> e :: ErrorNonEmpty
e@DontKnow{} = ErrorNonEmpty
e
FailBecause TCErr
err <> ErrorNonEmpty
_ = TCErr -> ErrorNonEmpty
FailBecause TCErr
err
ErrorNonEmpty
Fail <> ErrorNonEmpty
err = ErrorNonEmpty
err
instance Monoid ErrorNonEmpty where
mempty :: ErrorNonEmpty
mempty = ErrorNonEmpty
Fail
mappend :: ErrorNonEmpty -> ErrorNonEmpty -> ErrorNonEmpty
mappend = ErrorNonEmpty -> ErrorNonEmpty -> ErrorNonEmpty
forall a. Semigroup a => a -> a -> a
(Data.Semigroup.<>)
ensureEmptyType
:: Range
-> Type
-> TCM ()
ensureEmptyType :: Range -> Type -> TCM ()
ensureEmptyType Range
r Type
t = TCMT IO (Either ErrorNonEmpty ())
-> (ErrorNonEmpty -> TCM ()) -> (() -> TCM ()) -> TCM ()
forall (m :: * -> *) a b c.
Monad m =>
m (Either a b) -> (a -> m c) -> (b -> m c) -> m c
caseEitherM (Range -> Type -> TCMT IO (Either ErrorNonEmpty ())
checkEmptyType Range
r Type
t) ErrorNonEmpty -> TCM ()
failure () -> TCM ()
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return
where
failure :: ErrorNonEmpty -> TCM ()
failure (DontKnow Blocker
u) = Blocker -> Constraint -> TCM ()
forall (m :: * -> *).
MonadConstraint m =>
Blocker -> Constraint -> m ()
addConstraint Blocker
u (Constraint -> TCM ()) -> Constraint -> TCM ()
forall a b. (a -> b) -> a -> b
$ Range -> Type -> Constraint
IsEmpty Range
r Type
t
failure (FailBecause TCErr
err) = TCErr -> TCM ()
forall a. TCErr -> TCMT IO a
forall e (m :: * -> *) a. MonadError e m => e -> m a
throwError TCErr
err
failure ErrorNonEmpty
Fail = TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM ()) -> TypeError -> TCM ()
forall a b. (a -> b) -> a -> b
$ Type -> [DeBruijnPattern] -> TypeError
ShouldBeEmpty Type
t []
isEmptyType :: Type -> TCM Bool
isEmptyType :: Type -> TCM Bool
isEmptyType Type
ty = Either ErrorNonEmpty () -> Bool
forall a b. Either a b -> Bool
isRight (Either ErrorNonEmpty () -> Bool)
-> TCMT IO (Either ErrorNonEmpty ()) -> TCM Bool
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Range -> Type -> TCMT IO (Either ErrorNonEmpty ())
checkEmptyType Range
forall a. Range' a
noRange Type
ty
isEmptyTel :: Telescope -> TCM Bool
isEmptyTel :: Tele (Dom' Term Type) -> TCM Bool
isEmptyTel Tele (Dom' Term Type)
tel = Either ErrorNonEmpty Int -> Bool
forall a b. Either a b -> Bool
isRight (Either ErrorNonEmpty Int -> Bool)
-> TCMT IO (Either ErrorNonEmpty Int) -> TCM Bool
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Range
-> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
checkEmptyTel Range
forall a. Range' a
noRange Tele (Dom' Term Type)
tel
checkEmptyType :: Range -> Type -> TCM (Either ErrorNonEmpty ())
checkEmptyType :: Range -> Type -> TCMT IO (Either ErrorNonEmpty ())
checkEmptyType Range
range Type
t = do
mr <- Type -> TCMT IO (Either (Blocked Type) (QName, Args, RecordData))
forall (m :: * -> *).
PureTCM m =>
Type -> m (Either (Blocked Type) (QName, Args, RecordData))
tryRecordType Type
t
case mr of
Left (Blocked Blocker
b Type
t) -> Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ()))
-> Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a b. (a -> b) -> a -> b
$ ErrorNonEmpty -> Either ErrorNonEmpty ()
forall a b. a -> Either a b
Left (Blocker -> ErrorNonEmpty
DontKnow Blocker
b)
Left (NotBlocked NotBlocked' Term
nb Type
t) -> do
tel0 <- TCMT IO (Tele (Dom' Term Type))
forall (m :: * -> *).
(Applicative m, MonadTCEnv m) =>
m (Tele (Dom' Term Type))
getContextTelescope
let gamma = Tele (Dom' Term Type) -> [Dom (ArgName, Type)]
forall t. Tele (Dom t) -> [Dom (ArgName, t)]
telToList Tele (Dom' Term Type)
tel0 [Dom (ArgName, Type)]
-> [Dom (ArgName, Type)] -> [Dom (ArgName, Type)]
forall a. [a] -> [a] -> [a]
++ [Arg (ArgName, Type) -> Dom (ArgName, Type)
forall a. Arg a -> Dom a
domFromArg (Arg (ArgName, Type) -> Dom (ArgName, Type))
-> Arg (ArgName, Type) -> Dom (ArgName, Type)
forall a b. (a -> b) -> a -> b
$ (ArgName, Type) -> Arg (ArgName, Type)
forall a. a -> Arg a
defaultArg (ArgName
forall a. Underscore a => a
underscore, Type
t)]
tel = [Dom (ArgName, Type)] -> Tele (Dom' Term Type)
telFromList [Dom (ArgName, Type)]
gamma
ps = Tele (Dom' Term Type) -> [NamedArg DeBruijnPattern]
forall a t. DeBruijn a => Tele (Dom t) -> [NamedArg a]
teleNamedArgs Tele (Dom' Term Type)
tel
dontAssignMetas $ do
r <- splitLast Inductive tel ps
case r of
Left UnificationStuck{} -> do
blocker <- Tele (Dom' Term Type) -> Blocker
forall t. AllMetas t => t -> Blocker
unblockOnAnyMetaIn (Tele (Dom' Term Type) -> Blocker)
-> TCMT IO (Tele (Dom' Term Type)) -> TCMT IO Blocker
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Tele (Dom' Term Type) -> TCMT IO (Tele (Dom' Term Type))
forall a (m :: * -> *).
(InstantiateFull a, MonadReduce m) =>
a -> m a
instantiateFull Tele (Dom' Term Type)
tel
return $ Left $ DontKnow blocker
Left SplitError
_ -> Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ()))
-> Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a b. (a -> b) -> a -> b
$ ErrorNonEmpty -> Either ErrorNonEmpty ()
forall a b. a -> Either a b
Left ErrorNonEmpty
Fail
Right Covering
cov -> do
let ps :: [DeBruijnPattern]
ps = (SplitClause -> DeBruijnPattern)
-> [SplitClause] -> [DeBruijnPattern]
forall a b. (a -> b) -> [a] -> [b]
map (NamedArg DeBruijnPattern -> DeBruijnPattern
forall a. NamedArg a -> a
namedArg (NamedArg DeBruijnPattern -> DeBruijnPattern)
-> (SplitClause -> NamedArg DeBruijnPattern)
-> SplitClause
-> DeBruijnPattern
forall b c a. (b -> c) -> (a -> b) -> a -> c
. NamedArg DeBruijnPattern
-> [NamedArg DeBruijnPattern] -> NamedArg DeBruijnPattern
forall a. a -> [a] -> a
lastWithDefault NamedArg DeBruijnPattern
forall a. HasCallStack => a
__IMPOSSIBLE__ ([NamedArg DeBruijnPattern] -> NamedArg DeBruijnPattern)
-> (SplitClause -> [NamedArg DeBruijnPattern])
-> SplitClause
-> NamedArg DeBruijnPattern
forall b c a. (b -> c) -> (a -> b) -> a -> c
. [NamedArg SplitPattern] -> [NamedArg DeBruijnPattern]
fromSplitPatterns ([NamedArg SplitPattern] -> [NamedArg DeBruijnPattern])
-> (SplitClause -> [NamedArg SplitPattern])
-> SplitClause
-> [NamedArg DeBruijnPattern]
forall b c a. (b -> c) -> (a -> b) -> a -> c
. SplitClause -> [NamedArg SplitPattern]
scPats) ([SplitClause] -> [DeBruijnPattern])
-> [SplitClause] -> [DeBruijnPattern]
forall a b. (a -> b) -> a -> b
$ Covering -> [SplitClause]
splitClauses Covering
cov
if ([DeBruijnPattern] -> Bool
forall a. [a] -> Bool
forall (t :: * -> *) a. Foldable t => t a -> Bool
null [DeBruijnPattern]
ps) then Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (() -> Either ErrorNonEmpty ()
forall a b. b -> Either a b
Right ()) else
ErrorNonEmpty -> Either ErrorNonEmpty ()
forall a b. a -> Either a b
Left (ErrorNonEmpty -> Either ErrorNonEmpty ())
-> (TCErr -> ErrorNonEmpty) -> TCErr -> Either ErrorNonEmpty ()
forall b c a. (b -> c) -> (a -> b) -> a -> c
. TCErr -> ErrorNonEmpty
FailBecause (TCErr -> Either ErrorNonEmpty ())
-> TCMT IO TCErr -> TCMT IO (Either ErrorNonEmpty ())
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> do TypeError -> TCMT IO TCErr
forall (m :: * -> *).
(HasCallStack, MonadTCEnv m, ReadTCState m) =>
TypeError -> m TCErr
typeError_ (TypeError -> TCMT IO TCErr) -> TypeError -> TCMT IO TCErr
forall a b. (a -> b) -> a -> b
$ Type -> [DeBruijnPattern] -> TypeError
ShouldBeEmpty Type
t [DeBruijnPattern]
ps
Right (QName
r, Args
pars, RecordData
def) -> do
if Bool -> Bool
not (RecordData -> Bool
isEtaRecordDef RecordData
def) then Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ()))
-> Either ErrorNonEmpty () -> TCMT IO (Either ErrorNonEmpty ())
forall a b. (a -> b) -> a -> b
$ ErrorNonEmpty -> Either ErrorNonEmpty ()
forall a b. a -> Either a b
Left ErrorNonEmpty
Fail else
Either ErrorNonEmpty Int -> Either ErrorNonEmpty ()
forall (f :: * -> *) a. Functor f => f a -> f ()
void (Either ErrorNonEmpty Int -> Either ErrorNonEmpty ())
-> TCMT IO (Either ErrorNonEmpty Int)
-> TCMT IO (Either ErrorNonEmpty ())
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> do Range
-> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
checkEmptyTel Range
range (Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int))
-> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
forall a b. (a -> b) -> a -> b
$ RecordData -> Tele (Dom' Term Type)
_recTel RecordData
def Tele (Dom' Term Type) -> Args -> Tele (Dom' Term Type)
forall t. Apply t => t -> Args -> t
`apply` Args
pars
checkEmptyTel :: Range -> Telescope -> TCM (Either ErrorNonEmpty Int)
checkEmptyTel :: Range
-> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
checkEmptyTel Range
r = Int -> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
loop Int
0
where
loop :: Int -> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
loop Int
i Tele (Dom' Term Type)
EmptyTel = Either ErrorNonEmpty Int -> TCMT IO (Either ErrorNonEmpty Int)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Either ErrorNonEmpty Int -> TCMT IO (Either ErrorNonEmpty Int))
-> Either ErrorNonEmpty Int -> TCMT IO (Either ErrorNonEmpty Int)
forall a b. (a -> b) -> a -> b
$ ErrorNonEmpty -> Either ErrorNonEmpty Int
forall a b. a -> Either a b
Left ErrorNonEmpty
Fail
loop Int
i (ExtendTel Dom' Term Type
dom Abs (Tele (Dom' Term Type))
tel) = [TCMT IO (Either ErrorNonEmpty Int)]
-> TCMT IO (Either ErrorNonEmpty Int)
forall e (m :: * -> *) b.
(Monoid e, Monad m, Functor m) =>
[m (Either e b)] -> m (Either e b)
orEitherM
[ (Int
i Int -> Either ErrorNonEmpty () -> Either ErrorNonEmpty Int
forall a b. a -> Either ErrorNonEmpty b -> Either ErrorNonEmpty a
forall (f :: * -> *) a b. Functor f => a -> f b -> f a
<$) (Either ErrorNonEmpty () -> Either ErrorNonEmpty Int)
-> TCMT IO (Either ErrorNonEmpty ())
-> TCMT IO (Either ErrorNonEmpty Int)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Range -> Type -> TCMT IO (Either ErrorNonEmpty ())
checkEmptyType Range
r (Dom' Term Type -> Type
forall t e. Dom' t e -> e
unDom Dom' Term Type
dom)
, Dom' Term Type
-> Abs (Tele (Dom' Term Type))
-> (Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int))
-> TCMT IO (Either ErrorNonEmpty Int)
forall a (m :: * -> *) b.
(Subst a, MonadAddContext m) =>
Dom' Term Type -> Abs a -> (a -> m b) -> m b
underAbstraction Dom' Term Type
dom Abs (Tele (Dom' Term Type))
tel ((Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int))
-> TCMT IO (Either ErrorNonEmpty Int))
-> (Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int))
-> TCMT IO (Either ErrorNonEmpty Int)
forall a b. (a -> b) -> a -> b
$ Int -> Tele (Dom' Term Type) -> TCMT IO (Either ErrorNonEmpty Int)
loop (Int -> Int
forall a. Enum a => a -> a
succ Int
i)
]