{-# LANGUAGE NondecreasingIndentation #-}
module Agda.TypeChecking.Rules.Term where
import Prelude hiding ( null )
import Control.Monad.Except ( MonadError(..) )
import Data.Maybe
import Data.Either (partitionEithers, lefts)
import qualified Data.List as List
import qualified Data.Map as Map
import qualified Data.Set as Set
import Agda.Interaction.Options
import Agda.Interaction.Highlighting.Generate (disambiguateRecordFields)
import Agda.Syntax.Abstract (Binder, TypedBindingInfo (tbTacticAttr))
import qualified Agda.Syntax.Abstract as A
import Agda.Syntax.Abstract.Views as A
import qualified Agda.Syntax.Info as A
import Agda.Syntax.Concrete.Pretty ()
import Agda.Syntax.Concrete (FieldAssignment'(..), nameFieldA, TacticAttribute'(..))
import qualified Agda.Syntax.Concrete.Name as C
import Agda.Syntax.Common
import Agda.Syntax.Common.Pretty ( prettyShow )
import qualified Agda.Syntax.Common.Pretty as P
import Agda.Syntax.Internal as I
import Agda.Syntax.Internal.MetaVars
import Agda.Syntax.Position
import Agda.Syntax.Literal
import Agda.Syntax.Scope.Base ( ThingsInScope, AbstractName
, emptyScopeInfo
, exportedNamesInScope)
import Agda.Syntax.Scope.Monad (getNamedScope)
import Agda.TypeChecking.CompiledClause
import Agda.TypeChecking.Constraints
import Agda.TypeChecking.Conversion
import Agda.TypeChecking.Coverage.SplitTree
import Agda.TypeChecking.Datatypes
import Agda.TypeChecking.EtaContract
import Agda.TypeChecking.Generalize
import Agda.TypeChecking.Implicit
import Agda.TypeChecking.InstanceArguments
import Agda.TypeChecking.Irrelevance
import Agda.TypeChecking.IApplyConfluence
import Agda.TypeChecking.Level
import Agda.TypeChecking.MetaVars
import Agda.TypeChecking.Monad
import Agda.TypeChecking.Patterns.Abstract
import Agda.TypeChecking.Positivity.Occurrence
import Agda.TypeChecking.Pretty
import Agda.TypeChecking.Primitive
import Agda.TypeChecking.Quote
import Agda.TypeChecking.RecordPatterns
import Agda.TypeChecking.Records
import Agda.TypeChecking.Reduce
import Agda.TypeChecking.Rules.LHS
import Agda.TypeChecking.SizedTypes
import Agda.TypeChecking.SizedTypes.Solve
import Agda.TypeChecking.Sort
import Agda.TypeChecking.Substitute
import Agda.TypeChecking.Telescope
import Agda.TypeChecking.Unquote
import Agda.TypeChecking.Warnings
import {-# SOURCE #-} Agda.TypeChecking.Empty ( ensureEmptyType )
import {-# SOURCE #-} Agda.TypeChecking.Rules.Def (checkFunDef', useTerPragma)
import {-# SOURCE #-} Agda.TypeChecking.Rules.Decl (checkSectionApplication)
import {-# SOURCE #-} Agda.TypeChecking.Rules.Application
import Agda.Utils.Function
import Agda.Utils.Functor
import Agda.Utils.Lens
import Agda.Utils.List1 ( List1, pattern (:|) )
import Agda.Utils.List2 ( pattern List2 )
import qualified Agda.Utils.List1 as List1
import Agda.Utils.Maybe
import Agda.Utils.Monad
import Agda.Utils.Null
import qualified Agda.Utils.Set1 as Set1
import Agda.Utils.Singleton
import Agda.Utils.Size
import Agda.Utils.Tuple
import Agda.Utils.Impossible
isType :: A.Expr -> Sort -> TCM Type
isType :: Expr -> Sort' Term -> TCM Type
isType = Comparison -> Expr -> Sort' Term -> TCM Type
isType' Comparison
CmpLeq
isType' :: Comparison -> A.Expr -> Sort -> TCM Type
isType' :: Comparison -> Expr -> Sort' Term -> TCM Type
isType' Comparison
c Expr
e Sort' Term
s =
Call -> TCM Type -> TCM Type
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Comparison -> Expr -> Sort' Term -> Call
IsTypeCall Comparison
c Expr
e Sort' Term
s) (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ do
v <- Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
c Expr
e (Sort' Term -> Type
sort Sort' Term
s)
return $ El s v
isType_ :: A.Expr -> TCM Type
isType_ :: Expr -> TCM Type
isType_ Expr
e = Call -> TCM Type -> TCM Type
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Expr -> Call
IsType_ Expr
e) (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ do
ArgName -> Int -> (Type -> TCMT IO Doc) -> TCM Type -> TCM Type
forall (m :: * -> *) a.
MonadDebug m =>
ArgName -> Int -> (a -> TCMT IO Doc) -> m a -> m a
reportResult ArgName
"tc.term.istype" Int
15 (\Type
a -> [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"isType_" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<?> Expr -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Expr -> m Doc
prettyTCM Expr
e
, Int -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Functor m => Int -> m Doc -> m Doc
nest Int
2 (TCMT IO Doc -> TCMT IO Doc) -> TCMT IO Doc -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ TCMT IO Doc
"returns" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<?> Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
a
]) (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ do
let fallback :: TCM Type
fallback = Comparison -> Expr -> Sort' Term -> TCM Type
isType' Comparison
CmpEq Expr
e (Sort' Term -> TCM Type) -> TCMT IO (Sort' Term) -> TCM Type
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< do TCMT IO (Sort' Term) -> TCMT IO (Sort' Term)
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes (TCMT IO (Sort' Term) -> TCMT IO (Sort' Term))
-> TCMT IO (Sort' Term) -> TCMT IO (Sort' Term)
forall a b. (a -> b) -> a -> b
$ TCMT IO (Sort' Term)
forall (m :: * -> *). MonadMetaSolver m => m (Sort' Term)
newSortMeta
SortKit{..} <- TCMT IO SortKit
forall (m :: * -> *).
(HasBuiltins m, MonadTCError m, HasOptions m) =>
m SortKit
sortKit
case unScope e of
A.Fun ExprInfo
i (Arg ArgInfo
info Expr
t) Expr
b -> do
a <- ArgInfo -> Dom Type -> Dom Type
forall a. LensArgInfo a => ArgInfo -> a -> a
setArgInfo ArgInfo
info (Dom Type -> Dom Type) -> (Type -> Dom Type) -> Type -> Dom Type
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Type -> Dom Type
forall a. a -> Dom a
defaultDom (Type -> Dom Type) -> TCM Type -> TCMT IO (Dom Type)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> List1 ArgInfo -> Expr -> TCM Type
forall a.
(LensLock a, LensModality a) =>
List1 a -> Expr -> TCM Type
checkPiDomain (ArgInfo
info ArgInfo -> [ArgInfo] -> List1 ArgInfo
forall a. a -> [a] -> NonEmpty a
:| []) Expr
t
b <- isType_ b
s <- inferFunSort a (getSort b)
let t' = Sort' Term -> Term -> Type
forall t a. Sort' t -> a -> Type'' t a
El Sort' Term
s (Term -> Type) -> Term -> Type
forall a b. (a -> b) -> a -> b
$ Dom Type -> Abs Type -> Term
Pi Dom Type
a (Abs Type -> Term) -> Abs Type -> Term
forall a b. (a -> b) -> a -> b
$ ArgName -> Type -> Abs Type
forall a. ArgName -> a -> Abs a
NoAbs ArgName
forall a. Underscore a => a
underscore Type
b
checkTelePiSort t'
return t'
A.Pi ExprInfo
_ Telescope1
tel Expr
e -> do
(t0, t') <- Telescope -> (Telescope -> TCM (Type, Type)) -> TCM (Type, Type)
forall a. Telescope -> (Telescope -> TCM a) -> TCM a
checkPiTelescope (Telescope1 -> [Item Telescope1]
forall l. IsList l => l -> [Item l]
List1.toList Telescope1
tel) ((Telescope -> TCM (Type, Type)) -> TCM (Type, Type))
-> (Telescope -> TCM (Type, Type)) -> TCM (Type, Type)
forall a b. (a -> b) -> a -> b
$ \ Telescope
tel -> do
t0 <- Type -> TCM Type
forall a (m :: * -> *).
(InstantiateFull a, MonadReduce m) =>
a -> m a
instantiateFull (Type -> TCM Type) -> TCM Type -> TCM Type
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< Expr -> TCM Type
isType_ Expr
e
tel <- instantiateFull tel
return (t0, telePi tel t0)
checkTelePiSort t'
return t'
A.Generalized Set1 QName
s Expr
e -> do
(_, t') <- Set QName -> TCM Type -> TCM ([Maybe QName], Type)
generalizeType (Set1 QName -> Set QName
forall a. NESet a -> Set a
Set1.toSet Set1 QName
s) (TCM Type -> TCM ([Maybe QName], Type))
-> TCM Type -> TCM ([Maybe QName], Type)
forall a b. (a -> b) -> a -> b
$ Expr -> TCM Type
isType_ Expr
e
return t'
A.Def' QName
x Suffix
suffix
| Just (UnivSize
sz, Univ
u) <- QName -> Maybe (UnivSize, Univ)
isNameOfUniv QName
x
, let n :: Integer
n = Suffix -> Integer
suffixToLevel Suffix
suffix
-> do
Univ -> TCM ()
univChecks Univ
u
Type -> TCM Type
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Type -> TCM Type)
-> (Sort' Term -> Type) -> Sort' Term -> TCM Type
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Sort' Term -> Type
sort (Sort' Term -> TCM Type) -> Sort' Term -> TCM Type
forall a b. (a -> b) -> a -> b
$ case UnivSize
sz of
UnivSize
USmall -> Univ -> Level' Term -> Sort' Term
forall t. Univ -> Level' t -> Sort' t
Univ Univ
u (Level' Term -> Sort' Term) -> Level' Term -> Sort' Term
forall a b. (a -> b) -> a -> b
$ Integer -> Level' Term
ClosedLevel Integer
n
UnivSize
ULarge -> Univ -> Integer -> Sort' Term
forall t. Univ -> Integer -> Sort' t
Inf Univ
u Integer
n
A.App AppInfo
i Expr
s NamedArg Expr
arg
| NamedArg Expr -> Bool
forall a. LensHiding a => a -> Bool
visible NamedArg Expr
arg,
A.Def QName
x <- Expr -> Expr
unScope Expr
s,
Just (UnivSize
USmall, Univ
u) <- QName -> Maybe (UnivSize, Univ)
isNameOfUniv QName
x -> do
Univ -> TCM ()
univChecks Univ
u
TCMT IO Bool -> TCM () -> TCM ()
forall (m :: * -> *). Monad m => m Bool -> m () -> m ()
unlessM TCMT IO Bool
forall (m :: * -> *). HasOptions m => m Bool
hasUniversePolymorphism (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
NeedOptionUniversePolymorphism
Relevance -> TCM Type -> TCM Type
forall (tcm :: * -> *) r a.
(MonadTCEnv tcm, LensRelevance r) =>
r -> tcm a -> tcm a
applyRelevanceToContext Relevance
shapeIrrelevant (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$
Sort' Term -> Type
sort (Sort' Term -> Type)
-> (Level' Term -> Sort' Term) -> Level' Term -> Type
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Univ -> Level' Term -> Sort' Term
forall t. Univ -> Level' t -> Sort' t
Univ Univ
u (Level' Term -> Type) -> TCMT IO (Level' Term) -> TCM Type
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> NamedArg Expr -> TCMT IO (Level' Term)
checkLevel NamedArg Expr
arg
A.QuestionMark MetaInfo
minfo InteractionId
ii -> TCMT IO (Maybe MetaId)
-> TCM Type -> (MetaId -> TCM Type) -> TCM Type
forall (m :: * -> *) a b.
Monad m =>
m (Maybe a) -> m b -> (a -> m b) -> m b
caseMaybeM (InteractionId -> TCMT IO (Maybe MetaId)
forall (m :: * -> *).
ReadTCState m =>
InteractionId -> m (Maybe MetaId)
lookupInteractionMeta InteractionId
ii) TCM Type
fallback ((MetaId -> TCM Type) -> TCM Type)
-> (MetaId -> TCM Type) -> TCM Type
forall a b. (a -> b) -> a -> b
$ \ MetaId
x -> do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.ip" Int
20 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
fsep
[ TCMT IO Doc
"Rechecking meta "
, MetaId -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => MetaId -> m Doc
prettyTCM MetaId
x
, ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc) -> ArgName -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ ArgName
" for interaction point " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ InteractionId -> ArgName
forall a. Show a => a -> ArgName
show InteractionId
ii
]
mv <- MetaId -> TCMT IO MetaVariable
forall (m :: * -> *).
(HasCallStack, MonadDebug m, ReadTCState m) =>
MetaId -> m MetaVariable
lookupLocalMeta MetaId
x
let s0 = Judgement MetaId -> Type
forall a. Judgement a -> Type
jMetaType (Judgement MetaId -> Type)
-> (MetaVariable -> Judgement MetaId) -> MetaVariable -> Type
forall b c a. (b -> c) -> (a -> b) -> a -> c
. MetaVariable -> Judgement MetaId
mvJudgement (MetaVariable -> Type) -> MetaVariable -> Type
forall a b. (a -> b) -> a -> b
$ MetaVariable
mv
let n = [ContextEntry] -> Int
forall a. [a] -> Int
forall (t :: * -> *) a. Foldable t => t a -> Int
length ([ContextEntry] -> Int)
-> (MetaVariable -> [ContextEntry]) -> MetaVariable -> Int
forall b c a. (b -> c) -> (a -> b) -> a -> c
. TCEnv -> [ContextEntry]
envContext (TCEnv -> [ContextEntry])
-> (MetaVariable -> TCEnv) -> MetaVariable -> [ContextEntry]
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Closure Range -> TCEnv
forall a. Closure a -> TCEnv
clEnv (Closure Range -> TCEnv)
-> (MetaVariable -> Closure Range) -> MetaVariable -> TCEnv
forall b c a. (b -> c) -> (a -> b) -> a -> c
. MetaInfo -> Closure Range
miClosRange (MetaInfo -> Closure Range)
-> (MetaVariable -> MetaInfo) -> MetaVariable -> Closure Range
forall b c a. (b -> c) -> (a -> b) -> a -> c
. MetaVariable -> MetaInfo
mvInfo (MetaVariable -> Int) -> MetaVariable -> Int
forall a b. (a -> b) -> a -> b
$ MetaVariable
mv
(vs, rest) <- splitAt n <$> getContextArgs
reportSDoc "tc.ip" 20 $ vcat
[ " s0 = " <+> prettyTCM s0
, " vs = " <+> prettyTCM vs
, " rest = " <+> prettyTCM rest
]
if (length vs /= n) then fallback else do
s1 <- reduce =<< piApplyM s0 vs
reportSDoc "tc.ip" 20 $ vcat
[ " s1 = " <+> prettyTCM s1
]
reportSDoc "tc.ip" 70 $ vcat
[ " s1 = " <+> text (show s1)
]
case unEl s1 of
Sort Sort' Term
s -> Type -> TCM Type
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Type -> TCM Type) -> Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ Sort' Term -> Term -> Type
forall t a. Sort' t -> a -> Type'' t a
El Sort' Term
s (Term -> Type) -> Term -> Type
forall a b. (a -> b) -> a -> b
$ MetaId -> Elims -> Term
MetaV MetaId
x (Elims -> Term) -> Elims -> Term
forall a b. (a -> b) -> a -> b
$ (Arg Term -> Elim) -> [Arg Term] -> Elims
forall a b. (a -> b) -> [a] -> [b]
map Arg Term -> Elim
forall a. Arg a -> Elim' a
Apply [Arg Term]
vs
Term
_ -> TCM Type
forall a. HasCallStack => a
__IMPOSSIBLE__
Expr
_ -> TCM Type
fallback
checkLevel :: NamedArg A.Expr -> TCM Level
checkLevel :: NamedArg Expr -> TCMT IO (Level' Term)
checkLevel NamedArg Expr
arg = do
lvl <- TCM Type
forall (m :: * -> *). (HasBuiltins m, MonadTCError m) => m Type
levelType
levelView =<< checkNamedArg arg lvl
isTypeEqualTo :: A.Expr -> Type -> TCM Type
isTypeEqualTo :: Expr -> Type -> TCM Type
isTypeEqualTo Expr
e0 Type
t = Expr -> TCM Expr
scopedExpr Expr
e0 TCM Expr -> (Expr -> TCM Type) -> TCM Type
forall a b. TCMT IO a -> (a -> TCMT IO b) -> TCMT IO b
forall (m :: * -> *) a b. Monad m => m a -> (a -> m b) -> m b
>>= \case
A.ScopedExpr{} -> TCM Type
forall a. HasCallStack => a
__IMPOSSIBLE__
A.Underscore MetaInfo
i | Maybe MetaId -> Bool
forall a. Maybe a -> Bool
isNothing (MetaInfo -> Maybe MetaId
A.metaNumber MetaInfo
i) -> Type -> TCM Type
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Type
t
Expr
e -> TCM Type -> TCM Type
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ do
t' <- Expr -> Sort' Term -> TCM Type
isType Expr
e (Type -> Sort' Term
forall a. LensSort a => a -> Sort' Term
getSort Type
t)
t' <$ leqType t t'
leqType_ :: Type -> Type -> TCM ()
leqType_ :: Type -> Type -> TCM ()
leqType_ Type
t Type
t' = TCM () -> TCM ()
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ Type -> Type -> TCM ()
forall (m :: * -> *). MonadConversion m => Type -> Type -> m ()
leqType Type
t Type
t'
checkGeneralizeTelescope ::
Maybe ModuleName
-> A.GeneralizeTelescope
-> ([Maybe Name] -> Telescope -> TCM a)
-> TCM a
checkGeneralizeTelescope :: forall a.
Maybe ModuleName
-> GeneralizeTelescope
-> ([Maybe Name] -> Telescope -> TCM a)
-> TCM a
checkGeneralizeTelescope Maybe ModuleName
mm (A.GeneralizeTel Map QName Name
vars Telescope
tel) =
((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a
tr (Map QName Name
-> (forall a1. (Telescope -> TCM a1) -> TCM a1)
-> ([Maybe Name] -> Telescope -> TCMT IO a)
-> TCMT IO a
forall a.
Map QName Name
-> (forall a1. (Telescope -> TCM a1) -> TCM a1)
-> ([Maybe Name] -> Telescope -> TCM a)
-> TCM a
generalizeTelescope Map QName Name
vars (Telescope -> (Telescope -> TCM a1) -> TCM a1
forall a. Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope Telescope
tel) (([Maybe Name] -> Telescope -> TCMT IO a) -> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a)
-> [Maybe Name] -> Telescope -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall b c a. (b -> c) -> (a -> b) -> a -> c
. (([Maybe Name], Telescope) -> TCMT IO a)
-> [Maybe Name] -> Telescope -> TCMT IO a
forall a b c. ((a, b) -> c) -> a -> b -> c
curry) ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name] -> Telescope -> TCMT IO a)
-> ([Maybe Name], Telescope) -> TCMT IO a)
-> ([Maybe Name] -> Telescope -> TCMT IO a)
-> TCMT IO a
forall b c a. (b -> c) -> (a -> b) -> a -> c
. ([Maybe Name] -> Telescope -> TCMT IO a)
-> ([Maybe Name], Telescope) -> TCMT IO a
forall a b c. (a -> b -> c) -> (a, b) -> c
uncurry
where
tr :: ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a
tr = Bool
-> (((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall b a. IsBool b => b -> (a -> a) -> a -> a
applyUnless (Telescope -> Bool
forall a. Null a => a -> Bool
null Telescope
tel) ((((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a)
-> (((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall a b. (a -> b) -> a -> b
$ Maybe ModuleName
-> (ModuleName
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall b a. Maybe b -> (b -> a -> a) -> a -> a
applyWhenJust Maybe ModuleName
mm ((ModuleName
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a)
-> (ModuleName
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a)
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall a b. (a -> b) -> a -> b
$ \ ModuleName
m ->
Call
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall a b.
Call
-> ((a -> TCMT IO b) -> TCMT IO b) -> (a -> TCMT IO b) -> TCMT IO b
forall (m :: * -> *) a b.
MonadTrace m =>
Call -> ((a -> m b) -> m b) -> (a -> m b) -> m b
traceCallCPS (Call
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a)
-> Call
-> ((([Maybe Name], Telescope) -> TCMT IO a) -> TCMT IO a)
-> (([Maybe Name], Telescope) -> TCMT IO a)
-> TCMT IO a
forall a b. (a -> b) -> a -> b
$ ModuleName -> Telescope -> Call
CheckModuleParameters ModuleName
m Telescope
tel
checkTelescope :: A.Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope :: forall a. Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope = LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
forall a. LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope' LamOrPi
LamNotPi
checkPiTelescope :: A.Telescope -> (Telescope -> TCM a) -> TCM a
checkPiTelescope :: forall a. Telescope -> (Telescope -> TCM a) -> TCM a
checkPiTelescope = LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
forall a. LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope' LamOrPi
PiNotLam
data LamOrPi
= LamNotPi
| PiNotLam
deriving (LamOrPi -> LamOrPi -> Bool
(LamOrPi -> LamOrPi -> Bool)
-> (LamOrPi -> LamOrPi -> Bool) -> Eq LamOrPi
forall a. (a -> a -> Bool) -> (a -> a -> Bool) -> Eq a
$c== :: LamOrPi -> LamOrPi -> Bool
== :: LamOrPi -> LamOrPi -> Bool
$c/= :: LamOrPi -> LamOrPi -> Bool
/= :: LamOrPi -> LamOrPi -> Bool
Eq, Int -> LamOrPi -> ArgName -> ArgName
[LamOrPi] -> ArgName -> ArgName
LamOrPi -> ArgName
(Int -> LamOrPi -> ArgName -> ArgName)
-> (LamOrPi -> ArgName)
-> ([LamOrPi] -> ArgName -> ArgName)
-> Show LamOrPi
forall a.
(Int -> a -> ArgName -> ArgName)
-> (a -> ArgName) -> ([a] -> ArgName -> ArgName) -> Show a
$cshowsPrec :: Int -> LamOrPi -> ArgName -> ArgName
showsPrec :: Int -> LamOrPi -> ArgName -> ArgName
$cshow :: LamOrPi -> ArgName
show :: LamOrPi -> ArgName
$cshowList :: [LamOrPi] -> ArgName -> ArgName
showList :: [LamOrPi] -> ArgName -> ArgName
Show)
checkTelescope' :: LamOrPi -> A.Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope' :: forall a. LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope' LamOrPi
lamOrPi [] Telescope -> TCM a
ret = Telescope -> TCM a
ret Telescope
forall a. Tele a
EmptyTel
checkTelescope' LamOrPi
lamOrPi (TypedBinding
b : Telescope
tel) Telescope -> TCM a
ret =
LamOrPi -> TypedBinding -> (Telescope -> TCM a) -> TCM a
forall a. LamOrPi -> TypedBinding -> (Telescope -> TCM a) -> TCM a
checkTypedBindings LamOrPi
lamOrPi TypedBinding
b ((Telescope -> TCM a) -> TCM a) -> (Telescope -> TCM a) -> TCM a
forall a b. (a -> b) -> a -> b
$ \Telescope
tel1 ->
LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
forall a. LamOrPi -> Telescope -> (Telescope -> TCM a) -> TCM a
checkTelescope' LamOrPi
lamOrPi Telescope
tel ((Telescope -> TCM a) -> TCM a) -> (Telescope -> TCM a) -> TCM a
forall a b. (a -> b) -> a -> b
$ \Telescope
tel2 ->
Telescope -> TCM a
ret (Telescope -> TCM a) -> Telescope -> TCM a
forall a b. (a -> b) -> a -> b
$ Telescope -> Telescope -> Telescope
forall t. Abstract t => Telescope -> t -> t
abstract Telescope
tel1 Telescope
tel2
checkDomain :: (LensLock a, LensModality a) => LamOrPi -> List1 a -> A.Expr -> TCM Type
checkDomain :: forall a.
(LensLock a, LensModality a) =>
LamOrPi -> List1 a -> Expr -> TCM Type
checkDomain LamOrPi
lamOrPi List1 a
xs Expr
e = do
let (Cohesion
c :| [Cohesion]
cs) = (a -> Cohesion) -> List1 a -> NonEmpty Cohesion
forall a b. (a -> b) -> NonEmpty a -> NonEmpty b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap (Modality -> Cohesion
forall a. LensCohesion a => a -> Cohesion
getCohesion (Modality -> Cohesion) -> (a -> Modality) -> a -> Cohesion
forall b c a. (b -> c) -> (a -> b) -> a -> c
. a -> Modality
forall a. LensModality a => a -> Modality
getModality) List1 a
xs
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless ((Cohesion -> Bool) -> [Cohesion] -> Bool
forall (t :: * -> *) a. Foldable t => (a -> Bool) -> t a -> Bool
all (Cohesion
c Cohesion -> Cohesion -> Bool
forall a. Eq a => a -> a -> Bool
==) [Cohesion]
cs) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ TCM ()
forall a. HasCallStack => a
__IMPOSSIBLE__
let (Quantity
q :| [Quantity]
qs) = (a -> Quantity) -> List1 a -> NonEmpty Quantity
forall a b. (a -> b) -> NonEmpty a -> NonEmpty b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap (Modality -> Quantity
forall a. LensQuantity a => a -> Quantity
getQuantity (Modality -> Quantity) -> (a -> Modality) -> a -> Quantity
forall b c a. (b -> c) -> (a -> b) -> a -> c
. a -> Modality
forall a. LensModality a => a -> Modality
getModality) List1 a
xs
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless ((Quantity -> Bool) -> [Quantity] -> Bool
forall (t :: * -> *) a. Foldable t => (a -> Bool) -> t a -> Bool
all (Quantity
q Quantity -> Quantity -> Bool
forall a. Eq a => a -> a -> Bool
==) [Quantity]
qs) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ TCM ()
forall a. HasCallStack => a
__IMPOSSIBLE__
t <- Quantity -> TCM Type -> TCM Type
forall (tcm :: * -> *) q a.
(MonadTCEnv tcm, LensQuantity q) =>
q -> tcm a -> tcm a
applyQuantityToJudgement Quantity
q (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$
Cohesion -> TCM Type -> TCM Type
forall (tcm :: * -> *) m a.
(MonadTCEnv tcm, LensCohesion m) =>
m -> tcm a -> tcm a
applyCohesionToContext Cohesion
c (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$
LamOrPi -> TCM Type -> TCM Type
forall {m :: * -> *} {a}.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
LamOrPi -> m a -> m a
modEnv LamOrPi
lamOrPi (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ Expr -> TCM Type
isType_ Expr
e
when (any (\a
x -> case a -> Lock
forall a. LensLock a => a -> Lock
getLock a
x of { IsLock{} -> Bool
True ; Lock
_ -> Bool
False }) xs) $ do
unlessM (isJust <$> getName' builtinLockUniv) $ do
typeError $ NoBindingForPrimitive builtinLockUniv
equalSort (getSort t) LockUniv
return t
where
modEnv :: LamOrPi -> m a -> m a
modEnv LamOrPi
LamNotPi = m a -> m a
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes
modEnv LamOrPi
_ = m a -> m a
forall a. a -> a
id
checkPiDomain :: (LensLock a, LensModality a) => List1 a -> A.Expr -> TCM Type
checkPiDomain :: forall a.
(LensLock a, LensModality a) =>
List1 a -> Expr -> TCM Type
checkPiDomain = LamOrPi -> List1 a -> Expr -> TCM Type
forall a.
(LensLock a, LensModality a) =>
LamOrPi -> List1 a -> Expr -> TCM Type
checkDomain LamOrPi
PiNotLam
checkTypedBindings :: LamOrPi -> A.TypedBinding -> (Telescope -> TCM a) -> TCM a
checkTypedBindings :: forall a. LamOrPi -> TypedBinding -> (Telescope -> TCM a) -> TCM a
checkTypedBindings LamOrPi
lamOrPi (A.TBind Range
r TypedBindingInfo
tac List1 (NamedArg (Binder' BindName))
xps Expr
e) Telescope -> TCM a
ret = do
let xs :: NonEmpty (NamedArg Name)
xs = (NamedArg (Binder' BindName) -> NamedArg Name)
-> List1 (NamedArg (Binder' BindName)) -> NonEmpty (NamedArg Name)
forall a b. (a -> b) -> NonEmpty a -> NonEmpty b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap ((Binder' BindName -> Name)
-> NamedArg (Binder' BindName) -> NamedArg Name
forall a b. (a -> b) -> NamedArg a -> NamedArg b
updateNamedArg ((Binder' BindName -> Name)
-> NamedArg (Binder' BindName) -> NamedArg Name)
-> (Binder' BindName -> Name)
-> NamedArg (Binder' BindName)
-> NamedArg Name
forall a b. (a -> b) -> a -> b
$ BindName -> Name
A.unBind (BindName -> Name)
-> (Binder' BindName -> BindName) -> Binder' BindName -> Name
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Binder' BindName -> BindName
forall a. Binder' a -> a
A.binderName) List1 (NamedArg (Binder' BindName))
xps
tac <- (Ranged Expr -> TCM Term)
-> Maybe (Ranged Expr) -> TCMT IO (Maybe Term)
forall (t :: * -> *) (f :: * -> *) a b.
(Traversable t, Applicative f) =>
(a -> f b) -> t a -> f (t b)
forall (f :: * -> *) a b.
Applicative f =>
(a -> f b) -> Maybe a -> f (Maybe b)
traverse (LamOrPi -> Ranged Expr -> TCM Term
checkTacticAttribute LamOrPi
lamOrPi) (Maybe (Ranged Expr) -> TCMT IO (Maybe Term))
-> Maybe (Ranged Expr) -> TCMT IO (Maybe Term)
forall a b. (a -> b) -> a -> b
$ TacticAttribute -> Maybe (Ranged Expr)
forall a. TacticAttribute' a -> Maybe (Ranged a)
theTacticAttribute (TacticAttribute -> Maybe (Ranged Expr))
-> TacticAttribute -> Maybe (Ranged Expr)
forall a b. (a -> b) -> a -> b
$ TypedBindingInfo -> TacticAttribute
tbTacticAttr TypedBindingInfo
tac
whenJust tac $ \ Term
t -> ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.tactic" Int
30 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ TCMT IO Doc
"Checked tactic attribute:" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<?> Term -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Term -> m Doc
prettyTCM Term
t
experimental <- optExperimentalIrrelevance <$> pragmaOptions
t <- checkDomain lamOrPi xps e
List1.unlessNull (List1.filter isInstance xps) $ \ List1 (NamedArg (Binder' BindName))
ixs -> do
(tel, _, target) <- Type -> TCM (Telescope, Term, OutputTypeName)
getOutputTypeName Type
t
case target of
OutputTypeName{} -> () -> TCM ()
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ()
OutputTypeVar{} -> () -> TCM ()
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ()
OutputTypeNameNotYetKnown{} -> () -> TCM ()
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ()
OutputTypeVisiblePi{} -> Expr -> TCM () -> TCM ()
forall (m :: * -> *) x a.
(MonadTrace m, HasRange x) =>
x -> m a -> m a
setCurrentRange Expr
e (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$
Warning -> TCM ()
forall (m :: * -> *).
(HasCallStack, MonadWarning m) =>
Warning -> m ()
warning (Warning -> TCM ()) -> (Doc -> Warning) -> Doc -> TCM ()
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Doc -> Warning
InstanceArgWithExplicitArg (Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TypedBinding -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => TypedBinding -> m Doc
prettyTCM (Range
-> List1 (NamedArg (Binder' BindName)) -> Expr -> TypedBinding
A.mkTBind Range
r List1 (NamedArg (Binder' BindName))
ixs Expr
e)
OutputTypeName
NoOutputTypeName -> Expr -> TCM () -> TCM ()
forall (m :: * -> *) x a.
(MonadTrace m, HasRange x) =>
x -> m a -> m a
setCurrentRange Expr
e (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$
Warning -> TCM ()
forall (m :: * -> *).
(HasCallStack, MonadWarning m) =>
Warning -> m ()
warning (Warning -> TCM ()) -> (Doc -> Warning) -> Doc -> TCM ()
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Doc -> Warning
InstanceNoOutputTypeName (Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TypedBinding -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => TypedBinding -> m Doc
prettyTCM (Range
-> List1 (NamedArg (Binder' BindName)) -> Expr -> TypedBinding
A.mkTBind Range
r List1 (NamedArg (Binder' BindName))
ixs Expr
e)
let setTac Maybe t
tac Tele (Dom' t e)
EmptyTel = Tele (Dom' t e)
forall a. Tele a
EmptyTel
setTac Maybe t
tac (ExtendTel Dom' t e
dom Abs (Tele (Dom' t e))
tel) = Dom' t e -> Abs (Tele (Dom' t e)) -> Tele (Dom' t e)
forall a. a -> Abs (Tele a) -> Tele a
ExtendTel Dom' t e
dom{ domTactic = tac } (Abs (Tele (Dom' t e)) -> Tele (Dom' t e))
-> Abs (Tele (Dom' t e)) -> Tele (Dom' t e)
forall a b. (a -> b) -> a -> b
$ Maybe t -> Tele (Dom' t e) -> Tele (Dom' t e)
setTac (Int -> Maybe t -> Maybe t
forall a. Subst a => Int -> a -> a
raise Int
1 Maybe t
tac) (Tele (Dom' t e) -> Tele (Dom' t e))
-> Abs (Tele (Dom' t e)) -> Abs (Tele (Dom' t e))
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Abs (Tele (Dom' t e))
tel
xs' = (NamedArg Name -> NamedArg Name)
-> NonEmpty (NamedArg Name) -> NonEmpty (NamedArg Name)
forall a b. (a -> b) -> NonEmpty a -> NonEmpty b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap (LamOrPi -> Bool -> NamedArg Name -> NamedArg Name
forall {b} {a}.
(IsBool b, LensRelevance a) =>
LamOrPi -> b -> a -> a
modMod LamOrPi
lamOrPi Bool
experimental) NonEmpty (NamedArg Name)
xs
let tel = Maybe Term -> Telescope -> Telescope
forall {t} {t} {e}.
Subst t =>
Maybe t -> Tele (Dom' t e) -> Tele (Dom' t e)
setTac Maybe Term
tac (Telescope -> Telescope) -> Telescope -> Telescope
forall a b. (a -> b) -> a -> b
$ NonEmpty (NamedArg Name) -> Type -> Telescope
namedBindsToTel1 NonEmpty (NamedArg Name)
xs Type
t
addContext (xs', t) $ addTypedPatterns xps (ret tel)
where
modEnv :: LamOrPi -> m a -> m a
modEnv LamOrPi
LamNotPi = m a -> m a
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes
modEnv LamOrPi
_ = m a -> m a
forall a. a -> a
id
modMod :: LamOrPi -> b -> a -> a
modMod LamOrPi
PiNotLam b
xp = b -> (a -> a) -> a -> a
forall b a. IsBool b => b -> (a -> a) -> a -> a
applyWhen b
xp ((a -> a) -> a -> a) -> (a -> a) -> a -> a
forall a b. (a -> b) -> a -> b
$ (Relevance -> Relevance) -> a -> a
forall a. LensRelevance a => (Relevance -> Relevance) -> a -> a
mapRelevance Relevance -> Relevance
irrelevantToShapeIrrelevant
modMod LamOrPi
_ b
_ = a -> a
forall a. a -> a
id
checkTypedBindings LamOrPi
lamOrPi (A.TLet Range
_ List1 LetBinding
lbs) Telescope -> TCM a
ret = do
List1 LetBinding -> TCM a -> TCM a
forall (t :: * -> *) a.
Foldable t =>
t LetBinding -> TCM a -> TCM a
checkLetBindings List1 LetBinding
lbs (Telescope -> TCM a
ret Telescope
forall a. Tele a
EmptyTel)
addTypedPatterns :: List1 (NamedArg A.Binder) -> TCM a -> TCM a
addTypedPatterns :: forall a. List1 (NamedArg (Binder' BindName)) -> TCM a -> TCM a
addTypedPatterns List1 (NamedArg (Binder' BindName))
xps TCM a
ret = do
let
ps :: [(Pattern, BindName)]
ps = (NamedArg (Binder' BindName) -> Maybe (Pattern, BindName))
-> List1 (NamedArg (Binder' BindName)) -> [(Pattern, BindName)]
forall a b. (a -> Maybe b) -> List1 a -> [b]
List1.mapMaybe (Binder' BindName -> Maybe (Pattern, BindName)
forall a. Binder' a -> Maybe (Pattern, a)
A.extractPattern (Binder' BindName -> Maybe (Pattern, BindName))
-> (NamedArg (Binder' BindName) -> Binder' BindName)
-> NamedArg (Binder' BindName)
-> Maybe (Pattern, BindName)
forall b c a. (b -> c) -> (a -> b) -> a -> c
. NamedArg (Binder' BindName) -> Binder' BindName
forall a. NamedArg a -> a
namedArg) List1 (NamedArg (Binder' BindName))
xps
lbs :: [LetBinding]
lbs = ((Pattern, BindName) -> LetBinding)
-> [(Pattern, BindName)] -> [LetBinding]
forall a b. (a -> b) -> [a] -> [b]
map (Pattern, BindName) -> LetBinding
letBinding [(Pattern, BindName)]
ps
letBinding :: (A.Pattern, A.BindName) -> A.LetBinding
letBinding :: (Pattern, BindName) -> LetBinding
letBinding (Pattern
p, BindName
n) = LetInfo -> Pattern -> Expr -> LetBinding
A.LetPatBind (Range -> LetInfo
A.LetRange Range
r) Pattern
p (Name -> Expr
A.Var (Name -> Expr) -> Name -> Expr
forall a b. (a -> b) -> a -> b
$ BindName -> Name
A.unBind BindName
n)
where r :: Range
r = Pattern -> BindName -> Range
forall u t. (HasRange u, HasRange t) => u -> t -> Range
fuseRange Pattern
p BindName
n
[LetBinding] -> TCM a -> TCM a
forall (t :: * -> *) a.
Foldable t =>
t LetBinding -> TCM a -> TCM a
checkLetBindings' [LetBinding]
lbs TCM a
ret
checkTacticAttribute :: LamOrPi -> Ranged A.Expr -> TCM Term
checkTacticAttribute :: LamOrPi -> Ranged Expr -> TCM Term
checkTacticAttribute LamOrPi
LamNotPi (Ranged Range
r Expr
e) = Range -> TCM Term -> TCM Term
forall (m :: * -> *) x a.
(MonadTrace m, HasRange x) =>
x -> m a -> m a
setCurrentRange Range
r (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$
TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ TypeError
TacticAttributeNotAllowed
checkTacticAttribute LamOrPi
PiNotLam (Ranged Range
r Expr
e) = do
expectedType <- TCM Term -> TCM Type
forall (m :: * -> *). Functor m => m Term -> m Type
el TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primAgdaTerm TCM Type -> TCM Type -> TCM Type
forall (m :: * -> *). Applicative m => m Type -> m Type -> m Type
--> TCM Term -> TCM Type
forall (m :: * -> *). Functor m => m Term -> m Type
el (TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primAgdaTCM TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *). Applicative m => m Term -> m Term -> m Term
<#> TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primLevelZero TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *). Applicative m => m Term -> m Term -> m Term
<@> TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primUnit)
checkExpr e expectedType
checkPath :: NamedArg Binder -> A.Type -> A.Expr -> Type -> TCM Term
checkPath :: NamedArg (Binder' BindName) -> Expr -> Expr -> Type -> TCM Term
checkPath NamedArg (Binder' BindName)
xp Expr
typ Expr
body Type
ty = do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.lambda" Int
30 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
hsep [ TCMT IO Doc
"checking path lambda", NamedArg (Binder' BindName) -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA NamedArg (Binder' BindName)
xp ]
case (Binder' BindName -> Maybe (Pattern, BindName)
forall a. Binder' a -> Maybe (Pattern, a)
A.extractPattern (Binder' BindName -> Maybe (Pattern, BindName))
-> Binder' BindName -> Maybe (Pattern, BindName)
forall a b. (a -> b) -> a -> b
$ NamedArg (Binder' BindName) -> Binder' BindName
forall a. NamedArg a -> a
namedArg NamedArg (Binder' BindName)
xp) of
Just{} -> NamedArg (Binder' BindName) -> TCM Term -> TCM Term
forall (m :: * -> *) x a.
(MonadTrace m, HasRange x) =>
x -> m a -> m a
setCurrentRange NamedArg (Binder' BindName)
xp (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
PatternInPathLambda
Maybe (Pattern, BindName)
Nothing -> do
let x :: NamedArg Name
x = (Binder' BindName -> Name)
-> NamedArg (Binder' BindName) -> NamedArg Name
forall a b. (a -> b) -> NamedArg a -> NamedArg b
updateNamedArg (BindName -> Name
A.unBind (BindName -> Name)
-> (Binder' BindName -> BindName) -> Binder' BindName -> Name
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Binder' BindName -> BindName
forall a. Binder' a -> a
A.binderName) NamedArg (Binder' BindName)
xp
info :: ArgInfo
info = NamedArg Name -> ArgInfo
forall a. LensArgInfo a => a -> ArgInfo
getArgInfo NamedArg Name
x
PathType s path level typ lhs rhs <- Type -> TCMT IO PathView
forall (m :: * -> *). HasBuiltins m => Type -> m PathView
pathView Type
ty
interval <- primIntervalType
v <- addContext ([x], interval) $
checkExpr body (El (raise 1 s) (raise 1 (unArg typ) `apply` [argN $ var 0]))
iZero <- primIZero
iOne <- primIOne
let lhs' = Int -> SubstArg Term -> Term -> Term
forall a. Subst a => Int -> SubstArg a -> a -> a
subst Int
0 Term
SubstArg Term
iZero Term
v
rhs' = Int -> SubstArg Term -> Term -> Term
forall a. Subst a => Int -> SubstArg a -> a -> a
subst Int
0 Term
SubstArg Term
iOne Term
v
let t = ArgInfo -> Abs Term -> Term
Lam ArgInfo
info (Abs Term -> Term) -> Abs Term -> Term
forall a b. (a -> b) -> a -> b
$ ArgName -> Term -> Abs Term
forall a. ArgName -> a -> Abs a
Abs (NamedArg Name -> ArgName
namedArgName NamedArg Name
x) Term
v
let btyp Term
i = Sort' Term -> Term -> Type
forall t a. Sort' t -> a -> Type'' t a
El Sort' Term
s (Arg Term -> Term
forall e. Arg e -> e
unArg Arg Term
typ Term -> [Arg Term] -> Term
forall t. Apply t => t -> [Arg Term] -> t
`apply` [Term -> Arg Term
forall e. e -> Arg e
argN Term
i])
locallyTC eRange (const noRange) $ blockTerm ty $ setCurrentRange body $ do
equalTerm (btyp iZero) lhs' (unArg lhs)
equalTerm (btyp iOne) rhs' (unArg rhs)
return t
checkLambda :: Comparison -> A.TypedBinding -> A.Expr -> Type -> TCM Term
checkLambda :: Comparison -> TypedBinding -> Expr -> Type -> TCM Term
checkLambda Comparison
cmp (A.TLet Range
_ List1 LetBinding
lbs) Expr
body Type
target =
List1 LetBinding -> TCM Term -> TCM Term
forall (t :: * -> *) a.
Foldable t =>
t LetBinding -> TCM a -> TCM a
checkLetBindings List1 LetBinding
lbs (Expr -> Type -> TCM Term
checkExpr Expr
body Type
target)
checkLambda Comparison
cmp b :: TypedBinding
b@(A.TBind Range
r TypedBindingInfo
tac List1 (NamedArg (Binder' BindName))
xps0 Expr
typ) Expr
body Type
target = do
(tel, tgt0) <- NamedArg (Binder' BindName) -> Type -> TCM (Telescope, Type)
forall a. HasRange a => NamedArg a -> Type -> TCM (Telescope, Type)
splitImplicitBinderT (List1 (NamedArg (Binder' BindName)) -> NamedArg (Binder' BindName)
forall a. NonEmpty a -> a
List1.head List1 (NamedArg (Binder' BindName))
xps0) Type
target
teleLam tel <$> addContext tel do
checkLambda' cmp r tac xps0 typ body tgt0
checkLambda' ::
Comparison
-> Range
-> A.TypedBindingInfo
-> List1 (NamedArg Binder)
-> A.Type
-> A.Expr
-> Type
-> TCM Term
checkLambda' :: Comparison
-> Range
-> TypedBindingInfo
-> List1 (NamedArg (Binder' BindName))
-> Expr
-> Expr
-> Type
-> TCM Term
checkLambda' Comparison
cmp Range
r TypedBindingInfo
tac List1 (NamedArg (Binder' BindName))
xps Expr
typ Expr
body Type
target = do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.lambda" Int
30 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"checkLambda xs =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> List1 (NamedArg (Binder' BindName)) -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA List1 (NamedArg (Binder' BindName))
xps
, TCMT IO Doc
"possiblePath =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Bool -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Bool -> m Doc
prettyTCM Bool
possiblePath
, TCMT IO Doc
"numbinds =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Int -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Int -> m Doc
prettyTCM Int
numbinds
, TCMT IO Doc
"typ =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Expr -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA (Expr -> Expr
unScope Expr
typ)
, TCMT IO Doc
"tactic =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> TacticAttribute -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA (TypedBindingInfo -> TacticAttribute
tbTacticAttr TypedBindingInfo
tac)
]
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.lambda" Int
60 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"info =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> (ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc)
-> (ArgInfo -> ArgName) -> ArgInfo -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. ArgInfo -> ArgName
forall a. Show a => a -> ArgName
show) ArgInfo
info
]
case TypedBindingInfo
tac of
TypedBindingInfo
_ | TypedBindingInfo -> Bool
forall a. Null a => a -> Bool
null TypedBindingInfo
tac -> () -> TCM ()
forall a. a -> TCMT IO a
forall (f :: * -> *) a. Applicative f => a -> f a
pure ()
A.TypedBindingInfo{ tbTacticAttr :: TypedBindingInfo -> TacticAttribute
tbTacticAttr = TacticAttribute (Just Ranged Expr
tactic) } -> do
_tactic <- LamOrPi -> Ranged Expr -> TCM Term
checkTacticAttribute LamOrPi
LamNotPi Ranged Expr
tactic
__IMPOSSIBLE__
TypedBindingInfo
_ -> TCM ()
forall a. HasCallStack => a
__IMPOSSIBLE__
TelV tel btyp <- Int -> Type -> TCMT IO (TelV Type)
forall (m :: * -> *).
(MonadReduce m, MonadAddContext m) =>
Int -> Type -> m (TelV Type)
telViewUpTo Int
numbinds Type
target
if numbinds == 1 && not (null tel) then useTargetType tel btyp
else if possiblePath then trySeeingIfPath
else dontUseTargetType
where
b :: TypedBinding
b = Range
-> TypedBindingInfo
-> List1 (NamedArg (Binder' BindName))
-> Expr
-> TypedBinding
A.TBind Range
r TypedBindingInfo
tac List1 (NamedArg (Binder' BindName))
xps Expr
typ
xs :: NonEmpty (NamedArg Name)
xs = (NamedArg (Binder' BindName) -> NamedArg Name)
-> List1 (NamedArg (Binder' BindName)) -> NonEmpty (NamedArg Name)
forall a b. (a -> b) -> NonEmpty a -> NonEmpty b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap ((Binder' BindName -> Name)
-> NamedArg (Binder' BindName) -> NamedArg Name
forall a b. (a -> b) -> NamedArg a -> NamedArg b
updateNamedArg (BindName -> Name
A.unBind (BindName -> Name)
-> (Binder' BindName -> BindName) -> Binder' BindName -> Name
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Binder' BindName -> BindName
forall a. Binder' a -> a
A.binderName)) List1 (NamedArg (Binder' BindName))
xps
numbinds :: Int
numbinds = List1 (NamedArg (Binder' BindName)) -> Int
forall a. NonEmpty a -> Int
forall (t :: * -> *) a. Foldable t => t a -> Int
length List1 (NamedArg (Binder' BindName))
xps
possiblePath :: Bool
possiblePath = Int
numbinds Int -> Int -> Bool
forall a. Eq a => a -> a -> Bool
== Int
1 Bool -> Bool -> Bool
&& Expr -> Bool
forall a. Underscore a => a -> Bool
isUnderscore (Expr -> Expr
unScope Expr
typ)
Bool -> Bool -> Bool
&& ArgInfo -> Bool
forall a. LensRelevance a => a -> Bool
isRelevant ArgInfo
info Bool -> Bool -> Bool
&& ArgInfo -> Bool
forall a. LensHiding a => a -> Bool
visible ArgInfo
info
info :: ArgInfo
info = NamedArg Name -> ArgInfo
forall a. LensArgInfo a => a -> ArgInfo
getArgInfo (NamedArg Name -> ArgInfo) -> NamedArg Name -> ArgInfo
forall a b. (a -> b) -> a -> b
$ NonEmpty (NamedArg Name) -> NamedArg Name
forall a. NonEmpty a -> a
List1.head NonEmpty (NamedArg Name)
xs
trySeeingIfPath :: TCM Term
trySeeingIfPath = do
ArgName -> Int -> ArgName -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> ArgName -> m ()
reportSLn ArgName
"tc.term.lambda" Int
60 (ArgName -> TCM ()) -> ArgName -> TCM ()
forall a b. (a -> b) -> a -> b
$ ArgName
"trySeeingIfPath for " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ List1 (NamedArg (Binder' BindName)) -> ArgName
forall a. Show a => a -> ArgName
show List1 (NamedArg (Binder' BindName))
xps
let postpone' :: Blocker -> Type -> TCM Term
postpone' Blocker
blocker Type
tgt =
TCMT IO Bool -> TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *) a. Monad m => m Bool -> m a -> m a -> m a
ifM (Maybe Cubical -> Bool
forall a. Maybe a -> Bool
isNothing (Maybe Cubical -> Bool) -> TCMT IO (Maybe Cubical) -> TCMT IO Bool
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> TCMT IO (Maybe Cubical)
forall (m :: * -> *). HasOptions m => m (Maybe Cubical)
cubicalOption) TCM Term
dontUseTargetType (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ Blocker -> Type -> TCM Term
postpone Blocker
blocker Type
tgt
Type
-> (Blocker -> Type -> TCM Term)
-> (NotBlocked -> Type -> TCM Term)
-> TCM Term
forall t (m :: * -> *) a.
(Reduce t, IsMeta t, MonadReduce m) =>
t -> (Blocker -> t -> m a) -> (NotBlocked -> t -> m a) -> m a
ifBlocked Type
target Blocker -> Type -> TCM Term
postpone' ((NotBlocked -> Type -> TCM Term) -> TCM Term)
-> (NotBlocked -> Type -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ NotBlocked
_ Type
t -> do
TCMT IO Bool -> TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *) a. Monad m => m Bool -> m a -> m a -> m a
ifNotM (PathView -> Bool
isPathType (PathView -> Bool) -> TCMT IO PathView -> TCMT IO Bool
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Type -> TCMT IO PathView
forall (m :: * -> *). HasBuiltins m => Type -> m PathView
pathView Type
t) TCM Term
dontUseTargetType do
NamedArg (Binder' BindName) -> Expr -> Expr -> Type -> TCM Term
checkPath (List1 (NamedArg (Binder' BindName)) -> NamedArg (Binder' BindName)
forall a. NonEmpty a -> a
List1.head List1 (NamedArg (Binder' BindName))
xps) Expr
typ Expr
body Type
t
postpone :: Blocker -> Type -> TCM Term
postpone Blocker
blocker Type
tgt = (TypeCheckingProblem -> Blocker -> TCM Term)
-> Blocker -> TypeCheckingProblem -> TCM Term
forall a b c. (a -> b -> c) -> b -> a -> c
flip TypeCheckingProblem -> Blocker -> TCM Term
postponeTypeCheckingProblem Blocker
blocker (TypeCheckingProblem -> TCM Term)
-> TypeCheckingProblem -> TCM Term
forall a b. (a -> b) -> a -> b
$
Comparison -> Expr -> Type -> TypeCheckingProblem
CheckExpr Comparison
cmp (ExprInfo -> LamBinding -> Expr -> Expr
A.Lam ExprInfo
A.exprNoRange (TypedBinding -> LamBinding
A.DomainFull TypedBinding
b) Expr
body) Type
tgt
dontUseTargetType :: TCM Term
dontUseTargetType = do
ArgName -> Int -> TCM () -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> m () -> m ()
verboseS ArgName
"tc.term.lambda" Int
5 (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ ArgName -> TCM ()
forall (m :: * -> *). MonadStatistics m => ArgName -> m ()
tick ArgName
"lambda-no-target-type"
argsT <- TCM Type -> TCM Type
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ Expr -> TCM Type
isType_ Expr
typ
let tel = NonEmpty (NamedArg Name) -> Type -> Telescope
namedBindsToTel1 NonEmpty (NamedArg Name)
xs Type
argsT
reportSDoc "tc.term.lambda" 30 $ "dontUseTargetType tel =" <+> pretty tel
checkSizeLtSat $ unEl argsT
let postponeOnBlockedPattern TCM (Type, Term)
m = TCM (Type, Term)
m TCM (Type, Term)
-> ((TCErr, Blocker) -> TCM (Type, Term)) -> TCM (Type, Term)
forall a. TCM a -> ((TCErr, Blocker) -> TCM a) -> TCM a
`catchIlltypedPatternBlockedOnMeta` \(TCErr
err , Blocker
x) -> do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term" Int
50 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat ([TCMT IO Doc] -> TCMT IO Doc) -> [TCMT IO Doc] -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$
[ TCMT IO Doc
"checking record pattern stuck on meta: " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (Blocker -> ArgName
forall a. Show a => a -> ArgName
show Blocker
x) ]
t1 <- (NonEmpty (NamedArg Name), Type) -> TCM Type -> TCM Type
forall b (m :: * -> *) a.
(AddContext b, MonadAddContext m) =>
b -> m a -> m a
forall (m :: * -> *) a.
MonadAddContext m =>
(NonEmpty (NamedArg Name), Type) -> m a -> m a
addContext (NonEmpty (NamedArg Name)
xs, Type
argsT) (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ TCM Type -> TCM Type
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes TCM Type
newTypeMeta_
let e = ExprInfo -> LamBinding -> Expr -> Expr
A.Lam ExprInfo
A.exprNoRange (TypedBinding -> LamBinding
A.DomainFull TypedBinding
b) Expr
body
tgt' = Telescope -> Type -> Type
telePi Telescope
tel Type
t1
w <- postponeTypeCheckingProblem (CheckExpr cmp e tgt') x
return (tgt' , w)
(target0 , w) <- postponeOnBlockedPattern $
addContext (xs, argsT) $ addTypedPatterns xps $ do
t1 <- workOnTypes newTypeMeta_
v <- checkExpr' cmp body t1
return (telePi tel t1 , teleLam tel v)
if notVisible info || any notVisible xs then do
pid <- newProblem_ $ leqType target0 target
blockTermOnProblem target w pid
else do
coerce cmp w target0 target
useTargetType :: Telescope -> Type -> TCM Term
useTargetType tel :: Telescope
tel@(ExtendTel Dom Type
dom (Abs ArgName
y Telescope
EmptyTel)) Type
btyp = do
ArgName -> Int -> TCM () -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> m () -> m ()
verboseS ArgName
"tc.term.lambda" Int
5 (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ ArgName -> TCM ()
forall (m :: * -> *). MonadStatistics m => ArgName -> m ()
tick ArgName
"lambda-with-target-type"
ArgName -> Int -> ArgName -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> ArgName -> m ()
reportSLn ArgName
"tc.term.lambda" Int
30 (ArgName -> TCM ()) -> ArgName -> TCM ()
forall a b. (a -> b) -> a -> b
$ ArgName
"useTargetType y = " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ ArgName
y
let (NamedArg Name
x :| []) = NonEmpty (NamedArg Name)
xs
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless (Dom Type -> ArgInfo -> Bool
forall a b. (LensHiding a, LensHiding b) => a -> b -> Bool
sameHiding Dom Type
dom ArgInfo
info) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM ()) -> TypeError -> TCM ()
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
WrongHidingInLambda Type
target
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
when (Maybe (WithOrigin (Ranged ArgName)) -> Bool
forall a. Maybe a -> Bool
isJust (Maybe (WithOrigin (Ranged ArgName)) -> Bool)
-> Maybe (WithOrigin (Ranged ArgName)) -> Bool
forall a b. (a -> b) -> a -> b
$ NamedArg Name -> Maybe (NameOf (NamedArg Name))
forall a. LensNamed a => a -> Maybe (NameOf a)
getNameOf NamedArg Name
x) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless (Dom Type -> NamedArg Name -> Bool
forall a b.
(LensNamed a, LensNamed b, NameOf a ~ WithOrigin (Ranged ArgName),
NameOf b ~ WithOrigin (Ranged ArgName)) =>
a -> b -> Bool
namedSame Dom Type
dom NamedArg Name
x) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$
NamedArg Name -> TCM () -> TCM ()
forall (m :: * -> *) x a.
(MonadTrace m, HasRange x) =>
x -> m a -> m a
setCurrentRange NamedArg Name
x (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM ()) -> TypeError -> TCM ()
forall a b. (a -> b) -> a -> b
$ TypeError
WrongHidingInLHS
info <- Dom Type -> ArgInfo -> TCM ArgInfo
forall dom.
(LensAnnotation dom, LensModality dom) =>
dom -> ArgInfo -> TCM ArgInfo
lambdaModalityCheck Dom Type
dom ArgInfo
info
let a = Dom Type -> Type
forall t e. Dom' t e -> e
unDom Dom Type
dom
checkSizeLtSat $ unEl a
(pid, argT) <- newProblem $ isTypeEqualTo typ a
v <- lambdaAddContext (namedArg x) y (defaultArgDom info argT) $
addTypedPatterns xps $ checkExpr' cmp body btyp
blockTermOnProblem target (Lam info $ Abs (namedArgName x) v) pid
useTargetType Telescope
_ Type
_ = TCM Term
forall a. HasCallStack => a
__IMPOSSIBLE__
lambdaModalityCheck :: (LensAnnotation dom, LensModality dom) => dom -> ArgInfo -> TCM ArgInfo
lambdaModalityCheck :: forall dom.
(LensAnnotation dom, LensModality dom) =>
dom -> ArgInfo -> TCM ArgInfo
lambdaModalityCheck dom
dom = Annotation -> ArgInfo -> TCM ArgInfo
forall dom. LensAnnotation dom => dom -> ArgInfo -> TCM ArgInfo
lambdaAnnotationCheck (dom -> Annotation
forall a. LensAnnotation a => a -> Annotation
getAnnotation dom
dom) (ArgInfo -> TCM ArgInfo)
-> (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall (m :: * -> *) b c a.
Monad m =>
(b -> m c) -> (a -> m b) -> a -> m c
<=< Modality -> ArgInfo -> TCM ArgInfo
forall dom. LensCohesion dom => dom -> ArgInfo -> TCM ArgInfo
lambdaCohesionCheck Modality
m (ArgInfo -> TCM ArgInfo)
-> (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall (m :: * -> *) b c a.
Monad m =>
(b -> m c) -> (a -> m b) -> a -> m c
<=< Modality -> ArgInfo -> TCM ArgInfo
forall dom. LensQuantity dom => dom -> ArgInfo -> TCM ArgInfo
lambdaQuantityCheck Modality
m (ArgInfo -> TCM ArgInfo)
-> (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall (m :: * -> *) b c a.
Monad m =>
(b -> m c) -> (a -> m b) -> a -> m c
<=< Modality -> ArgInfo -> TCM ArgInfo
forall dom. LensRelevance dom => dom -> ArgInfo -> TCM ArgInfo
lambdaIrrelevanceCheck Modality
m
where m :: Modality
m = dom -> Modality
forall a. LensModality a => a -> Modality
getModality dom
dom
lambdaIrrelevanceCheck :: LensRelevance dom => dom -> ArgInfo -> TCM ArgInfo
lambdaIrrelevanceCheck :: forall dom. LensRelevance dom => dom -> ArgInfo -> TCM ArgInfo
lambdaIrrelevanceCheck dom
dom ArgInfo
info
| ArgInfo -> Relevance
forall a. LensRelevance a => a -> Relevance
getRelevance ArgInfo
info Relevance -> Relevance -> Bool
forall a. Eq a => a -> a -> Bool
== Relevance
defaultRelevance = ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall a b. (a -> b) -> a -> b
$ Relevance -> ArgInfo -> ArgInfo
forall a. LensRelevance a => Relevance -> a -> a
setRelevance (dom -> Relevance
forall a. LensRelevance a => a -> Relevance
getRelevance dom
dom) ArgInfo
info
| Bool
otherwise = do
let rPi :: Relevance
rPi = dom -> Relevance
forall a. LensRelevance a => a -> Relevance
getRelevance dom
dom
let rLam :: Relevance
rLam = ArgInfo -> Relevance
forall a. LensRelevance a => a -> Relevance
getRelevance ArgInfo
info
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless (Relevance -> Relevance -> Bool
sameRelevance Relevance
rPi Relevance
rLam) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$
TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
WrongIrrelevanceInLambda
ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ArgInfo
info
lambdaQuantityCheck :: LensQuantity dom => dom -> ArgInfo -> TCM ArgInfo
lambdaQuantityCheck :: forall dom. LensQuantity dom => dom -> ArgInfo -> TCM ArgInfo
lambdaQuantityCheck dom
dom ArgInfo
info
| ArgInfo -> Bool
forall a. LensQuantity a => a -> Bool
noUserQuantity ArgInfo
info = ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall a b. (a -> b) -> a -> b
$ Quantity -> ArgInfo -> ArgInfo
forall a. LensQuantity a => Quantity -> a -> a
setQuantity (dom -> Quantity
forall a. LensQuantity a => a -> Quantity
getQuantity dom
dom) ArgInfo
info
| Bool
otherwise = do
let qPi :: Quantity
qPi = dom -> Quantity
forall a. LensQuantity a => a -> Quantity
getQuantity dom
dom
let qLam :: Quantity
qLam = ArgInfo -> Quantity
forall a. LensQuantity a => a -> Quantity
getQuantity ArgInfo
info
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless (Quantity
qPi Quantity -> Quantity -> Bool
`sameQuantity` Quantity
qLam) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ do
TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
WrongQuantityInLambda
ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ArgInfo
info
lambdaAnnotationCheck :: LensAnnotation dom => dom -> ArgInfo -> TCM ArgInfo
lambdaAnnotationCheck :: forall dom. LensAnnotation dom => dom -> ArgInfo -> TCM ArgInfo
lambdaAnnotationCheck dom
dom ArgInfo
info
| ArgInfo -> Annotation
forall a. LensAnnotation a => a -> Annotation
getAnnotation ArgInfo
info Annotation -> Annotation -> Bool
forall a. Eq a => a -> a -> Bool
== Annotation
defaultAnnotation = ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall a b. (a -> b) -> a -> b
$ Annotation -> ArgInfo -> ArgInfo
forall a. LensAnnotation a => Annotation -> a -> a
setAnnotation (dom -> Annotation
forall a. LensAnnotation a => a -> Annotation
getAnnotation dom
dom) ArgInfo
info
| Bool
otherwise = do
let aPi :: Annotation
aPi = dom -> Annotation
forall a. LensAnnotation a => a -> Annotation
getAnnotation dom
dom
let aLam :: Annotation
aLam = ArgInfo -> Annotation
forall a. LensAnnotation a => a -> Annotation
getAnnotation ArgInfo
info
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless (Annotation
aPi Annotation -> Annotation -> Bool
forall a. Eq a => a -> a -> Bool
== Annotation
aLam) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ do
TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
WrongAnnotationInLambda
ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ArgInfo
info
lambdaCohesionCheck :: LensCohesion dom => dom -> ArgInfo -> TCM ArgInfo
lambdaCohesionCheck :: forall dom. LensCohesion dom => dom -> ArgInfo -> TCM ArgInfo
lambdaCohesionCheck dom
dom ArgInfo
info
| ArgInfo -> Cohesion
forall a. LensCohesion a => a -> Cohesion
getCohesion ArgInfo
info Cohesion -> Cohesion -> Bool
forall a. Eq a => a -> a -> Bool
== Cohesion
defaultCohesion = ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (ArgInfo -> TCM ArgInfo) -> ArgInfo -> TCM ArgInfo
forall a b. (a -> b) -> a -> b
$ Cohesion -> ArgInfo -> ArgInfo
forall a. LensCohesion a => Cohesion -> a -> a
setCohesion (dom -> Cohesion
forall a. LensCohesion a => a -> Cohesion
getCohesion dom
dom) ArgInfo
info
| Bool
otherwise = do
let cPi :: Cohesion
cPi = dom -> Cohesion
forall a. LensCohesion a => a -> Cohesion
getCohesion dom
dom
let cLam :: Cohesion
cLam = ArgInfo -> Cohesion
forall a. LensCohesion a => a -> Cohesion
getCohesion ArgInfo
info
Bool -> TCM () -> TCM ()
forall b (m :: * -> *). (IsBool b, Monad m) => b -> m () -> m ()
unless (Cohesion
cPi Cohesion -> Cohesion -> Bool
`sameCohesion` Cohesion
cLam) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ do
TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
WrongCohesionInLambda
ArgInfo -> TCM ArgInfo
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ArgInfo
info
lambdaAddContext :: MonadAddContext m => Name -> ArgName -> Dom Type -> m a -> m a
lambdaAddContext :: forall (m :: * -> *) a.
MonadAddContext m =>
Name -> ArgName -> Dom Type -> m a -> m a
lambdaAddContext Name
x ArgName
y Dom Type
dom
| Name -> Bool
forall a. IsNoName a => a -> Bool
isNoName Name
x = (ArgName, Dom Type) -> m a -> m a
forall b (m :: * -> *) a.
(AddContext b, MonadAddContext m) =>
b -> m a -> m a
forall (m :: * -> *) a.
MonadAddContext m =>
(ArgName, Dom Type) -> m a -> m a
addContext (ArgName
y, Dom Type
dom)
| Bool
otherwise = (Name, Dom Type) -> m a -> m a
forall b (m :: * -> *) a.
(AddContext b, MonadAddContext m) =>
b -> m a -> m a
forall (m :: * -> *) a.
MonadAddContext m =>
(Name, Dom Type) -> m a -> m a
addContext (Name
x, Dom Type
dom)
checkPostponedLambda :: Comparison -> Arg (List1 (WithHiding Name), Maybe Type) -> A.Expr -> Type -> TCM Term
checkPostponedLambda :: Comparison
-> Arg (List1 (WithHiding Name), Maybe Type)
-> Expr
-> Type
-> TCM Term
checkPostponedLambda Comparison
cmp args :: Arg (List1 (WithHiding Name), Maybe Type)
args@(Arg ArgInfo
info (WithHiding Hiding
h Name
x :| [WithHiding Name]
xs, Maybe Type
mt)) Expr
body Type
target = do
let postpone :: Blocker -> Type -> TCM Term
postpone Blocker
_ Type
t = TypeCheckingProblem -> TCM Term
postponeTypeCheckingProblem_ (TypeCheckingProblem -> TCM Term)
-> TypeCheckingProblem -> TCM Term
forall a b. (a -> b) -> a -> b
$ Comparison
-> Arg (List1 (WithHiding Name), Maybe Type)
-> Expr
-> Type
-> TypeCheckingProblem
CheckLambda Comparison
cmp Arg (List1 (WithHiding Name), Maybe Type)
args Expr
body Type
t
lamHiding :: Hiding
lamHiding = Hiding -> Hiding -> Hiding
forall a. Monoid a => a -> a -> a
mappend Hiding
h (Hiding -> Hiding) -> Hiding -> Hiding
forall a b. (a -> b) -> a -> b
$ ArgInfo -> Hiding
forall a. LensHiding a => a -> Hiding
getHiding ArgInfo
info
Hiding
-> Type
-> (Blocker -> Type -> TCM Term)
-> (Type -> TCM Term)
-> TCM Term
insertHiddenLambdas Hiding
lamHiding Type
target Blocker -> Type -> TCM Term
postpone ((Type -> TCM Term) -> TCM Term) -> (Type -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ t :: Type
t@(El Sort' Term
_ (Pi Dom Type
dom Abs Type
b)) -> do
info' <- Hiding -> ArgInfo -> ArgInfo
forall a. LensHiding a => Hiding -> a -> a
setHiding Hiding
lamHiding (ArgInfo -> ArgInfo) -> TCM ArgInfo -> TCM ArgInfo
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Dom Type -> ArgInfo -> TCM ArgInfo
forall dom.
(LensAnnotation dom, LensModality dom) =>
dom -> ArgInfo -> TCM ArgInfo
lambdaModalityCheck Dom Type
dom ArgInfo
info
mpid <- caseMaybe mt (return Nothing) $ \ Type
ascribedType -> ProblemId -> Maybe ProblemId
forall a. a -> Maybe a
Just (ProblemId -> Maybe ProblemId)
-> TCMT IO ProblemId -> TCMT IO (Maybe ProblemId)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> do
TCM () -> TCMT IO ProblemId
forall (m :: * -> *) a.
(MonadFresh ProblemId m, MonadConstraint m) =>
m a -> m ProblemId
newProblem_ (TCM () -> TCMT IO ProblemId) -> TCM () -> TCMT IO ProblemId
forall a b. (a -> b) -> a -> b
$ Type -> Type -> TCM ()
forall (m :: * -> *). MonadConversion m => Type -> Type -> m ()
leqType (Dom Type -> Type
forall t e. Dom' t e -> e
unDom Dom Type
dom) Type
ascribedType
let dom' = Relevance -> Dom Type -> Dom Type
forall a. LensRelevance a => Relevance -> a -> a
setRelevance (ArgInfo -> Relevance
forall a. LensRelevance a => a -> Relevance
getRelevance ArgInfo
info') (Dom Type -> Dom Type)
-> (Dom Type -> Dom Type) -> Dom Type -> Dom Type
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Hiding -> Dom Type -> Dom Type
forall a. LensHiding a => Hiding -> a -> a
setHiding Hiding
lamHiding (Dom Type -> Dom Type) -> Dom Type -> Dom Type
forall a b. (a -> b) -> a -> b
$
Dom Type -> (Type -> Dom Type) -> Maybe Type -> Dom Type
forall b a. b -> (a -> b) -> Maybe a -> b
maybe Dom Type
dom (Dom Type
dom Dom Type -> Type -> Dom Type
forall (f :: * -> *) a b. Functor f => f a -> b -> f b
$>) Maybe Type
mt
v <- lambdaAddContext x (absName b) dom' $
checkPostponedLambda0 cmp (Arg info (xs, mt)) body $ absBody b
let v' = ArgInfo -> Abs Term -> Term
Lam ArgInfo
info' (Abs Term -> Term) -> Abs Term -> Term
forall a b. (a -> b) -> a -> b
$ ArgName -> Term -> Abs Term
forall a. ArgName -> a -> Abs a
Abs (Name -> ArgName
nameToArgName Name
x) Term
v
maybe (return v') (blockTermOnProblem t v') mpid
checkPostponedLambda0 :: Comparison -> Arg ([WithHiding Name], Maybe Type) -> A.Expr -> Type -> TCM Term
checkPostponedLambda0 :: Comparison
-> Arg ([WithHiding Name], Maybe Type) -> Expr -> Type -> TCM Term
checkPostponedLambda0 Comparison
cmp (Arg ArgInfo
_ ([] , Maybe Type
_ )) Expr
body Type
target =
Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp Expr
body Type
target
checkPostponedLambda0 Comparison
cmp (Arg ArgInfo
info (WithHiding Name
x : [WithHiding Name]
xs, Maybe Type
mt)) Expr
body Type
target =
Comparison
-> Arg (List1 (WithHiding Name), Maybe Type)
-> Expr
-> Type
-> TCM Term
checkPostponedLambda Comparison
cmp (ArgInfo
-> (List1 (WithHiding Name), Maybe Type)
-> Arg (List1 (WithHiding Name), Maybe Type)
forall e. ArgInfo -> e -> Arg e
Arg ArgInfo
info (WithHiding Name
x WithHiding Name -> [WithHiding Name] -> List1 (WithHiding Name)
forall a. a -> [a] -> NonEmpty a
:| [WithHiding Name]
xs, Maybe Type
mt)) Expr
body Type
target
insertHiddenLambdas
:: Hiding
-> Type
-> (Blocker -> Type -> TCM Term)
-> (Type -> TCM Term)
-> TCM Term
insertHiddenLambdas :: Hiding
-> Type
-> (Blocker -> Type -> TCM Term)
-> (Type -> TCM Term)
-> TCM Term
insertHiddenLambdas Hiding
h Type
target Blocker -> Type -> TCM Term
postpone Type -> TCM Term
ret = do
Type
-> (Blocker -> Type -> TCM Term)
-> (NotBlocked -> Type -> TCM Term)
-> TCM Term
forall t (m :: * -> *) a.
(Reduce t, IsMeta t, MonadReduce m) =>
t -> (Blocker -> t -> m a) -> (NotBlocked -> t -> m a) -> m a
ifBlocked Type
target Blocker -> Type -> TCM Term
postpone ((NotBlocked -> Type -> TCM Term) -> TCM Term)
-> (NotBlocked -> Type -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ NotBlocked
_ Type
t -> do
case Type -> Term
forall t a. Type'' t a -> a
unEl Type
t of
Pi Dom Type
dom Abs Type
b -> do
let h' :: Hiding
h' = Dom Type -> Hiding
forall a. LensHiding a => a -> Hiding
getHiding Dom Type
dom
if Hiding -> Hiding -> Bool
forall a b. (LensHiding a, LensHiding b) => a -> b -> Bool
sameHiding Hiding
h Hiding
h' then Type -> TCM Term
ret Type
t else do
if Hiding -> Bool
forall a. LensHiding a => a -> Bool
visible Hiding
h' then TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
WrongHidingInLambda Type
target else do
let x :: ArgName
x = Abs Type -> ArgName
forall a. Abs a -> ArgName
absName Abs Type
b
ArgInfo -> Abs Term -> Term
Lam (Origin -> ArgInfo -> ArgInfo
forall a. LensOrigin a => Origin -> a -> a
setOrigin Origin
Inserted (ArgInfo -> ArgInfo) -> ArgInfo -> ArgInfo
forall a b. (a -> b) -> a -> b
$ Dom Type -> ArgInfo
forall t e. Dom' t e -> ArgInfo
domInfo Dom Type
dom) (Abs Term -> Term) -> (Term -> Abs Term) -> Term -> Term
forall b c a. (b -> c) -> (a -> b) -> a -> c
. ArgName -> Term -> Abs Term
forall a. ArgName -> a -> Abs a
Abs ArgName
x (Term -> Term) -> TCM Term -> TCM Term
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> do
(ArgName, Dom Type) -> TCM Term -> TCM Term
forall b (m :: * -> *) a.
(AddContext b, MonadAddContext m) =>
b -> m a -> m a
forall (m :: * -> *) a.
MonadAddContext m =>
(ArgName, Dom Type) -> m a -> m a
addContext (ArgName
x, Dom Type
dom) (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ Hiding
-> Type
-> (Blocker -> Type -> TCM Term)
-> (Type -> TCM Term)
-> TCM Term
insertHiddenLambdas Hiding
h (Abs Type -> Type
forall a. Subst a => Abs a -> a
absBody Abs Type
b) Blocker -> Type -> TCM Term
postpone Type -> TCM Term
ret
Term
_ -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
ShouldBePi Type
target
checkAbsurdLambda :: Comparison -> A.ExprInfo -> Hiding -> A.Expr -> Type -> TCM Term
checkAbsurdLambda :: Comparison -> ExprInfo -> Hiding -> Expr -> Type -> TCM Term
checkAbsurdLambda Comparison
cmp ExprInfo
i Hiding
h Expr
e Type
t =
TCM Term -> TCM Term
forall a. TCM a -> TCM a
setRunTimeModeUnlessInHardCompileTimeMode (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ do
t <- Type -> TCM Type
forall a (m :: * -> *).
(InstantiateFull a, MonadReduce m) =>
a -> m a
instantiateFull Type
t
ifBlocked t (\ Blocker
blocker Type
t' -> TypeCheckingProblem -> Blocker -> TCM Term
postponeTypeCheckingProblem (Comparison -> Expr -> Type -> TypeCheckingProblem
CheckExpr Comparison
cmp Expr
e Type
t') Blocker
blocker) $ \ NotBlocked
_ Type
t' -> do
case Type -> Term
forall t a. Type'' t a -> a
unEl Type
t' of
Pi dom :: Dom Type
dom@(Dom{domInfo :: forall t e. Dom' t e -> ArgInfo
domInfo = ArgInfo
info', unDom :: forall t e. Dom' t e -> e
unDom = Type
a}) Abs Type
b
| Bool -> Bool
not (Hiding -> ArgInfo -> Bool
forall a b. (LensHiding a, LensHiding b) => a -> b -> Bool
sameHiding Hiding
h ArgInfo
info') -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
WrongHidingInLambda Type
t'
| Bool
otherwise -> Type -> TCM Term -> TCM Term
forall (m :: * -> *).
(MonadMetaSolver m, MonadConstraint m, MonadFresh Int m,
MonadFresh ProblemId m) =>
Type -> m Term -> m Term
blockTerm Type
t' (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ do
Range -> Type -> TCM ()
ensureEmptyType (ExprInfo -> Range
forall a. HasRange a => a -> Range
getRange ExprInfo
i) Type
a
top <- TCMT IO ModuleName
forall (m :: * -> *). MonadTCEnv m => m ModuleName
currentModule
aux <- qualify top <$> freshName_ (getRange i, absurdLambdaName)
mod <- currentModality
reportSDoc "tc.term.absurd" 10 $ vcat
[ ("Adding absurd function" <+> prettyTCM mod) <> prettyTCM aux
, nest 2 $ "of type" <+> prettyTCM t'
]
lang <- getLanguage
fun <- emptyFunctionData
addConstant aux $
(\ Defn
d -> (ArgInfo -> QName -> Type -> Language -> Defn -> Definition
defaultDefn (Modality -> ArgInfo -> ArgInfo
forall a. LensModality a => Modality -> a -> a
setModality Modality
mod ArgInfo
info') QName
aux Type
t' Language
lang Defn
d)
{ defPolarity = [Nonvariant]
, defArgOccurrences = [Unused] })
$ FunctionDefn fun
{ _funClauses =
[ Clause
{ clauseLHSRange = getRange e
, clauseFullRange = getRange e
, clauseTel = telFromList [fmap (absurdPatternName,) dom]
, namedClausePats = [Arg info' $ Named (Just $ WithOrigin Inserted $ unranged $ absName b) $ absurdP 0]
, clauseBody = Nothing
, clauseType = Just $ setModality mod $ defaultArg $ absBody b
, clauseCatchall = True
, clauseRecursive = Just False
, clauseUnreachable = Just True
, clauseEllipsis = NoEllipsis
, clauseWhereModule = Nothing
}
]
, _funCompiled = Just $ Fail [Arg info' "()"]
, _funSplitTree = Just $ SplittingDone 0
, _funMutual = Just []
, _funTerminates = Just True
, _funExtLam = Just $ ExtLamInfo top True empty
}
Def aux . map Apply . teleArgs <$> getContextTelescope
Term
_ -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
ShouldBePi Type
t'
checkExtendedLambda ::
Comparison -> A.ExprInfo -> A.DefInfo -> Erased -> QName ->
List1 A.Clause -> A.Expr -> Type -> TCM Term
checkExtendedLambda :: Comparison
-> ExprInfo
-> DefInfo
-> Erased
-> QName
-> List1 Clause
-> Expr
-> Type
-> TCM Term
checkExtendedLambda Comparison
cmp ExprInfo
i DefInfo
di Erased
erased QName
qname List1 Clause
cs Expr
e Type
t = do
mod <- TCMT IO Modality
forall (m :: * -> *). MonadTCEnv m => m Modality
currentModality
when (isErased erased && not (hasQuantity0 mod)) $ typeError LambdaIsErased
setModeUnlessInHardCompileTimeMode erased do
solveSizeConstraints DontDefaultToInfty
lamMod <- inFreshModuleIfFreeParams currentModule
t <- instantiateFull t
ifBlocked t (\ Blocker
m Type
t' -> TypeCheckingProblem -> TCM Term
postponeTypeCheckingProblem_ (TypeCheckingProblem -> TCM Term)
-> TypeCheckingProblem -> TCM Term
forall a b. (a -> b) -> a -> b
$ Comparison -> Expr -> Type -> TypeCheckingProblem
CheckExpr Comparison
cmp Expr
e Type
t') \ NotBlocked
_ Type
t -> do
j <- TCM MutualId
currentOrFreshMutualBlock
mod <- currentModality
let info = Modality -> ArgInfo -> ArgInfo
forall a. LensModality a => Modality -> a -> a
setModality Modality
mod ArgInfo
defaultArgInfo
reportSDoc "tc.term.exlam" 20 $ vcat
[ hsep
[ text $ show $ A.defAbstract di
, "extended lambda's implementation"
, doubleQuotes $ prettyTCM qname
, "has type:"
]
, prettyTCM t
]
args <- getContextArgs
abstract (A.defAbstract di) do
addConstant qname =<< do
lang <- getLanguage
fun <- emptyFunction
useTerPragma $
(defaultDefn info qname t lang fun)
{ defMutual = j }
checkFunDef' t info (Just $ ExtLamInfo lamMod False empty) Nothing di qname $
List1.toList cs
whenNothingM (asksTC envMutualBlock) $
checkIApplyConfluence_ qname
return $ Def qname $ map Apply args
where
abstract :: IsAbstract -> m a -> m a
abstract IsAbstract
ConcreteDef = m a -> m a
forall (m :: * -> *) a. MonadTCEnv m => m a -> m a
inConcreteMode
abstract IsAbstract
AbstractDef = m a -> m a
forall (m :: * -> *) a. MonadTCEnv m => m a -> m a
inAbstractMode
catchIlltypedPatternBlockedOnMeta :: TCM a -> ((TCErr, Blocker) -> TCM a) -> TCM a
catchIlltypedPatternBlockedOnMeta :: forall a. TCM a -> ((TCErr, Blocker) -> TCM a) -> TCM a
catchIlltypedPatternBlockedOnMeta TCM a
m (TCErr, Blocker) -> TCM a
handle = do
st <- TCMT IO TCState
forall (m :: * -> *). MonadTCState m => m TCState
getTC
m `catchError` \ TCErr
err -> do
let reraise :: MonadError TCErr m => m a
reraise :: forall (m :: * -> *) a. MonadError TCErr m => m a
reraise = TCErr -> m a
forall a. TCErr -> m a
forall e (m :: * -> *) a. MonadError e m => e -> m a
throwError TCErr
err
blocker <- TCMT IO Blocker
-> (Blocker -> TCMT IO Blocker) -> Maybe Blocker -> TCMT IO Blocker
forall b a. b -> (a -> b) -> Maybe a -> b
maybe TCMT IO Blocker
forall (m :: * -> *) a. MonadError TCErr m => m a
reraise Blocker -> TCMT IO Blocker
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Maybe Blocker -> TCMT IO Blocker)
-> Maybe Blocker -> TCMT IO Blocker
forall a b. (a -> b) -> a -> b
$ case TCErr
err of
TypeError CallStack
_ TCState
s Closure TypeError
cl -> case Closure TypeError -> TypeError
forall a. Closure a -> a
clValue Closure TypeError
cl of
SortOfSplitVarError Maybe Blocker
b Doc
_ -> Maybe Blocker
b
SplitError (UnificationStuck Maybe Blocker
b QName
c Telescope
tel [Arg Term]
us [Arg Term]
vs [UnificationFailure]
_) -> Maybe Blocker
b
SplitError (BlockedType Blocker
b Closure Type
aClosure) -> Blocker -> Maybe Blocker
forall a. a -> Maybe a
Just Blocker
b
CannotEliminateWithPattern Maybe Blocker
b NamedArg Pattern
p Type
a -> Maybe Blocker
b
TypeError
_ -> Maybe Blocker
forall a. Maybe a
Nothing
TCErr
_ -> Maybe Blocker
forall a. Maybe a
Nothing
reportSDoc "tc.postpone" 20 $ vcat $
[ "checking definition blocked on: " <+> prettyTCM blocker ]
putTC st
blocker <- (`onBlockingMetasM` blocker) $ \ MetaId
x ->
MetaId -> TCMT IO (Maybe (Either RemoteMetaVariable MetaVariable))
forall (m :: * -> *).
ReadTCState m =>
MetaId -> m (Maybe (Either RemoteMetaVariable MetaVariable))
lookupMeta MetaId
x TCMT IO (Maybe (Either RemoteMetaVariable MetaVariable))
-> (Maybe (Either RemoteMetaVariable MetaVariable)
-> TCMT IO Blocker)
-> TCMT IO Blocker
forall a b. TCMT IO a -> (a -> TCMT IO b) -> TCMT IO b
forall (m :: * -> *) a b. Monad m => m a -> (a -> m b) -> m b
>>= \ case
Maybe (Either RemoteMetaVariable MetaVariable)
Nothing -> Blocker -> TCMT IO Blocker
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Blocker
neverUnblock
Just Left{} -> Blocker -> TCMT IO Blocker
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Blocker
alwaysUnblock
Just (Right MetaVariable
m)
| InstV{} <- MetaVariable -> MetaInstantiation
mvInstantiation MetaVariable
m -> Blocker -> TCMT IO Blocker
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Blocker
alwaysUnblock
| Bool
otherwise -> Blocker -> TCMT IO Blocker
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Blocker -> TCMT IO Blocker) -> Blocker -> TCMT IO Blocker
forall a b. (a -> b) -> a -> b
$ MetaId -> Blocker
unblockOnMeta MetaId
x
if blocker `elem` [neverUnblock, alwaysUnblock] then reraise else handle (err, blocker)
expandModuleAssigns
:: [Either A.Assign A.ModuleName]
-> [C.Name]
-> TCM A.Assigns
expandModuleAssigns :: [Either (FieldAssignment' Expr) ModuleName]
-> [Name] -> TCM Assigns
expandModuleAssigns [Either (FieldAssignment' Expr) ModuleName]
mfs [Name]
xs = do
let (Assigns
fs , [ModuleName]
ms) = [Either (FieldAssignment' Expr) ModuleName]
-> (Assigns, [ModuleName])
forall a b. [Either a b] -> ([a], [b])
partitionEithers [Either (FieldAssignment' Expr) ModuleName]
mfs
fs' <- [Name]
-> (Name -> TCMT IO (Maybe (FieldAssignment' Expr)))
-> TCMT IO [Maybe (FieldAssignment' Expr)]
forall (t :: * -> *) (m :: * -> *) a b.
(Traversable t, Monad m) =>
t a -> (a -> m b) -> m (t b)
forM ([Name]
xs [Name] -> [Name] -> [Name]
forall a. Eq a => [a] -> [a] -> [a]
List.\\ (FieldAssignment' Expr -> Name) -> Assigns -> [Name]
forall a b. (a -> b) -> [a] -> [b]
map (Lens' (FieldAssignment' Expr) Name -> FieldAssignment' Expr -> Name
forall o (m :: * -> *) i. MonadReader o m => Lens' o i -> m i
view (Name -> f Name)
-> FieldAssignment' Expr -> f (FieldAssignment' Expr)
forall a (f :: * -> *).
Functor f =>
(Name -> f Name) -> FieldAssignment' a -> f (FieldAssignment' a)
Lens' (FieldAssignment' Expr) Name
nameFieldA) Assigns
fs) ((Name -> TCMT IO (Maybe (FieldAssignment' Expr)))
-> TCMT IO [Maybe (FieldAssignment' Expr)])
-> (Name -> TCMT IO (Maybe (FieldAssignment' Expr)))
-> TCMT IO [Maybe (FieldAssignment' Expr)]
forall a b. (a -> b) -> a -> b
$ \ Name
f -> do
pms <- [ModuleName]
-> (ModuleName
-> TCMT IO (Maybe (ModuleName, FieldAssignment' Expr)))
-> TCMT IO [Maybe (ModuleName, FieldAssignment' Expr)]
forall (t :: * -> *) (m :: * -> *) a b.
(Traversable t, Monad m) =>
t a -> (a -> m b) -> m (t b)
forM [ModuleName]
ms ((ModuleName
-> TCMT IO (Maybe (ModuleName, FieldAssignment' Expr)))
-> TCMT IO [Maybe (ModuleName, FieldAssignment' Expr)])
-> (ModuleName
-> TCMT IO (Maybe (ModuleName, FieldAssignment' Expr)))
-> TCMT IO [Maybe (ModuleName, FieldAssignment' Expr)]
forall a b. (a -> b) -> a -> b
$ \ ModuleName
m -> do
modScope <- ModuleName -> ScopeM Scope
getNamedScope ModuleName
m
let names :: ThingsInScope AbstractName
names = Scope -> ThingsInScope AbstractName
forall a. InScope a => Scope -> ThingsInScope a
exportedNamesInScope Scope
modScope
return $
case Map.lookup f names of
Just (AbstractName
n :| []) -> (ModuleName, FieldAssignment' Expr)
-> Maybe (ModuleName, FieldAssignment' Expr)
forall a. a -> Maybe a
Just (ModuleName
m, Name -> Expr -> FieldAssignment' Expr
forall a. Name -> a -> FieldAssignment' a
FieldAssignment Name
f (Expr -> FieldAssignment' Expr) -> Expr -> FieldAssignment' Expr
forall a b. (a -> b) -> a -> b
$ Expr -> Expr
forall a. KillRange a => KillRangeT a
killRange (Expr -> Expr) -> Expr -> Expr
forall a b. (a -> b) -> a -> b
$ AbstractName -> Expr
forall a. NameToExpr a => a -> Expr
A.nameToExpr AbstractName
n)
Maybe (List1 AbstractName)
_ -> Maybe (ModuleName, FieldAssignment' Expr)
forall a. Maybe a
Nothing
case catMaybes pms of
[] -> Maybe (FieldAssignment' Expr)
-> TCMT IO (Maybe (FieldAssignment' Expr))
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Maybe (FieldAssignment' Expr)
forall a. Maybe a
Nothing
[(ModuleName
_, FieldAssignment' Expr
fa)] -> Maybe (FieldAssignment' Expr)
-> TCMT IO (Maybe (FieldAssignment' Expr))
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (FieldAssignment' Expr -> Maybe (FieldAssignment' Expr)
forall a. a -> Maybe a
Just FieldAssignment' Expr
fa)
(ModuleName, FieldAssignment' Expr)
x:(ModuleName, FieldAssignment' Expr)
y:[(ModuleName, FieldAssignment' Expr)]
zs -> TypeError -> TCMT IO (Maybe (FieldAssignment' Expr))
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCMT IO (Maybe (FieldAssignment' Expr)))
-> TypeError -> TCMT IO (Maybe (FieldAssignment' Expr))
forall a b. (a -> b) -> a -> b
$ Name -> List2 ModuleName -> TypeError
AmbiguousField Name
f (List2 ModuleName -> TypeError) -> List2 ModuleName -> TypeError
forall a b. (a -> b) -> a -> b
$ ((ModuleName, FieldAssignment' Expr) -> ModuleName)
-> List2 (ModuleName, FieldAssignment' Expr) -> List2 ModuleName
forall a b. (a -> b) -> List2 a -> List2 b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap (ModuleName, FieldAssignment' Expr) -> ModuleName
forall a b. (a, b) -> a
fst (List2 (ModuleName, FieldAssignment' Expr) -> List2 ModuleName)
-> List2 (ModuleName, FieldAssignment' Expr) -> List2 ModuleName
forall a b. (a -> b) -> a -> b
$ (ModuleName, FieldAssignment' Expr)
-> (ModuleName, FieldAssignment' Expr)
-> [(ModuleName, FieldAssignment' Expr)]
-> List2 (ModuleName, FieldAssignment' Expr)
forall a. a -> a -> [a] -> List2 a
List2 (ModuleName, FieldAssignment' Expr)
x (ModuleName, FieldAssignment' Expr)
y [(ModuleName, FieldAssignment' Expr)]
zs
return (fs ++ catMaybes fs')
checkRecordExpression
:: Comparison
-> A.RecStyle
-> A.RecordAssigns
-> A.Expr
-> Type
-> TCM Term
checkRecordExpression :: Comparison
-> RecStyle
-> [Either (FieldAssignment' Expr) ModuleName]
-> Expr
-> Type
-> TCM Term
checkRecordExpression Comparison
cmp RecStyle
style [Either (FieldAssignment' Expr) ModuleName]
mfs Expr
e Type
t = do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.rec" Int
10 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ TCMT IO Doc
"checking record expression"
, Expr -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA Expr
e
]
Type
-> (Blocker -> Type -> TCM Term)
-> (NotBlocked -> Type -> TCM Term)
-> TCM Term
forall t (m :: * -> *) a.
(Reduce t, IsMeta t, MonadReduce m) =>
t -> (Blocker -> t -> m a) -> (NotBlocked -> t -> m a) -> m a
ifBlocked Type
t (\ Blocker
_ Type
t -> Type -> TCM Term
guessRecordType Type
t) ((NotBlocked -> Type -> TCM Term) -> TCM Term)
-> (NotBlocked -> Type -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ NotBlocked
_ Type
t -> do
case Type -> Term
forall t a. Type'' t a -> a
unEl Type
t of
Def QName
r Elims
es -> do
let ~(Just [Arg Term]
vs) = Elims -> Maybe [Arg Term]
forall a. [Elim' a] -> Maybe [Arg a]
allApplyElims Elims
es
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.rec" Int
20 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ TCMT IO Doc
" r = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall a. Semigroup a => a -> a -> a
<> Doc -> TCMT IO Doc
forall a. a -> TCMT IO a
forall (f :: * -> *) a. Applicative f => a -> f a
pure (QName -> Doc
forall a. Pretty a => a -> Doc
P.pretty QName
r)
def <- QName -> TCMT IO RecordData
forall (m :: * -> *).
(HasConstInfo m, ReadTCState m, MonadError TCErr m) =>
QName -> m RecordData
getRecordDef QName
r
let
cxs = (Dom Name -> Arg Name) -> [Dom Name] -> [Arg Name]
forall a b. (a -> b) -> [a] -> [b]
map Dom Name -> Arg Name
forall t a. Dom' t a -> Arg a
argFromDom ([Dom Name] -> [Arg Name]) -> [Dom Name] -> [Arg Name]
forall a b. (a -> b) -> a -> b
$ RecordData -> [Dom Name]
recordFieldNames RecordData
def
xs = (Arg Name -> Name) -> [Arg Name] -> [Name]
forall a b. (a -> b) -> [a] -> [b]
map Arg Name -> Name
forall e. Arg e -> e
unArg [Arg Name]
cxs
con = KillRangeT ConHead
forall a. KillRange a => KillRangeT a
killRange KillRangeT ConHead -> KillRangeT ConHead
forall a b. (a -> b) -> a -> b
$ RecordData -> ConHead
_recConHead RecordData
def
reportSDoc "tc.term.rec" 20 $ vcat
[ " xs = " <> pure (P.pretty xs)
, " ftel= " <> prettyTCM (_recTel def)
, " con = " <> pure (P.pretty con)
]
constructorQ <- getQuantity <$> getConstInfo (conName con)
currentQ <- viewTC eQuantity
unless (constructorQ `moreQuantity` currentQ) $ typeError RecordIsErased
disambiguateRecordFields (map _nameFieldA $ lefts mfs) (map unDom $ _recFields def)
fs <- expandModuleAssigns mfs xs
scope <- getScope
let re = Expr -> Range
forall a. HasRange a => a -> Range
getRange Expr
e
meta Name
x = MetaInfo -> Expr
A.Underscore (MetaInfo -> Expr) -> MetaInfo -> Expr
forall a b. (a -> b) -> a -> b
$ Range
-> ScopeInfo -> Maybe MetaId -> ArgName -> MetaKind -> MetaInfo
A.MetaInfo Range
re ScopeInfo
scope Maybe MetaId
forall a. Maybe a
Nothing (Name -> ArgName
forall a. Pretty a => a -> ArgName
prettyShow Name
x) MetaKind
A.UnificationMeta
es <- insertMissingFieldsWarn style r meta fs cxs
args <- checkArguments_ cmp ExpandLast re es (_recTel def `apply` vs) >>= \case
(Elims
elims, Telescope
remainingTel) | Telescope -> Bool
forall a. Null a => a -> Bool
null Telescope
remainingTel
, Just [Arg Term]
args <- Elims -> Maybe [Arg Term]
forall a. [Elim' a] -> Maybe [Arg a]
allApplyElims Elims
elims -> [Arg Term] -> TCMT IO [Arg Term]
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return [Arg Term]
args
(Elims, Telescope)
_ -> TCMT IO [Arg Term]
forall a. HasCallStack => a
__IMPOSSIBLE__
reportSDoc "tc.term.rec" 20 $ text $ "finished record expression"
let origin = case RecStyle
style of
RecStyle
A.RecStyleBrace -> ConOrigin
ConORec
RecStyle
A.RecStyleWhere -> ConOrigin
ConORecWhere
return $ Con con origin (map Apply args)
Term
_ -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
ShouldBeRecordType Type
t
where
guessRecordType :: Type -> TCM Term
guessRecordType Type
t = do
let fields :: [Name]
fields = [ Name
x | Left (FieldAssignment Name
x Expr
_) <- [Either (FieldAssignment' Expr) ModuleName]
mfs ]
rs <- [Name] -> TCM [QName]
findPossibleRecords [Name]
fields
reportSDoc "tc.term.rec" 30 $ "Possible records for" <+> prettyTCM t <+> "are" <?> pretty rs
case rs of
[] -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ [Name] -> TypeError
NoKnownRecordWithSuchFields [Name]
fields
[QName
r] -> do
def <- Definition -> TCMT IO Definition
forall (m :: * -> *).
(Functor m, HasConstInfo m, HasOptions m, ReadTCState m,
MonadTCEnv m, MonadDebug m) =>
Definition -> m Definition
instantiateDef (Definition -> TCMT IO Definition)
-> TCMT IO Definition -> TCMT IO Definition
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< QName -> TCMT IO Definition
forall (m :: * -> *). HasConstInfo m => QName -> m Definition
getConstInfo QName
r
ps <- freeVarsToApply r
let rt = Definition -> Type
defType Definition
def
reportSDoc "tc.term.rec" 30 $ "Type of unique record" <+> prettyTCM rt
vs <- newArgsMeta rt
target <- reduce $ piApply rt vs
s <- case unEl target of
Sort Sort' Term
s -> Sort' Term -> TCMT IO (Sort' Term)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Sort' Term
s
Term
v -> do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"impossible" Int
10 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"The impossible happened when checking record expression against meta"
, TCMT IO Doc
"Candidate record type r = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> QName -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => QName -> m Doc
prettyTCM QName
r
, TCMT IO Doc
"Type of r = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
rt
, TCMT IO Doc
"Ends in (should be sort)= " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Term -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Term -> m Doc
prettyTCM Term
v
, ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc) -> ArgName -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ ArgName
" Raw = " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ Term -> ArgName
forall a. Show a => a -> ArgName
show Term
v
]
TCMT IO (Sort' Term)
forall a. HasCallStack => a
__IMPOSSIBLE__
let inferred = Sort' Term -> Term -> Type
forall t a. Sort' t -> a -> Type'' t a
El Sort' Term
s (Term -> Type) -> Term -> Type
forall a b. (a -> b) -> a -> b
$ QName -> Elims -> Term
Def QName
r (Elims -> Term) -> Elims -> Term
forall a b. (a -> b) -> a -> b
$ (Arg Term -> Elim) -> [Arg Term] -> Elims
forall a b. (a -> b) -> [a] -> [b]
map Arg Term -> Elim
forall a. Arg a -> Elim' a
Apply ([Arg Term]
ps [Arg Term] -> [Arg Term] -> [Arg Term]
forall a. [a] -> [a] -> [a]
++ [Arg Term]
vs)
v <- checkExpr e inferred
coerce cmp v inferred t
QName
_:QName
_:[QName]
_ -> do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.expr.rec" Int
10 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ TCMT IO Doc
"Postponing type checking of"
, Int -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Functor m => Int -> m Doc -> m Doc
nest Int
2 (TCMT IO Doc -> TCMT IO Doc) -> TCMT IO Doc -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ Expr -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA Expr
e TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> TCMT IO Doc
":" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
t
]
TypeCheckingProblem -> TCM Term
postponeTypeCheckingProblem_ (TypeCheckingProblem -> TCM Term)
-> TypeCheckingProblem -> TCM Term
forall a b. (a -> b) -> a -> b
$ Comparison -> Expr -> Type -> TypeCheckingProblem
CheckExpr Comparison
cmp Expr
e Type
t
checkRecordUpdate
:: Comparison
-> A.RecInfo
-> A.Expr
-> A.Assigns
-> A.Expr
-> Type
-> TCM Term
checkRecordUpdate :: Comparison
-> RecInfo -> Expr -> Assigns -> Expr -> Type -> TCM Term
checkRecordUpdate Comparison
cmp ei :: RecInfo
ei@(A.RecInfo Range
_ RecStyle
style) Expr
recexpr Assigns
fs Expr
eupd Type
t = do
Type
-> (Blocker -> Type -> TCM Term)
-> (NotBlocked -> Type -> TCM Term)
-> TCM Term
forall t (m :: * -> *) a.
(Reduce t, IsMeta t, MonadReduce m) =>
t -> (Blocker -> t -> m a) -> (NotBlocked -> t -> m a) -> m a
ifBlocked Type
t (\ Blocker
_ Type
_ -> TCM Term
tryInfer) ((NotBlocked -> Type -> TCM Term) -> TCM Term)
-> (NotBlocked -> Type -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ NotBlocked
_ Type
t' -> do
TCMT IO (Maybe (QName, [Arg Term], RecordData))
-> TCM Term
-> ((QName, [Arg Term], RecordData) -> TCM Term)
-> TCM Term
forall (m :: * -> *) a b.
Monad m =>
m (Maybe a) -> m b -> (a -> m b) -> m b
caseMaybeM (Type -> TCMT IO (Maybe (QName, [Arg Term], RecordData))
forall (m :: * -> *).
PureTCM m =>
Type -> m (Maybe (QName, [Arg Term], RecordData))
isRecordType Type
t') TCM Term
should (((QName, [Arg Term], RecordData) -> TCM Term) -> TCM Term)
-> ((QName, [Arg Term], RecordData) -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ (QName
r, [Arg Term]
_pars, RecordData
defn) -> do
v <- Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp Expr
recexpr Type
t'
name <- freshNoName $ getRange recexpr
addLetBinding defaultArgInfo Inserted name v t' $ do
let projs = (Dom QName -> Arg QName) -> [Dom QName] -> [Arg QName]
forall a b. (a -> b) -> [a] -> [b]
map Dom QName -> Arg QName
forall t a. Dom' t a -> Arg a
argFromDom ([Dom QName] -> [Arg QName]) -> [Dom QName] -> [Arg QName]
forall a b. (a -> b) -> a -> b
$ RecordData -> [Dom QName]
_recFields RecordData
defn
disambiguateRecordFields (map _nameFieldA fs) (map unArg projs)
let fs' = (FieldAssignment' Expr -> (Name, Maybe Expr))
-> Assigns -> [(Name, Maybe Expr)]
forall a b. (a -> b) -> [a] -> [b]
map (\ (FieldAssignment Name
x Expr
e) -> (Name
x, Expr -> Maybe Expr
forall a. a -> Maybe a
Just Expr
e)) Assigns
fs
let axs = (Dom Name -> Arg Name) -> [Dom Name] -> [Arg Name]
forall a b. (a -> b) -> [a] -> [b]
map Dom Name -> Arg Name
forall t a. Dom' t a -> Arg a
argFromDom ([Dom Name] -> [Arg Name]) -> [Dom Name] -> [Arg Name]
forall a b. (a -> b) -> a -> b
$ RecordData -> [Dom Name]
recordFieldNames RecordData
defn
es <- orderFieldsWarn style r (const Nothing) axs fs'
let es' = (Arg QName -> Maybe Expr -> Maybe Expr)
-> [Arg QName] -> [Maybe Expr] -> [Maybe Expr]
forall a b c. (a -> b -> c) -> [a] -> [b] -> [c]
zipWith (Name -> RecInfo -> Arg QName -> Maybe Expr -> Maybe Expr
replaceFields Name
name RecInfo
ei) [Arg QName]
projs [Maybe Expr]
es
let erec = RecInfo -> [Either (FieldAssignment' Expr) ModuleName] -> Expr
A.Rec RecInfo
ei [ FieldAssignment' Expr -> Either (FieldAssignment' Expr) ModuleName
forall a b. a -> Either a b
Left (Name -> Expr -> FieldAssignment' Expr
forall a. Name -> a -> FieldAssignment' a
FieldAssignment Name
x Expr
e) | (Arg ArgInfo
_ Name
x, Just Expr
e) <- [Arg Name] -> [Maybe Expr] -> [(Arg Name, Maybe Expr)]
forall a b. [a] -> [b] -> [(a, b)]
zip [Arg Name]
axs [Maybe Expr]
es' ]
checkExpr' cmp erec t
where
replaceFields :: Name -> A.RecInfo -> Arg A.QName -> Maybe A.Expr -> Maybe A.Expr
replaceFields :: Name -> RecInfo -> Arg QName -> Maybe Expr -> Maybe Expr
replaceFields Name
name RecInfo
ei (Arg ArgInfo
ai QName
p) Maybe Expr
Nothing | ArgInfo -> Bool
forall a. LensHiding a => a -> Bool
visible ArgInfo
ai = Expr -> Maybe Expr
forall a. a -> Maybe a
Just (Expr -> Maybe Expr) -> Expr -> Maybe Expr
forall a b. (a -> b) -> a -> b
$
AppInfo -> Expr -> NamedArg Expr -> Expr
A.App
(Range -> AppInfo
A.defaultAppInfo (Range -> AppInfo) -> Range -> AppInfo
forall a b. (a -> b) -> a -> b
$ RecInfo -> Range
forall a. HasRange a => a -> Range
getRange RecInfo
ei)
(ProjOrigin -> AmbiguousQName -> Expr
A.Proj ProjOrigin
ProjSystem (AmbiguousQName -> Expr) -> AmbiguousQName -> Expr
forall a b. (a -> b) -> a -> b
$ QName -> AmbiguousQName
unambiguous QName
p)
(Expr -> NamedArg Expr
forall a. a -> NamedArg a
defaultNamedArg (Expr -> NamedArg Expr) -> Expr -> NamedArg Expr
forall a b. (a -> b) -> a -> b
$ Name -> Expr
A.Var Name
name)
replaceFields Name
_ RecInfo
_ Arg QName
_ Maybe Expr
me = Maybe Expr
me
tryInfer :: TCM Term
tryInfer = do
(_, trec) <- Expr -> TCM (Term, Type)
inferExpr Expr
recexpr
ifBlocked trec (\ Blocker
_ Type
_ -> TCM Term
postpone) $ \ NotBlocked
_ Type
_ -> do
v <- Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp Expr
eupd Type
trec
coerce cmp v trec t
postpone :: TCM Term
postpone = TypeCheckingProblem -> TCM Term
postponeTypeCheckingProblem_ (TypeCheckingProblem -> TCM Term)
-> TypeCheckingProblem -> TCM Term
forall a b. (a -> b) -> a -> b
$ Comparison -> Expr -> Type -> TypeCheckingProblem
CheckExpr Comparison
cmp Expr
eupd Type
t
should :: TCM Term
should = TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ Type -> TypeError
ShouldBeRecordType Type
t
checkLiteral :: Literal -> Type -> TCM Term
checkLiteral :: Literal -> Type -> TCM Term
checkLiteral Literal
lit Type
t = do
t' <- Literal -> TCM Type
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
Literal -> m Type
litType Literal
lit
coerce CmpEq (Lit lit) t' t
scopedExpr :: A.Expr -> TCM A.Expr
scopedExpr :: Expr -> TCM Expr
scopedExpr (A.ScopedExpr ScopeInfo
scope Expr
e) = ScopeInfo -> TCM ()
setScope ScopeInfo
scope TCM () -> TCM Expr -> TCM Expr
forall a b. TCMT IO a -> TCMT IO b -> TCMT IO b
forall (m :: * -> *) a b. Monad m => m a -> m b -> m b
>> Expr -> TCM Expr
scopedExpr Expr
e
scopedExpr Expr
e = Expr -> TCM Expr
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Expr
e
checkExpr :: A.Expr -> Type -> TCM Term
checkExpr :: Expr -> Type -> TCM Term
checkExpr = Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
CmpLeq
checkExpr'
:: Comparison
-> A.Expr
-> Type
-> TCM Term
checkExpr' :: Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp Expr
e Type
t =
ArgName -> Int -> ArgName -> TCM Term -> TCM Term
forall a. ArgName -> Int -> ArgName -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a.
MonadDebug m =>
ArgName -> Int -> ArgName -> m a -> m a
verboseBracket ArgName
"tc.term.expr.top" Int
5 ArgName
"checkExpr" (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$
ArgName -> Int -> (Term -> TCMT IO Doc) -> TCM Term -> TCM Term
forall (m :: * -> *) a.
MonadDebug m =>
ArgName -> Int -> (a -> TCMT IO Doc) -> m a -> m a
reportResult ArgName
"tc.term.expr.top" Int
15 (\ Term
v -> [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"checkExpr" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<?> [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
fsep [ Expr -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Expr -> m Doc
prettyTCM Expr
e, TCMT IO Doc
":", Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
t ]
, TCMT IO Doc
" returns" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<?> Term -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Term -> m Doc
prettyTCM Term
v ]) (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$
Call -> TCM Term -> TCM Term
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Comparison -> Expr -> Type -> Call
CheckExprCall Comparison
cmp Expr
e Type
t) (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ TCM Term -> TCM Term
forall a. TCM a -> TCM a
localScope (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ TCM Term -> TCM Term
forall a. TCM a -> TCM a
doExpandLast (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ Term -> TCM Term
forall (m :: * -> *). PureTCM m => Term -> m Term
unfoldInlined (Term -> TCM Term) -> TCM Term -> TCM Term
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.expr.top" Int
15 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$
TCMT IO Doc
"Checking" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
fsep [ Expr -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Expr -> m Doc
prettyTCM Expr
e, TCMT IO Doc
":", Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
t ]
, Int -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Functor m => Int -> m Doc -> m Doc
nest Int
2 (TCMT IO Doc -> TCMT IO Doc) -> TCMT IO Doc -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ TCMT IO Doc
"at " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> (ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc)
-> (Range -> ArgName) -> Range -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Range -> ArgName
forall a. Pretty a => a -> ArgName
prettyShow (Range -> TCMT IO Doc) -> TCMT IO Range -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TCMT IO Range
forall (m :: * -> *). MonadTCEnv m => m Range
getCurrentRange)
]
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.expr.top.detailed" Int
80 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$
TCMT IO Doc
"Checking" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
fsep [ Expr -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Expr -> m Doc
prettyTCM Expr
e, TCMT IO Doc
":", ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (Type -> ArgName
forall a. Show a => a -> ArgName
show Type
t) ]
tReduced <- Type -> TCM Type
forall a (m :: * -> *). (Reduce a, MonadReduce m) => a -> m a
reduce Type
t
reportSDoc "tc.term.expr.top" 15 $
" --> " <+> prettyTCM tReduced
e <- scopedExpr e
irrelevantIfProp <- runBlocked (isPropM t) >>= \case
Right Bool
True -> do
let mod :: Modality
mod = Modality
unitModality { modRelevance = irrelevant }
(TCM Term -> TCM Term) -> TCMT IO (TCM Term -> TCM Term)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ((TCM Term -> TCM Term) -> TCMT IO (TCM Term -> TCM Term))
-> (TCM Term -> TCM Term) -> TCMT IO (TCM Term -> TCM Term)
forall a b. (a -> b) -> a -> b
$ (Term -> Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> TCMT IO a -> TCMT IO b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap Term -> Term
dontCare (TCM Term -> TCM Term)
-> (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Modality -> TCM Term -> TCM Term
forall (tcm :: * -> *) m a.
(MonadTCEnv tcm, LensModality m) =>
m -> tcm a -> tcm a
applyModalityToContext Modality
mod
Either Blocker Bool
_ -> (TCM Term -> TCM Term) -> TCMT IO (TCM Term -> TCM Term)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return TCM Term -> TCM Term
forall a. a -> a
id
irrelevantIfProp $ tryInsertHiddenLambda e tReduced $ case e of
A.ScopedExpr ScopeInfo
scope Expr
e -> TCM Term
forall a. HasCallStack => a
__IMPOSSIBLE__
A.QuestionMark MetaInfo
i InteractionId
ii -> (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison -> Type -> MetaInfo -> InteractionId -> TCM Term
checkQuestionMark (RunMetaOccursCheck -> Comparison -> Type -> TCM (MetaId, Term)
forall (m :: * -> *).
MonadMetaSolver m =>
RunMetaOccursCheck -> Comparison -> Type -> m (MetaId, Term)
newValueMeta' RunMetaOccursCheck
RunMetaOccursCheck) Comparison
cmp Type
t MetaInfo
i InteractionId
ii
A.Underscore MetaInfo
i -> MetaInfo -> Comparison -> Type -> TCM Term
checkUnderscore MetaInfo
i Comparison
cmp Type
t
A.WithApp ExprInfo
_ Expr
e List1 Expr
es -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ ArgName -> TypeError
NotImplemented ArgName
"type checking of with application"
e0 :: Expr
e0@(A.App AppInfo
i Expr
q (Arg ArgInfo
ai Named_ Expr
e))
| A.Quote ExprInfo
_ <- Expr -> Expr
unScope Expr
q -> do
if ArgInfo -> Bool
forall a. LensHiding a => a -> Bool
visible ArgInfo
ai then do
x <- Expr -> TCMT IO QName
forall (m :: * -> *).
(MonadTCError m, MonadAbsToCon m) =>
Expr -> m QName
quotedName (Expr -> TCMT IO QName) -> Expr -> TCMT IO QName
forall a b. (a -> b) -> a -> b
$ Named_ Expr -> Expr
forall name a. Named name a -> a
namedThing Named_ Expr
e
ty <- qNameType
coerce cmp (quoteName x) ty t
else TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ CannotQuote -> TypeError
CannotQuote CannotQuote
CannotQuoteHidden
| A.QuoteTerm ExprInfo
_ <- Expr -> Expr
unScope Expr
q -> do
if ArgInfo -> Bool
forall a. LensHiding a => a -> Bool
visible ArgInfo
ai then do
(et, _) <- Expr -> TCM (Term, Type)
inferExpr (Named_ Expr -> Expr
forall name a. Named name a -> a
namedThing Named_ Expr
e)
doQuoteTerm cmp et t
else TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ CannotQuoteTerm -> TypeError
CannotQuoteTerm CannotQuoteTerm
CannotQuoteTermHidden
A.Quote{} -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ CannotQuote -> TypeError
CannotQuote CannotQuote
CannotQuoteNothing
A.QuoteTerm{} -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM Term) -> TypeError -> TCM Term
forall a b. (a -> b) -> a -> b
$ CannotQuoteTerm -> TypeError
CannotQuoteTerm CannotQuoteTerm
CannotQuoteTermNothing
A.Unquote{} -> UnquoteError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
UnquoteError -> m a
unquoteError UnquoteError
NakedUnquote
A.AbsurdLam ExprInfo
i Hiding
h -> Comparison -> ExprInfo -> Hiding -> Expr -> Type -> TCM Term
checkAbsurdLambda Comparison
cmp ExprInfo
i Hiding
h Expr
e Type
t
A.ExtendedLam ExprInfo
i DefInfo
di Erased
erased QName
qname List1 Clause
cs ->
Comparison
-> ExprInfo
-> DefInfo
-> Erased
-> QName
-> List1 Clause
-> Expr
-> Type
-> TCM Term
checkExtendedLambda Comparison
cmp ExprInfo
i DefInfo
di Erased
erased QName
qname List1 Clause
cs Expr
e Type
t
A.Lam ExprInfo
i (A.DomainFull TypedBinding
b) Expr
e -> Comparison -> TypedBinding -> Expr -> Type -> TCM Term
checkLambda Comparison
cmp TypedBinding
b Expr
e Type
t
A.Lam ExprInfo
i (A.DomainFree TacticAttribute
_ NamedArg (Binder' BindName)
x) Expr
e0
| Maybe (WithOrigin (Ranged ArgName)) -> Bool
forall a. Maybe a -> Bool
isNothing (Named (WithOrigin (Ranged ArgName)) (Binder' BindName)
-> Maybe (WithOrigin (Ranged ArgName))
forall name a. Named name a -> Maybe name
nameOf (Named (WithOrigin (Ranged ArgName)) (Binder' BindName)
-> Maybe (WithOrigin (Ranged ArgName)))
-> Named (WithOrigin (Ranged ArgName)) (Binder' BindName)
-> Maybe (WithOrigin (Ranged ArgName))
forall a b. (a -> b) -> a -> b
$ NamedArg (Binder' BindName)
-> Named (WithOrigin (Ranged ArgName)) (Binder' BindName)
forall e. Arg e -> e
unArg NamedArg (Binder' BindName)
x) Bool -> Bool -> Bool
&& Maybe Pattern -> Bool
forall a. Maybe a -> Bool
isNothing (Binder' BindName -> Maybe Pattern
forall a. Binder' a -> Maybe Pattern
A.binderPattern (Binder' BindName -> Maybe Pattern)
-> Binder' BindName -> Maybe Pattern
forall a b. (a -> b) -> a -> b
$ NamedArg (Binder' BindName) -> Binder' BindName
forall a. NamedArg a -> a
namedArg NamedArg (Binder' BindName)
x) ->
Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp (ExprInfo -> LamBinding -> Expr -> Expr
A.Lam ExprInfo
i (ArgInfo -> Binder' Name -> LamBinding
domainFree (NamedArg (Binder' BindName) -> ArgInfo
forall a. LensArgInfo a => a -> ArgInfo
getArgInfo NamedArg (Binder' BindName)
x) (Binder' Name -> LamBinding) -> Binder' Name -> LamBinding
forall a b. (a -> b) -> a -> b
$ BindName -> Name
A.unBind (BindName -> Name) -> Binder' BindName -> Binder' Name
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> NamedArg (Binder' BindName) -> Binder' BindName
forall a. NamedArg a -> a
namedArg NamedArg (Binder' BindName)
x) Expr
e0) Type
t
| Bool
otherwise -> TCM Term
forall a. HasCallStack => a
__IMPOSSIBLE__
A.Lit ExprInfo
_ Literal
lit -> Literal -> Type -> TCM Term
checkLiteral Literal
lit Type
t
A.Let ExprInfo
i List1 LetBinding
ds Expr
e -> List1 LetBinding -> TCM Term -> TCM Term
forall (t :: * -> *) a.
Foldable t =>
t LetBinding -> TCM a -> TCM a
checkLetBindings List1 LetBinding
ds (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp Expr
e Type
t
e :: Expr
e@A.Pi{} -> do
t' <- Expr -> TCM Type
isType_ Expr
e
let s = Type -> Sort' Term
forall a. LensSort a => a -> Sort' Term
getSort Type
t'
v = Type -> Term
forall t a. Type'' t a -> a
unEl Type
t'
coerce cmp v (sort s) t
A.Generalized Set1 QName
s Expr
e -> do
(_, t') <- Set QName -> TCM Type -> TCM ([Maybe QName], Type)
generalizeType (Set1 QName -> Set QName
forall a. NESet a -> Set a
Set1.toSet Set1 QName
s) (TCM Type -> TCM ([Maybe QName], Type))
-> TCM Type -> TCM ([Maybe QName], Type)
forall a b. (a -> b) -> a -> b
$ Expr -> TCM Type
isType_ Expr
e
let s = Type -> Sort' Term
forall a. LensSort a => a -> Sort' Term
getSort Type
t'
v = Type -> Term
forall t a. Type'' t a -> a
unEl Type
t'
coerce cmp v (sort s) t
e :: Expr
e@A.Fun{} -> do
t' <- Expr -> TCM Type
isType_ Expr
e
let s = Type -> Sort' Term
forall a. LensSort a => a -> Sort' Term
getSort Type
t'
v = Type -> Term
forall t a. Type'' t a -> a
unEl Type
t'
coerce cmp v (sort s) t
A.Rec (A.RecInfo Range
_ RecStyle
style) [Either (FieldAssignment' Expr) ModuleName]
fs -> Comparison
-> RecStyle
-> [Either (FieldAssignment' Expr) ModuleName]
-> Expr
-> Type
-> TCM Term
checkRecordExpression Comparison
cmp RecStyle
style [Either (FieldAssignment' Expr) ModuleName]
fs Expr
e Type
t
A.RecUpdate RecInfo
ei Expr
recexpr Assigns
fs -> Comparison
-> RecInfo -> Expr -> Assigns -> Expr -> Type -> TCM Term
checkRecordUpdate Comparison
cmp RecInfo
ei Expr
recexpr Assigns
fs Expr
e Type
t
A.DontCare Expr
e -> do
rel <- Lens' TCEnv Relevance -> TCMT IO Relevance
forall (m :: * -> *) a. MonadTCEnv m => Lens' TCEnv a -> m a
viewTC (Relevance -> f Relevance) -> TCEnv -> f TCEnv
Lens' TCEnv Relevance
eRelevance
if isIrrelevant rel then dontCare <$> do
applyRelevanceToContext rel $ checkExpr' cmp e t
else
internalError "DontCare may only appear in irrelevant contexts"
A.Dot{} -> TypeError -> TCM Term
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError TypeError
InvalidDottedExpression
Expr
_ | Application Expr
hd [NamedArg Expr]
args <- Expr -> AppView' Expr
appView Expr
e -> Comparison -> Expr -> [NamedArg Expr] -> Expr -> Type -> TCM Term
checkApplication Comparison
cmp Expr
hd [NamedArg Expr]
args Expr
e Type
t
`catchIlltypedPatternBlockedOnMeta` \ (TCErr
err, Blocker
x) -> do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term" Int
50 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat ([TCMT IO Doc] -> TCMT IO Doc) -> [TCMT IO Doc] -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$
[ TCMT IO Doc
"checking pattern got stuck on meta: " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Blocker -> TCMT IO Doc
forall (m :: * -> *) a. (Applicative m, Pretty a) => a -> m Doc
pretty Blocker
x ]
TypeCheckingProblem -> Blocker -> TCM Term
postponeTypeCheckingProblem (Comparison -> Expr -> Type -> TypeCheckingProblem
CheckExpr Comparison
cmp Expr
e Type
t) Blocker
x
where
tryInsertHiddenLambda
:: A.Expr
-> Type
-> TCM Term
-> TCM Term
tryInsertHiddenLambda :: Expr -> Type -> TCM Term -> TCM Term
tryInsertHiddenLambda Expr
e Type
tReduced TCM Term
fallback
| Pi (Dom{domInfo :: forall t e. Dom' t e -> ArgInfo
domInfo = ArgInfo
info, unDom :: forall t e. Dom' t e -> e
unDom = Type
a}) Abs Type
b <- Type -> Term
forall t a. Type'' t a -> a
unEl Type
tReduced
, let h :: Hiding
h = ArgInfo -> Hiding
forall a. LensHiding a => a -> Hiding
getHiding ArgInfo
info
, Hiding -> Bool
forall a. LensHiding a => a -> Bool
notVisible Hiding
h
, Bool -> Bool
not (Hiding -> Expr -> Bool
forall {a}. LensHiding a => a -> Expr -> Bool
hiddenLambdaOrHole Hiding
h Expr
e)
= do
let proceed :: TCM Term
proceed = ArgInfo -> ArgName -> TCM Term
doInsert (Origin -> ArgInfo -> ArgInfo
forall a. LensOrigin a => Origin -> a -> a
setOrigin Origin
Inserted ArgInfo
info) (ArgName -> TCM Term) -> ArgName -> TCM Term
forall a b. (a -> b) -> a -> b
$ Abs Type -> ArgName
forall a. Abs a -> ArgName
absName Abs Type
b
expandHidden <- (TCEnv -> ExpandHidden) -> TCMT IO ExpandHidden
forall (m :: * -> *) a. MonadTCEnv m => (TCEnv -> a) -> m a
asksTC TCEnv -> ExpandHidden
envExpandLast
if definitelyIntroduction then proceed else
if expandHidden == ReallyDontExpandLast then fallback else do
reduce a >>= isSizeType >>= \case
Just (BoundedLt Term
u) -> Term
-> (Blocker -> Term -> TCM Term)
-> (NotBlocked -> Term -> TCM Term)
-> TCM Term
forall t (m :: * -> *) a.
(Reduce t, IsMeta t, MonadReduce m) =>
t -> (Blocker -> t -> m a) -> (NotBlocked -> t -> m a) -> m a
ifBlocked Term
u (\ Blocker
_ Term
_ -> TCM Term
fallback) ((NotBlocked -> Term -> TCM Term) -> TCM Term)
-> (NotBlocked -> Term -> TCM Term) -> TCM Term
forall a b. (a -> b) -> a -> b
$ \ NotBlocked
_ Term
v -> do
TCMT IO Bool -> TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *) a. Monad m => m Bool -> m a -> m a -> m a
ifM (Term -> TCMT IO Bool
checkSizeNeverZero Term
v) TCM Term
proceed TCM Term
fallback
TCM Term -> (TCErr -> TCM Term) -> TCM Term
forall a. TCMT IO a -> (TCErr -> TCMT IO a) -> TCMT IO a
forall e (m :: * -> *) a.
MonadError e m =>
m a -> (e -> m a) -> m a
`catchError` \TCErr
_ -> TCM Term
fallback
Maybe BoundedSize
_ -> TCM Term
proceed
| Bool
otherwise = TCM Term
fallback
where
re :: Range
re = Expr -> Range
forall a. HasRange a => a -> Range
getRange Expr
e
rx :: Range
rx = Maybe (Position' SrcFile)
-> Range -> (Position' SrcFile -> Range) -> Range
forall a b. Maybe a -> b -> (a -> b) -> b
caseMaybe (Range -> Maybe (Position' SrcFile)
forall a. Range' a -> Maybe (Position' a)
rStart Range
re) Range
forall a. Range' a
noRange ((Position' SrcFile -> Range) -> Range)
-> (Position' SrcFile -> Range) -> Range
forall a b. (a -> b) -> a -> b
$ \ Position' SrcFile
pos -> Position' SrcFile -> Position' SrcFile -> Range
forall a. Position' a -> Position' a -> Range' a
posToRange Position' SrcFile
pos Position' SrcFile
pos
doInsert :: ArgInfo -> ArgName -> TCM Term
doInsert ArgInfo
info ArgName
y = do
x <- Name -> Name
forall a. LensInScope a => a -> a
C.setNotInScope (Name -> Name) -> TCMT IO Name -> TCMT IO Name
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Range -> ArgName -> TCMT IO Name
forall (m :: * -> *).
MonadFresh NameId m =>
Range -> ArgName -> m Name
freshName Range
rx ArgName
y
reportSLn "tc.term.expr.impl" 15 $ "Inserting implicit lambda"
checkExpr' cmp (A.Lam (A.ExprRange re) (domainFree info $ A.mkBinder x) e) tReduced
hiddenLambdaOrHole :: a -> Expr -> Bool
hiddenLambdaOrHole a
h = \case
A.AbsurdLam ExprInfo
_ Hiding
h' -> a -> Hiding -> Bool
forall a b. (LensHiding a, LensHiding b) => a -> b -> Bool
sameHiding a
h Hiding
h'
A.ExtendedLam ExprInfo
_ DefInfo
_ Erased
_ QName
_ List1 Clause
cls -> (Clause -> Bool) -> List1 Clause -> Bool
forall (t :: * -> *) a. Foldable t => (a -> Bool) -> t a -> Bool
any Clause -> Bool
hiddenLHS List1 Clause
cls
A.Lam ExprInfo
_ LamBinding
bind Expr
_ -> a -> LamBinding -> Bool
forall a b. (LensHiding a, LensHiding b) => a -> b -> Bool
sameHiding a
h LamBinding
bind
A.QuestionMark{} -> Bool
True
Expr
_ -> Bool
False
hiddenLHS :: Clause -> Bool
hiddenLHS (A.Clause (A.LHS LHSInfo
_ (A.LHSHead QName
_ (NamedArg Pattern
a : [NamedArg Pattern]
_))) [ProblemEq]
_ RHS
_ WhereDeclarations
_ Bool
_) = NamedArg Pattern -> Bool
forall a. LensHiding a => a -> Bool
notVisible NamedArg Pattern
a
hiddenLHS Clause
_ = Bool
False
definitelyIntroduction :: Bool
definitelyIntroduction = case Expr
e of
A.Lam{} -> Bool
True
A.AbsurdLam{} -> Bool
True
A.Lit{} -> Bool
True
A.Pi{} -> Bool
True
A.Fun{} -> Bool
True
A.Rec{} -> Bool
True
A.RecUpdate{} -> Bool
True
A.ScopedExpr{} -> Bool
forall a. HasCallStack => a
__IMPOSSIBLE__
Expr
_ -> Bool
False
doQuoteTerm :: Comparison -> Term -> Type -> TCM Term
doQuoteTerm :: Comparison -> Term -> Type -> TCM Term
doQuoteTerm Comparison
cmp Term
et Type
t = do
et' <- Term -> TCM Term
forall (m :: * -> *) a.
(MonadTCEnv m, HasConstInfo m, HasOptions m, TermLike a) =>
a -> m a
etaContract (Term -> TCM Term) -> TCM Term -> TCM Term
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< Term -> TCM Term
forall a (m :: * -> *).
(InstantiateFull a, MonadReduce m) =>
a -> m a
instantiateFull Term
et
case allMetasList et' of
[] -> do
q <- Term -> TCM Term
quoteTerm Term
et'
ty <- el primAgdaTerm
coerce cmp q ty t
[MetaId]
metas -> TypeCheckingProblem -> Blocker -> TCM Term
postponeTypeCheckingProblem (Comparison -> Term -> Type -> TypeCheckingProblem
DoQuoteTerm Comparison
cmp Term
et Type
t) (Blocker -> TCM Term) -> Blocker -> TCM Term
forall a b. (a -> b) -> a -> b
$ Set MetaId -> Blocker
unblockOnAllMetas (Set MetaId -> Blocker) -> Set MetaId -> Blocker
forall a b. (a -> b) -> a -> b
$ [MetaId] -> Set MetaId
forall a. Ord a => [a] -> Set a
Set.fromList [MetaId]
metas
unquoteM :: A.Expr -> Term -> Type -> TCM ()
unquoteM :: Expr -> Term -> Type -> TCM ()
unquoteM Expr
tacA Term
hole Type
holeType = do
tac <- Quantity -> TCM Term -> TCM Term
forall (tcm :: * -> *) q a.
(MonadTCEnv tcm, LensQuantity q) =>
q -> tcm a -> tcm a
applyQuantityToJudgement Quantity
zeroQuantity (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$
Expr -> Type -> TCM Term
checkExpr Expr
tacA (Type -> TCM Term) -> TCM Type -> TCM Term
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< (TCM Term -> TCM Type
forall (m :: * -> *). Functor m => m Term -> m Type
el TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primAgdaTerm TCM Type -> TCM Type -> TCM Type
forall (m :: * -> *). Applicative m => m Type -> m Type -> m Type
--> TCM Term -> TCM Type
forall (m :: * -> *). Functor m => m Term -> m Type
el (TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primAgdaTCM TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *). Applicative m => m Term -> m Term -> m Term
<#> TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primLevelZero TCM Term -> TCM Term -> TCM Term
forall (m :: * -> *). Applicative m => m Term -> m Term -> m Term
<@> TCM Term
forall (m :: * -> *).
(HasBuiltins m, MonadError TCErr m, MonadTCEnv m, ReadTCState m) =>
m Term
primUnit))
inFreshModuleIfFreeParams $ unquoteTactic tac hole holeType
unquoteTactic :: Term -> Term -> Type -> TCM ()
unquoteTactic :: Term -> Term -> Type -> TCM ()
unquoteTactic Term
tac Term
hole Type
goal = do
TCMT IO Bool -> TCM () -> TCM () -> TCM ()
forall (m :: * -> *) a. Monad m => m Bool -> m a -> m a -> m a
ifM (Lens' TCState Bool -> TCMT IO Bool
forall (m :: * -> *) a. ReadTCState m => Lens' TCState a -> m a
useTC (Bool -> f Bool) -> TCState -> f TCState
Lens' TCState Bool
stConsideringInstance) (Blocker -> Constraint -> TCM ()
forall (m :: * -> *).
MonadConstraint m =>
Blocker -> Constraint -> m ()
addConstraint Blocker
neverUnblock (Term -> Term -> Type -> Constraint
UnquoteTactic Term
tac Term
hole Type
goal)) do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.tactic" Int
40 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ TCMT IO Doc
"Running tactic" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Term -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Term -> m Doc
prettyTCM Term
tac
, Int -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Functor m => Int -> m Doc -> m Doc
nest Int
2 (TCMT IO Doc -> TCMT IO Doc) -> TCMT IO Doc -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ TCMT IO Doc
"on" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Term -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Term -> m Doc
prettyTCM Term
hole TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> TCMT IO Doc
":" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
goal ]
ok <- UnquoteM Term -> TCM (Either UnquoteError (Term, [QName]))
forall a. UnquoteM a -> TCM (Either UnquoteError (a, [QName]))
runUnquoteM (UnquoteM Term -> TCM (Either UnquoteError (Term, [QName])))
-> UnquoteM Term -> TCM (Either UnquoteError (Term, [QName]))
forall a b. (a -> b) -> a -> b
$ Term -> Term -> UnquoteM Term
unquoteTCM Term
tac Term
hole
case ok of
Left (BlockedOnMeta TCState
oldState Blocker
blocker) -> do
TCState -> TCM ()
forall (m :: * -> *). MonadTCState m => TCState -> m ()
putTC TCState
oldState
let stripFreshMeta :: MetaId -> f Blocker
stripFreshMeta MetaId
x = Blocker
-> (MetaVariable -> Blocker) -> Maybe MetaVariable -> Blocker
forall b a. b -> (a -> b) -> Maybe a -> b
maybe Blocker
neverUnblock (Blocker -> MetaVariable -> Blocker
forall a b. a -> b -> a
const (Blocker -> MetaVariable -> Blocker)
-> Blocker -> MetaVariable -> Blocker
forall a b. (a -> b) -> a -> b
$ MetaId -> Blocker
unblockOnMeta MetaId
x) (Maybe MetaVariable -> Blocker)
-> f (Maybe MetaVariable) -> f Blocker
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> MetaId -> f (Maybe MetaVariable)
forall (m :: * -> *).
ReadTCState m =>
MetaId -> m (Maybe MetaVariable)
lookupLocalMeta' MetaId
x
blocker' <- (MetaId -> TCMT IO Blocker) -> Blocker -> TCMT IO Blocker
forall (m :: * -> *).
Monad m =>
(MetaId -> m Blocker) -> Blocker -> m Blocker
onBlockingMetasM MetaId -> TCMT IO Blocker
forall {f :: * -> *}. ReadTCState f => MetaId -> f Blocker
stripFreshMeta Blocker
blocker
r <- case Set.toList $ allBlockingMetas blocker' of
MetaId
x : [MetaId]
_ -> Maybe MetaVariable -> Range
forall a. HasRange a => a -> Range
getRange (Maybe MetaVariable -> Range)
-> TCMT IO (Maybe MetaVariable) -> TCMT IO Range
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> MetaId -> TCMT IO (Maybe MetaVariable)
forall (m :: * -> *).
ReadTCState m =>
MetaId -> m (Maybe MetaVariable)
lookupLocalMeta' MetaId
x
[] -> Range -> TCMT IO Range
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Range
forall a. Range' a
noRange
setCurrentRange r $
addConstraint blocker' (UnquoteTactic tac hole goal)
Left UnquoteError
err -> TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM ()) -> TypeError -> TCM ()
forall a b. (a -> b) -> a -> b
$ UnquoteError -> TypeError
UnquoteFailed UnquoteError
err
Right (Term, [QName])
_ -> () -> TCM ()
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ()
checkQuestionMark
:: (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison
-> Type
-> A.MetaInfo
-> InteractionId
-> TCM Term
checkQuestionMark :: (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison -> Type -> MetaInfo -> InteractionId -> TCM Term
checkQuestionMark Comparison -> Type -> TCM (MetaId, Term)
new Comparison
cmp Type
t0 MetaInfo
i InteractionId
ii = do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.interaction" Int
20 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ TCMT IO Doc
"Found interaction point"
, ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc)
-> (IsAbstract -> ArgName) -> IsAbstract -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. IsAbstract -> ArgName
forall a. Show a => a -> ArgName
show (IsAbstract -> TCMT IO Doc) -> TCMT IO IsAbstract -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< (TCEnv -> IsAbstract) -> TCMT IO IsAbstract
forall (m :: * -> *) a. MonadTCEnv m => (TCEnv -> a) -> m a
asksTC (TCEnv -> Lens' TCEnv IsAbstract -> IsAbstract
forall o i. o -> Lens' o i -> i
^. (IsAbstract -> f IsAbstract) -> TCEnv -> f TCEnv
forall a. LensIsAbstract a => Lens' a IsAbstract
Lens' TCEnv IsAbstract
lensIsAbstract)
, InteractionId -> TCMT IO Doc
forall (m :: * -> *) a. (Applicative m, Pretty a) => a -> m Doc
pretty InteractionId
ii
, TCMT IO Doc
":"
, Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
t0
]
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.interaction" Int
60 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ TCMT IO Doc
"Raw:"
, ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (Type -> ArgName
forall a. Show a => a -> ArgName
show Type
t0)
]
MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison
-> Type
-> TCM Term
checkMeta MetaInfo
i ((Comparison -> Type -> TCM (MetaId, Term))
-> InteractionId -> Comparison -> Type -> TCM (MetaId, Term)
newQuestionMark' Comparison -> Type -> TCM (MetaId, Term)
new InteractionId
ii) Comparison
cmp Type
t0
checkUnderscore :: A.MetaInfo -> Comparison -> Type -> TCM Term
checkUnderscore :: MetaInfo -> Comparison -> Type -> TCM Term
checkUnderscore MetaInfo
i = MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison
-> Type
-> TCM Term
checkMeta MetaInfo
i (MetaInfo
-> RunMetaOccursCheck -> Comparison -> Type -> TCM (MetaId, Term)
forall (m :: * -> *).
MonadMetaSolver m =>
MetaInfo
-> RunMetaOccursCheck -> Comparison -> Type -> m (MetaId, Term)
newValueMetaOfKind MetaInfo
i RunMetaOccursCheck
RunMetaOccursCheck)
checkMeta :: A.MetaInfo -> (Comparison -> Type -> TCM (MetaId, Term)) -> Comparison -> Type -> TCM Term
checkMeta :: MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison
-> Type
-> TCM Term
checkMeta MetaInfo
i Comparison -> Type -> TCM (MetaId, Term)
newMeta Comparison
cmp Type
t = (Term, Type) -> Term
forall a b. (a, b) -> a
fst ((Term, Type) -> Term) -> TCM (Term, Type) -> TCM Term
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Maybe (Comparison, Type)
-> TCM (Term, Type)
checkOrInferMeta MetaInfo
i Comparison -> Type -> TCM (MetaId, Term)
newMeta ((Comparison, Type) -> Maybe (Comparison, Type)
forall a. a -> Maybe a
Just (Comparison
cmp , Type
t))
inferMeta :: A.MetaInfo -> (Comparison -> Type -> TCM (MetaId, Term)) -> TCM (Elims -> Term, Type)
inferMeta :: MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> TCM (Elims -> Term, Type)
inferMeta MetaInfo
i Comparison -> Type -> TCM (MetaId, Term)
newMeta = (Term -> Elims -> Term) -> (Term, Type) -> (Elims -> Term, Type)
forall a c b. (a -> c) -> (a, b) -> (c, b)
mapFst Term -> Elims -> Term
forall t. Apply t => t -> Elims -> t
applyE ((Term, Type) -> (Elims -> Term, Type))
-> TCM (Term, Type) -> TCM (Elims -> Term, Type)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Maybe (Comparison, Type)
-> TCM (Term, Type)
checkOrInferMeta MetaInfo
i Comparison -> Type -> TCM (MetaId, Term)
newMeta Maybe (Comparison, Type)
forall a. Maybe a
Nothing
checkOrInferMeta
:: A.MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Maybe (Comparison , Type)
-> TCM (Term, Type)
checkOrInferMeta :: MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Maybe (Comparison, Type)
-> TCM (Term, Type)
checkOrInferMeta MetaInfo
i Comparison -> Type -> TCM (MetaId, Term)
newMeta Maybe (Comparison, Type)
mt = do
case MetaInfo -> Maybe MetaId
A.metaNumber MetaInfo
i of
Maybe MetaId
Nothing -> do
ScopeInfo -> (ScopeInfo -> TCM ()) -> TCM ()
forall (m :: * -> *) a.
(Monad m, Null a) =>
a -> (a -> m ()) -> m ()
unlessNull (MetaInfo -> ScopeInfo
A.metaScope MetaInfo
i) ScopeInfo -> TCM ()
setScope
(cmp , t) <- TCMT IO (Comparison, Type)
-> ((Comparison, Type) -> TCMT IO (Comparison, Type))
-> Maybe (Comparison, Type)
-> TCMT IO (Comparison, Type)
forall b a. b -> (a -> b) -> Maybe a -> b
maybe ((Comparison
CmpEq,) (Type -> (Comparison, Type))
-> TCM Type -> TCMT IO (Comparison, Type)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> TCM Type -> TCM Type
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes TCM Type
newTypeMeta_) (Comparison, Type) -> TCMT IO (Comparison, Type)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return Maybe (Comparison, Type)
mt
(x, v) <- newMeta cmp t
setMetaNameSuggestion x (A.metaNameSuggestion i)
return (v, t)
Just MetaId
x -> do
let v :: Term
v = MetaId -> Elims -> Term
MetaV MetaId
x []
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.meta.check" Int
20 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$
TCMT IO Doc
"checking existing meta " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Term -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Term -> m Doc
prettyTCM Term
v
t' <- MetaId -> TCM Type
forall (m :: * -> *). ReadTCState m => MetaId -> m Type
metaType MetaId
x
reportSDoc "tc.meta.check" 20 $
nest 2 $ "of type " <+> prettyTCM t'
case mt of
Maybe (Comparison, Type)
Nothing -> (Term, Type) -> TCM (Term, Type)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Term
v, Type
t')
Just (Comparison
cmp , Type
t) -> (,Type
t) (Term -> (Term, Type)) -> TCM Term -> TCM (Term, Type)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Comparison -> Term -> Type -> Type -> TCM Term
forall (m :: * -> *).
(MonadConversion m, MonadTCM m) =>
Comparison -> Term -> Type -> Type -> m Term
coerce Comparison
cmp Term
v Type
t' Type
t
domainFree :: ArgInfo -> A.Binder' A.Name -> A.LamBinding
domainFree :: ArgInfo -> Binder' Name -> LamBinding
domainFree ArgInfo
info Binder' Name
x =
TypedBinding -> LamBinding
A.DomainFull (TypedBinding -> LamBinding) -> TypedBinding -> LamBinding
forall a b. (a -> b) -> a -> b
$ Range
-> List1 (NamedArg (Binder' BindName)) -> Expr -> TypedBinding
A.mkTBind Range
r (NamedArg (Binder' BindName) -> List1 (NamedArg (Binder' BindName))
forall el coll. Singleton el coll => el -> coll
singleton (NamedArg (Binder' BindName)
-> List1 (NamedArg (Binder' BindName)))
-> NamedArg (Binder' BindName)
-> List1 (NamedArg (Binder' BindName))
forall a b. (a -> b) -> a -> b
$ ArgInfo -> Binder' BindName -> NamedArg (Binder' BindName)
forall a. ArgInfo -> a -> NamedArg a
unnamedArg ArgInfo
info (Binder' BindName -> NamedArg (Binder' BindName))
-> Binder' BindName -> NamedArg (Binder' BindName)
forall a b. (a -> b) -> a -> b
$ (Name -> BindName) -> Binder' Name -> Binder' BindName
forall a b. (a -> b) -> Binder' a -> Binder' b
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap Name -> BindName
A.mkBindName Binder' Name
x)
(Expr -> TypedBinding) -> Expr -> TypedBinding
forall a b. (a -> b) -> a -> b
$ MetaInfo -> Expr
A.Underscore MetaInfo
underscoreInfo
where
r :: Range
r = Binder' Name -> Range
forall a. HasRange a => a -> Range
getRange Binder' Name
x
underscoreInfo :: MetaInfo
underscoreInfo = A.MetaInfo
{ metaRange :: Range
A.metaRange = Range
r
, metaScope :: ScopeInfo
A.metaScope = ScopeInfo
emptyScopeInfo
, metaNumber :: Maybe MetaId
A.metaNumber = Maybe MetaId
forall a. Maybe a
Nothing
, metaNameSuggestion :: ArgName
A.metaNameSuggestion = Name -> ArgName
forall a. Pretty a => a -> ArgName
prettyShow (Name -> ArgName) -> Name -> ArgName
forall a b. (a -> b) -> a -> b
$ Name -> Name
A.nameConcrete (Name -> Name) -> Name -> Name
forall a b. (a -> b) -> a -> b
$ Binder' Name -> Name
forall a. Binder' a -> a
A.binderName Binder' Name
x
, metaKind :: MetaKind
A.metaKind = MetaKind
A.UnificationMeta
}
checkKnownArguments
:: [NamedArg A.Expr]
-> Args
-> Type
-> TCM (Args, Type)
checkKnownArguments :: [NamedArg Expr] -> [Arg Term] -> Type -> TCM ([Arg Term], Type)
checkKnownArguments [] [Arg Term]
vs Type
t = ([Arg Term], Type) -> TCM ([Arg Term], Type)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ([Arg Term]
vs, Type
t)
checkKnownArguments (NamedArg Expr
arg : [NamedArg Expr]
args) [Arg Term]
vs Type
t = do
(vs', t') <- NamedArg Expr -> TCM ([Arg Term], Type) -> TCM ([Arg Term], Type)
forall (m :: * -> *) x a.
(MonadTrace m, HasRange x) =>
x -> m a -> m a
setCurrentRange NamedArg Expr
arg (TCM ([Arg Term], Type) -> TCM ([Arg Term], Type))
-> TCM ([Arg Term], Type) -> TCM ([Arg Term], Type)
forall a b. (a -> b) -> a -> b
$ NamedArg Expr -> [Arg Term] -> Type -> TCM ([Arg Term], Type)
checkKnownArgument NamedArg Expr
arg [Arg Term]
vs Type
t
checkKnownArguments args vs' t'
checkKnownArgument
:: NamedArg A.Expr
-> Args
-> Type
-> TCM (Args, Type)
checkKnownArgument :: NamedArg Expr -> [Arg Term] -> Type -> TCM ([Arg Term], Type)
checkKnownArgument NamedArg Expr
arg [] Type
_ = TypeError -> TCM ([Arg Term], Type)
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM ([Arg Term], Type))
-> TypeError -> TCM ([Arg Term], Type)
forall a b. (a -> b) -> a -> b
$ NamedArg Expr -> TypeError
InvalidProjectionParameter NamedArg Expr
arg
checkKnownArgument NamedArg Expr
arg (Arg ArgInfo
_ Term
v : [Arg Term]
vs) Type
t = do
(dom@Dom{ unDom = a }, b) <- Type -> TCMT IO (Dom Type, Abs Type)
forall (m :: * -> *).
MonadReduce m =>
Type -> m (Dom Type, Abs Type)
mustBePi Type
t
if not $ fromMaybe __IMPOSSIBLE__ $ fittingNamedArg arg dom
then checkKnownArgument arg vs (b `absApp` v)
else do
u <- checkNamedArg arg a
equalTerm a u v
return (vs, b `absApp` v)
checkNamedArg :: NamedArg A.Expr -> Type -> TCM Term
checkNamedArg :: NamedArg Expr -> Type -> TCM Term
checkNamedArg arg :: NamedArg Expr
arg@(Arg ArgInfo
info Named_ Expr
e0) Type
t0 = do
let e :: Expr
e = Named_ Expr -> Expr
forall name a. Named name a -> a
namedThing Named_ Expr
e0
let x :: ArgName
x = ArgName -> Named_ Expr -> ArgName
forall a.
(LensNamed a, NameOf a ~ WithOrigin (Ranged ArgName)) =>
ArgName -> a -> ArgName
bareNameWithDefault ArgName
"" Named_ Expr
e0
Call -> TCM Term -> TCM Term
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Comparison -> Expr -> Type -> Call
CheckExprCall Comparison
CmpLeq Expr
e Type
t0) (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.args.named" Int
15 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ do
TCMT IO Doc
"Checking named arg" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
sep
[ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
fsep [ NamedArg Expr -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => NamedArg Expr -> m Doc
prettyTCM NamedArg Expr
arg, TCMT IO Doc
":", Type -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Type -> m Doc
prettyTCM Type
t0 ]
]
ArgName -> Int -> ArgName -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> ArgName -> m ()
reportSLn ArgName
"tc.term.args.named" Int
75 (ArgName -> TCM ()) -> ArgName -> TCM ()
forall a b. (a -> b) -> a -> b
$ ArgName
" arg = " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ NamedArg Expr -> ArgName
forall a. Show a => a -> ArgName
show (NamedArg Expr -> NamedArg Expr
forall a. ExprLike a => a -> a
deepUnscope NamedArg Expr
arg)
let checkU :: MetaInfo -> TCM Term
checkU MetaInfo
i = MetaInfo
-> (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison
-> Type
-> TCM Term
checkMeta MetaInfo
i (MetaKind
-> ArgInfo -> ArgName -> Comparison -> Type -> TCM (MetaId, Term)
forall (m :: * -> *).
(PureTCM m, MonadMetaSolver m) =>
MetaKind
-> ArgInfo -> ArgName -> Comparison -> Type -> m (MetaId, Term)
newMetaArg (MetaInfo -> MetaKind
A.metaKind MetaInfo
i) ArgInfo
info ArgName
x) Comparison
CmpLeq Type
t0
let checkQ :: MetaInfo -> InteractionId -> TCM Term
checkQ = (Comparison -> Type -> TCM (MetaId, Term))
-> Comparison -> Type -> MetaInfo -> InteractionId -> TCM Term
checkQuestionMark (ArgInfo -> ArgName -> Comparison -> Type -> TCM (MetaId, Term)
newInteractionMetaArg ArgInfo
info ArgName
x) Comparison
CmpLeq Type
t0
if Bool -> Bool
not (Bool -> Bool) -> Bool -> Bool
forall a b. (a -> b) -> a -> b
$ Expr -> Bool
isHole Expr
e then Expr -> Type -> TCM Term
checkExpr Expr
e Type
t0 else TCM Term -> TCM Term
forall a. TCM a -> TCM a
localScope (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ do
Expr -> TCM Expr
scopedExpr Expr
e TCM Expr -> (Expr -> TCM Term) -> TCM Term
forall a b. TCMT IO a -> (a -> TCMT IO b) -> TCMT IO b
forall (m :: * -> *) a b. Monad m => m a -> (a -> m b) -> m b
>>= \case
A.Underscore MetaInfo
i -> MetaInfo -> TCM Term
checkU MetaInfo
i
A.QuestionMark MetaInfo
i InteractionId
ii -> MetaInfo -> InteractionId -> TCM Term
checkQ MetaInfo
i InteractionId
ii
Expr
_ -> TCM Term
forall a. HasCallStack => a
__IMPOSSIBLE__
where
isHole :: Expr -> Bool
isHole A.Underscore{} = Bool
True
isHole A.QuestionMark{} = Bool
True
isHole (A.ScopedExpr ScopeInfo
_ Expr
e) = Expr -> Bool
isHole Expr
e
isHole Expr
_ = Bool
False
inferExpr :: A.Expr -> TCM (Term, Type)
inferExpr :: Expr -> TCM (Term, Type)
inferExpr = ExpandHidden -> Expr -> TCM (Term, Type)
inferExpr' ExpandHidden
DontExpandLast
inferExpr' :: ExpandHidden -> A.Expr -> TCM (Term, Type)
inferExpr' :: ExpandHidden -> Expr -> TCM (Term, Type)
inferExpr' ExpandHidden
exh Expr
e = Call -> TCM (Term, Type) -> TCM (Term, Type)
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Expr -> Call
InferExpr Expr
e) (TCM (Term, Type) -> TCM (Term, Type))
-> TCM (Term, Type) -> TCM (Term, Type)
forall a b. (a -> b) -> a -> b
$ do
let Application Expr
hd [NamedArg Expr]
args = Expr -> AppView' Expr
appView Expr
e
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.infer" Int
30 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"inferExpr': appView of " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Expr -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA Expr
e
, TCMT IO Doc
" hd = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Expr -> TCMT IO Doc
forall a (m :: * -> *).
(ToConcrete a, Pretty (ConOfAbs a), MonadAbsToCon m) =>
a -> m Doc
prettyA Expr
hd
, TCMT IO Doc
" args = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> [NamedArg Expr] -> TCMT IO Doc
forall a ce (m :: * -> *).
(ToConcrete a, ConOfAbs a ~ [ce], Pretty ce, MonadAbsToCon m) =>
a -> m Doc
prettyAs [NamedArg Expr]
args
]
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.infer" Int
60 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc) -> ArgName -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ ArgName
" hd (raw) = " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ Expr -> ArgName
forall a. Show a => a -> ArgName
show Expr
hd
]
ExpandHidden -> Expr -> [NamedArg Expr] -> Expr -> TCM (Term, Type)
inferApplication ExpandHidden
exh Expr
hd [NamedArg Expr]
args Expr
e
defOrVar :: A.Expr -> Bool
defOrVar :: Expr -> Bool
defOrVar A.Var{} = Bool
True
defOrVar A.Def'{} = Bool
True
defOrVar A.Proj{} = Bool
True
defOrVar (A.ScopedExpr ScopeInfo
_ Expr
e) = Expr -> Bool
defOrVar Expr
e
defOrVar Expr
_ = Bool
False
checkDontExpandLast :: Comparison -> A.Expr -> Type -> TCM Term
checkDontExpandLast :: Comparison -> Expr -> Type -> TCM Term
checkDontExpandLast Comparison
cmp Expr
e Type
t = case Expr
e of
Expr
_ | Application Expr
hd [NamedArg Expr]
args <- Expr -> AppView' Expr
appView Expr
e, Expr -> Bool
defOrVar Expr
hd ->
Call -> TCM Term -> TCM Term
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Comparison -> Expr -> Type -> Call
CheckExprCall Comparison
cmp Expr
e Type
t) (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ TCM Term -> TCM Term
forall a. TCM a -> TCM a
localScope (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ TCM Term -> TCM Term
forall a. TCM a -> TCM a
dontExpandLast (TCM Term -> TCM Term) -> TCM Term -> TCM Term
forall a b. (a -> b) -> a -> b
$ do
Comparison -> Expr -> [NamedArg Expr] -> Expr -> Type -> TCM Term
checkApplication Comparison
cmp Expr
hd [NamedArg Expr]
args Expr
e Type
t
Expr
_ -> Comparison -> Expr -> Type -> TCM Term
checkExpr' Comparison
cmp Expr
e Type
t
isModuleFreeVar :: Int -> TCM Bool
isModuleFreeVar :: Int -> TCMT IO Bool
isModuleFreeVar Int
i = do
params <- ModuleName -> TCMT IO [Arg Term]
forall (m :: * -> *).
(Functor m, Applicative m, HasOptions m, MonadTCEnv m,
ReadTCState m, MonadDebug m) =>
ModuleName -> m [Arg Term]
moduleParamsToApply (ModuleName -> TCMT IO [Arg Term])
-> TCMT IO ModuleName -> TCMT IO [Arg Term]
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TCMT IO ModuleName
forall (m :: * -> *). MonadTCEnv m => m ModuleName
currentModule
return $ any ((== Var i []) . unArg) params
inferExprForWith :: Arg A.Expr -> TCM (Term, Type)
inferExprForWith :: Arg Expr -> TCM (Term, Type)
inferExprForWith (Arg ArgInfo
info Expr
e) = ArgName -> Int -> ArgName -> TCM (Term, Type) -> TCM (Term, Type)
forall a. ArgName -> Int -> ArgName -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a.
MonadDebug m =>
ArgName -> Int -> ArgName -> m a -> m a
verboseBracket ArgName
"tc.with.infer" Int
20 ArgName
"inferExprForWith" (TCM (Term, Type) -> TCM (Term, Type))
-> TCM (Term, Type) -> TCM (Term, Type)
forall a b. (a -> b) -> a -> b
$
Relevance -> TCM (Term, Type) -> TCM (Term, Type)
forall (tcm :: * -> *) r a.
(MonadTCEnv tcm, LensRelevance r) =>
r -> tcm a -> tcm a
applyRelevanceToContext (ArgInfo -> Relevance
forall a. LensRelevance a => a -> Relevance
getRelevance ArgInfo
info) (TCM (Term, Type) -> TCM (Term, Type))
-> TCM (Term, Type) -> TCM (Term, Type)
forall a b. (a -> b) -> a -> b
$ do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.with.infer" Int
20 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ TCMT IO Doc
"inferExprForWith " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Expr -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Expr -> m Doc
prettyTCM Expr
e
ArgName -> Int -> ArgName -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> ArgName -> m ()
reportSLn ArgName
"tc.with.infer" Int
80 (ArgName -> TCM ()) -> ArgName -> TCM ()
forall a b. (a -> b) -> a -> b
$ ArgName
"inferExprForWith " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ Expr -> ArgName
forall a. Show a => a -> ArgName
show (Expr -> Expr
forall a. ExprLike a => a -> a
deepUnscope Expr
e)
Call -> TCM (Term, Type) -> TCM (Term, Type)
forall a. Call -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) a. MonadTrace m => Call -> m a -> m a
traceCall (Expr -> Call
InferExpr Expr
e) (TCM (Term, Type) -> TCM (Term, Type))
-> TCM (Term, Type) -> TCM (Term, Type)
forall a b. (a -> b) -> a -> b
$ do
(v, t) <- (Term, Type) -> TCM (Term, Type)
forall a (m :: * -> *).
(InstantiateFull a, MonadReduce m) =>
a -> m a
instantiateFull ((Term, Type) -> TCM (Term, Type))
-> TCM (Term, Type) -> TCM (Term, Type)
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< Expr -> TCM (Term, Type)
inferExpr Expr
e
v <- reduce v
case v of
Var Int
i [] -> TCMT IO Bool -> TCM () -> TCM ()
forall (m :: * -> *). Monad m => m Bool -> m () -> m ()
whenM (Int -> TCMT IO Bool
isModuleFreeVar Int
i) (TCM () -> TCM ()) -> TCM () -> TCM ()
forall a b. (a -> b) -> a -> b
$ do
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.with.infer" Int
80 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc) -> ArgName -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ ArgName
"with expression is variable " ArgName -> ArgName -> ArgName
forall a. [a] -> [a] -> [a]
++ Int -> ArgName
forall a. Show a => a -> ArgName
show Int
i
, TCMT IO Doc
"current modules = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> do ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc)
-> (ModuleName -> ArgName) -> ModuleName -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. ModuleName -> ArgName
forall a. Show a => a -> ArgName
show (ModuleName -> TCMT IO Doc) -> TCMT IO ModuleName -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TCMT IO ModuleName
forall (m :: * -> *). MonadTCEnv m => m ModuleName
currentModule
, TCMT IO Doc
"current module free vars = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> do ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc) -> (Int -> ArgName) -> Int -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Int -> ArgName
forall a. Show a => a -> ArgName
show (Int -> TCMT IO Doc) -> TCMT IO Int -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TCMT IO Int
getCurrentModuleFreeVars
, TCMT IO Doc
"context size = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> do ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc) -> (Int -> ArgName) -> Int -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. Int -> ArgName
forall a. Show a => a -> ArgName
show (Int -> TCMT IO Doc) -> TCMT IO Int -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TCMT IO Int
forall (m :: * -> *). (Applicative m, MonadTCEnv m) => m Int
getContextSize
, TCMT IO Doc
"current context = " TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> do Telescope -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Telescope -> m Doc
prettyTCM (Telescope -> TCMT IO Doc) -> TCMT IO Telescope -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< TCMT IO Telescope
forall (m :: * -> *). (Applicative m, MonadTCEnv m) => m Telescope
getContextTelescope
]
TypeError -> TCM ()
forall (m :: * -> *) a.
(HasCallStack, MonadTCError m) =>
TypeError -> m a
typeError (TypeError -> TCM ()) -> TypeError -> TCM ()
forall a b. (a -> b) -> a -> b
$ Expr -> Term -> TypeError
WithOnFreeVariable Expr
e Term
v
Term
_ -> () -> TCM ()
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return ()
TelV tel t0 <- telViewUpTo' (-1) (not . visible) t
(v, t) <- case unEl t0 of
Def QName
d Elims
vs -> do
QName -> TCM (Maybe DataOrRecord)
isDataOrRecordType QName
d TCM (Maybe DataOrRecord)
-> (Maybe DataOrRecord -> TCM (Term, Type)) -> TCM (Term, Type)
forall a b. TCMT IO a -> (a -> TCMT IO b) -> TCMT IO b
forall (m :: * -> *) a b. Monad m => m a -> (a -> m b) -> m b
>>= \case
Maybe DataOrRecord
Nothing -> (Term, Type) -> TCM (Term, Type)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Term
v, Type
t)
Just{} -> do
(args, t1) <- Int -> (Hiding -> Bool) -> Type -> TCM ([Arg Term], Type)
forall (m :: * -> *).
(PureTCM m, MonadMetaSolver m, MonadTCM m) =>
Int -> (Hiding -> Bool) -> Type -> m ([Arg Term], Type)
implicitArgs (-Int
1) Hiding -> Bool
forall a. LensHiding a => a -> Bool
notVisible Type
t
return (v `apply` args, t1)
Term
_ -> (Term, Type) -> TCM (Term, Type)
forall a. a -> TCMT IO a
forall (m :: * -> *) a. Monad m => a -> m a
return (Term
v, Type
t)
solveAwakeConstraints
return (v, t)
checkLetBindings' :: Foldable t => t A.LetBinding -> TCM a -> TCM a
checkLetBindings' :: forall (t :: * -> *) a.
Foldable t =>
t LetBinding -> TCM a -> TCM a
checkLetBindings' = (LetBinding -> (TCM a -> TCM a) -> TCM a -> TCM a)
-> (TCM a -> TCM a) -> t LetBinding -> TCM a -> TCM a
forall a b. (a -> b -> b) -> b -> t a -> b
forall (t :: * -> *) a b.
Foldable t =>
(a -> b -> b) -> b -> t a -> b
foldr ((TCM a -> TCM a) -> (TCM a -> TCM a) -> TCM a -> TCM a
forall b c a. (b -> c) -> (a -> b) -> a -> c
(.) ((TCM a -> TCM a) -> (TCM a -> TCM a) -> TCM a -> TCM a)
-> (LetBinding -> TCM a -> TCM a)
-> LetBinding
-> (TCM a -> TCM a)
-> TCM a
-> TCM a
forall b c a. (b -> c) -> (a -> b) -> a -> c
. LetBinding -> TCM a -> TCM a
forall a. LetBinding -> TCM a -> TCM a
checkLetBinding') TCM a -> TCM a
forall a. a -> a
id
checkLetBinding' :: A.LetBinding -> TCM a -> TCM a
checkLetBinding' :: forall a. LetBinding -> TCM a -> TCM a
checkLetBinding' b :: LetBinding
b@(A.LetBind LetInfo
i ArgInfo
info BindName
x Expr
t Expr
e) TCM a
ret = do
let
check :: Comparison -> Expr -> Type -> TCM Term
check
| ArgInfo -> Origin
forall a. LensOrigin a => a -> Origin
getOrigin ArgInfo
info Origin -> Origin -> Bool
forall a. Eq a => a -> a -> Bool
== Origin
Inserted = Comparison -> Expr -> Type -> TCM Term
checkDontExpandLast
| Bool
otherwise = Comparison -> Expr -> Type -> TCM Term
checkExpr'
t <- TCM Type -> TCM Type
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ Expr -> TCM Type
isType_ Expr
t
v <- applyModalityToContext info $ check CmpLeq e t
addLetBinding info UserWritten (A.unBind x) v t ret
checkLetBinding' b :: LetBinding
b@(A.LetAxiom LetInfo
i ArgInfo
info BindName
x Expr
t) TCM a
ret = do
t <- TCM Type -> TCM Type
forall (m :: * -> *) a.
(MonadTCEnv m, HasOptions m, MonadDebug m) =>
m a -> m a
workOnTypes (TCM Type -> TCM Type) -> TCM Type -> TCM Type
forall a b. (a -> b) -> a -> b
$ Expr -> TCM Type
isType_ Expr
t
current <- currentModule
axn <- qualify current <$> freshName_ (A.unBind x)
addConstant' axn info t defaultAxiom
val <- Def axn . fmap Apply <$> getContextArgs
addLetBinding info UserWritten (A.unBind x) val t ret
checkLetBinding' b :: LetBinding
b@(A.LetPatBind LetInfo
i Pattern
p Expr
e) TCM a
ret = do
p <- Pattern -> TCM Pattern
forall a. ExpandPatternSynonyms a => a -> TCM a
expandPatternSynonyms Pattern
p
(v, t) <- inferExpr' ExpandLast e
let
t0 = Sort' Term -> Term -> Type
forall t a. Sort' t -> a -> Type'' t a
El (Type -> Sort' Term
forall a. LensSort a => a -> Sort' Term
getSort Type
t) (Term -> Type) -> Term -> Type
forall a b. (a -> b) -> a -> b
$ Dom Type -> Abs Type -> Term
Pi (Type -> Dom Type
forall a. a -> Dom a
defaultDom Type
t) (ArgName -> Type -> Abs Type
forall a. ArgName -> a -> Abs a
NoAbs ArgName
forall a. Underscore a => a
underscore Type
HasCallStack => Type
__DUMMY_TYPE__)
p0 = ArgInfo
-> Named (WithOrigin (Ranged ArgName)) Pattern -> NamedArg Pattern
forall e. ArgInfo -> e -> Arg e
Arg ArgInfo
defaultArgInfo (Maybe (WithOrigin (Ranged ArgName))
-> Pattern -> Named (WithOrigin (Ranged ArgName)) Pattern
forall name a. Maybe name -> a -> Named name a
Named Maybe (WithOrigin (Ranged ArgName))
forall a. Maybe a
Nothing Pattern
p)
reportSDoc "tc.term.let.pattern" 10 $ vcat
[ "let-binding pattern p at type t"
, nest 2 $ vcat
[ "p (A) =" <+> prettyA p
, "t =" <+> prettyTCM t
, "cxtRel=" <+> do pretty =<< viewTC eRelevance
, "cxtQnt=" <+> do pretty =<< viewTC eQuantity
]
]
fvs <- getContextSize
checkLeftHandSide (CheckPattern p EmptyTel t) noRange Nothing [p0] t0 Nothing [] $ \ (LHSResult Int
_ Telescope
delta0 NAPs
ps Bool
_ Arg Type
_t Substitution
_ [AsBinding]
asb IntSet
_ Bool
_) -> [AsBinding] -> TCM a -> TCM a
forall a. [AsBinding] -> TCM a -> TCM a
bindAsPatterns [AsBinding]
asb (TCM a -> TCM a) -> TCM a -> TCM a
forall a b. (a -> b) -> a -> b
$ do
let p :: DeBruijnPattern
p = case Int -> NAPs -> NAPs
forall a. Int -> [a] -> [a]
drop Int
fvs NAPs
ps of [Arg (Named_ DeBruijnPattern)
p] -> Arg (Named_ DeBruijnPattern) -> DeBruijnPattern
forall a. NamedArg a -> a
namedArg Arg (Named_ DeBruijnPattern)
p; NAPs
_ -> DeBruijnPattern
forall a. HasCallStack => a
__IMPOSSIBLE__
delta :: Telescope
delta = ListTel -> Telescope
telFromList (ListTel -> Telescope) -> ListTel -> Telescope
forall a b. (a -> b) -> a -> b
$ Int -> ListTel -> ListTel
forall a. Int -> [a] -> [a]
drop Int
fvs (ListTel -> ListTel) -> ListTel -> ListTel
forall a b. (a -> b) -> a -> b
$ Telescope -> ListTel
forall t. Tele (Dom t) -> [Dom (ArgName, t)]
telToList Telescope
delta0
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.let.pattern" Int
20 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ Int -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Functor m => Int -> m Doc -> m Doc
nest Int
2 (TCMT IO Doc -> TCMT IO Doc) -> TCMT IO Doc -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"p (I) =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> DeBruijnPattern -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => DeBruijnPattern -> m Doc
prettyTCM DeBruijnPattern
p
, TCMT IO Doc
"delta =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> Telescope -> TCMT IO Doc
forall a (m :: * -> *). (PrettyTCM a, MonadPretty m) => a -> m Doc
forall (m :: * -> *). MonadPretty m => Telescope -> m Doc
prettyTCM Telescope
delta
, TCMT IO Doc
"cxtRel=" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> do Relevance -> TCMT IO Doc
forall (m :: * -> *) a. (Applicative m, Pretty a) => a -> m Doc
pretty (Relevance -> TCMT IO Doc) -> TCMT IO Relevance -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< Lens' TCEnv Relevance -> TCMT IO Relevance
forall (m :: * -> *) a. MonadTCEnv m => Lens' TCEnv a -> m a
viewTC (Relevance -> f Relevance) -> TCEnv -> f TCEnv
Lens' TCEnv Relevance
eRelevance
, TCMT IO Doc
"cxtQnt=" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> do Quantity -> TCMT IO Doc
forall (m :: * -> *) a. (Applicative m, Pretty a) => a -> m Doc
pretty (Quantity -> TCMT IO Doc) -> TCMT IO Quantity -> TCMT IO Doc
forall (m :: * -> *) a b. Monad m => (a -> m b) -> m a -> m b
=<< Lens' TCEnv Quantity -> TCMT IO Quantity
forall (m :: * -> *) a. MonadTCEnv m => Lens' TCEnv a -> m a
viewTC (Quantity -> f Quantity) -> TCEnv -> f TCEnv
Lens' TCEnv Quantity
eQuantity
]
ArgName -> Int -> TCMT IO Doc -> TCM ()
forall (m :: * -> *).
MonadDebug m =>
ArgName -> Int -> TCMT IO Doc -> m ()
reportSDoc ArgName
"tc.term.let.pattern" Int
80 (TCMT IO Doc -> TCM ()) -> TCMT IO Doc -> TCM ()
forall a b. (a -> b) -> a -> b
$ Int -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Functor m => Int -> m Doc -> m Doc
nest Int
2 (TCMT IO Doc -> TCMT IO Doc) -> TCMT IO Doc -> TCMT IO Doc
forall a b. (a -> b) -> a -> b
$ [TCMT IO Doc] -> TCMT IO Doc
forall (m :: * -> *) (t :: * -> *).
(Applicative m, Foldable t) =>
t (m Doc) -> m Doc
vcat
[ TCMT IO Doc
"p (I) =" TCMT IO Doc -> TCMT IO Doc -> TCMT IO Doc
forall (m :: * -> *). Applicative m => m Doc -> m Doc -> m Doc
<+> (ArgName -> TCMT IO Doc
forall (m :: * -> *). Applicative m => ArgName -> m Doc
text (ArgName -> TCMT IO Doc)
-> (DeBruijnPattern -> ArgName) -> DeBruijnPattern -> TCMT IO Doc
forall b c a. (b -> c) -> (a -> b) -> a -> c
. DeBruijnPattern -> ArgName
forall a. Show a => a -> ArgName
show) DeBruijnPattern
p
]
fs <- DeBruijnPattern -> TCM [Term -> Term]
recordPatternToProjections DeBruijnPattern
p
cxt0 <- getContext
let (binds, cxt) = splitAt (size delta) cxt0
toDrop = [ContextEntry] -> Int
forall a. [a] -> Int
forall (t :: * -> *) a. Foldable t => t a -> Int
length [ContextEntry]
binds
sigma = ((Term -> Term) -> Term) -> [Term -> Term] -> [Term]
forall a b. (a -> b) -> [a] -> [b]
map ((Term -> Term) -> Term -> Term
forall a b. (a -> b) -> a -> b
$ Term
v) [Term -> Term]
fs
sub = [Term] -> Substitution
forall a. DeBruijn a => [a] -> Substitution' a
parallelS ([Term] -> [Term]
forall a. [a] -> [a]
reverse [Term]
sigma)
updateContext sub (drop toDrop) $ do
reportSDoc "tc.term.let.pattern" 20 $ nest 2 $ vcat
[ "delta =" <+> prettyTCM delta
, "binds =" <+> prettyTCM binds
]
let fdelta = Telescope -> [Dom Type]
forall a. TermSubst a => Tele (Dom a) -> [Dom a]
flattenTel Telescope
delta
reportSDoc "tc.term.let.pattern" 20 $ nest 2 $ vcat
[ "fdelta =" <+> addContext delta (prettyTCM fdelta)
]
let tsl = Substitution' (SubstArg [Dom Type]) -> [Dom Type] -> [Dom Type]
forall a. Subst a => Substitution' (SubstArg a) -> a -> a
applySubst Substitution
Substitution' (SubstArg [Dom Type])
sub [Dom Type]
fdelta
let ts = (Dom Type -> Type) -> [Dom Type] -> [Type]
forall a b. (a -> b) -> [a] -> [b]
map Dom Type -> Type
forall t e. Dom' t e -> e
unDom [Dom Type]
tsl
let infos = (Dom Type -> ArgInfo) -> [Dom Type] -> [ArgInfo]
forall a b. (a -> b) -> [a] -> [b]
map Dom Type -> ArgInfo
forall t e. Dom' t e -> ArgInfo
domInfo [Dom Type]
tsl
let xs = (ContextEntry -> Name) -> [ContextEntry] -> [Name]
forall a b. (a -> b) -> [a] -> [b]
map ((Name, Type) -> Name
forall a b. (a, b) -> a
fst ((Name, Type) -> Name)
-> (ContextEntry -> (Name, Type)) -> ContextEntry -> Name
forall b c a. (b -> c) -> (a -> b) -> a -> c
. ContextEntry -> (Name, Type)
forall t e. Dom' t e -> e
unDom) ([ContextEntry] -> [ContextEntry]
forall a. [a] -> [a]
reverse [ContextEntry]
binds)
foldr (uncurry4 $ flip addLetBinding UserWritten) ret $ List.zip4 infos xs sigma ts
checkLetBinding' (A.LetApply ModuleInfo
i Erased
erased ModuleName
x ModuleApplication
modapp ScopeCopyInfo
copyInfo ImportDirective
dir) TCM a
ret = do
fv <- TCMT IO Int
getCurrentModuleFreeVars
n <- getContextSize
let new = Int
n Int -> Int -> Int
forall a. Num a => a -> a -> a
- Int
fv
reportSDoc "tc.term.let.apply" 10 $ "Applying" <+> pretty x <+> prettyA modapp <?> ("with" <+> pshow new <+> "free variables")
reportSDoc "tc.term.let.apply" 20 $ vcat
[ "context =" <+> (prettyTCM =<< getContextTelescope)
, "module =" <+> (prettyTCM =<< currentModule)
, "fv =" <+> text (show fv)
]
checkSectionApplication i erased x modapp copyInfo
dir{ publicOpen = Nothing }
withAnonymousModule x new ret
checkLetBinding' A.LetOpen{} TCM a
ret = TCM a
ret
checkLetBinding' (A.LetDeclaredVariable BindName
_) TCM a
ret = TCM a
ret
checkLetBinding :: A.LetBinding -> TCM a -> TCM a
checkLetBinding :: forall a. LetBinding -> TCM a -> TCM a
checkLetBinding LetBinding
b = Call -> (TCMT IO a -> TCMT IO a) -> TCMT IO a -> TCMT IO a
forall (m :: * -> *) b.
MonadTrace m =>
Call -> (m b -> m b) -> m b -> m b
traceCallCPS' (LetBinding -> Call
CheckLetBinding LetBinding
b) (LetBinding -> TCMT IO a -> TCMT IO a
forall a. LetBinding -> TCM a -> TCM a
checkLetBinding' LetBinding
b)
checkLetBindings :: Foldable t => t A.LetBinding -> TCM a -> TCM a
checkLetBindings :: forall (t :: * -> *) a.
Foldable t =>
t LetBinding -> TCM a -> TCM a
checkLetBindings = (LetBinding -> (TCM a -> TCM a) -> TCM a -> TCM a)
-> (TCM a -> TCM a) -> t LetBinding -> TCM a -> TCM a
forall a b. (a -> b -> b) -> b -> t a -> b
forall (t :: * -> *) a b.
Foldable t =>
(a -> b -> b) -> b -> t a -> b
foldr ((TCM a -> TCM a) -> (TCM a -> TCM a) -> TCM a -> TCM a
forall b c a. (b -> c) -> (a -> b) -> a -> c
(.) ((TCM a -> TCM a) -> (TCM a -> TCM a) -> TCM a -> TCM a)
-> (LetBinding -> TCM a -> TCM a)
-> LetBinding
-> (TCM a -> TCM a)
-> TCM a
-> TCM a
forall b c a. (b -> c) -> (a -> b) -> a -> c
. LetBinding -> TCM a -> TCM a
forall a. LetBinding -> TCM a -> TCM a
checkLetBinding) TCM a -> TCM a
forall a. a -> a
id