module GHC.Core.Lint (
lintCoreBindings, lintUnfolding,
lintPassResult, lintInteractiveExpr, lintExpr,
lintAnnots, lintAxioms,
endPass, endPassIO,
dumpPassResult,
GHC.Core.Lint.dumpIfSet,
) where
#include "HsVersions.h"
import GHC.Prelude
import GHC.Core
import GHC.Core.FVs
import GHC.Core.Utils
import GHC.Core.Stats ( coreBindsStats )
import GHC.Core.Opt.Monad
import GHC.Data.Bag
import GHC.Types.Literal
import GHC.Core.DataCon
import GHC.Builtin.Types.Prim
import GHC.Builtin.Types ( multiplicityTy )
import GHC.Tc.Utils.TcType ( isFloatingTy, isTyFamFree )
import GHC.Types.Var as Var
import GHC.Types.Var.Env
import GHC.Types.Var.Set
import GHC.Types.Unique.Set( nonDetEltsUniqSet )
import GHC.Types.Name
import GHC.Types.Name.Env
import GHC.Types.Id
import GHC.Types.Id.Info
import GHC.Core.Ppr
import GHC.Utils.Error
import GHC.Core.Coercion
import GHC.Types.SrcLoc
import GHC.Core.Type as Type
import GHC.Core.Multiplicity
import GHC.Core.UsageEnv
import GHC.Types.RepType
import GHC.Core.TyCo.Rep
import GHC.Core.TyCo.Subst
import GHC.Core.TyCo.FVs
import GHC.Core.TyCo.Ppr ( pprTyVar, pprTyVars )
import GHC.Core.TyCon as TyCon
import GHC.Core.Coercion.Axiom
import GHC.Core.Unify
import GHC.Types.Basic
import GHC.Utils.Error as Err
import GHC.Data.List.SetOps
import GHC.Builtin.Names
import GHC.Utils.Outputable as Outputable
import GHC.Data.FastString
import GHC.Utils.Misc
import GHC.Core.InstEnv ( instanceDFunId )
import GHC.Core.Coercion.Opt ( checkAxInstCo )
import GHC.Core.Opt.Arity ( typeArity )
import GHC.Types.Demand ( splitStrictSig, isDeadEndDiv )
import GHC.Driver.Types hiding (Usage)
import GHC.Driver.Session
import Control.Monad
import GHC.Utils.Monad
import Data.Foldable ( toList )
import Data.List.NonEmpty ( NonEmpty(..), groupWith )
import Data.List ( partition )
import Data.Maybe
import GHC.Data.Pair
import qualified GHC.LanguageExtensions as LangExt
endPass :: CoreToDo -> CoreProgram -> [CoreRule] -> CoreM ()
endPass pass binds rules
= do { hsc_env <- getHscEnv
; print_unqual <- getPrintUnqualified
; liftIO $ endPassIO hsc_env print_unqual pass binds rules }
endPassIO :: HscEnv -> PrintUnqualified
-> CoreToDo -> CoreProgram -> [CoreRule] -> IO ()
endPassIO hsc_env print_unqual pass binds rules
= do { dumpPassResult dflags print_unqual mb_flag
(ppr pass) (pprPassDetails pass) binds rules
; lintPassResult hsc_env pass binds }
where
dflags = hsc_dflags hsc_env
mb_flag = case coreDumpFlag pass of
Just flag | dopt flag dflags -> Just flag
| dopt Opt_D_verbose_core2core dflags -> Just flag
_ -> Nothing
dumpIfSet :: DynFlags -> Bool -> CoreToDo -> SDoc -> SDoc -> IO ()
dumpIfSet dflags dump_me pass extra_info doc
= Err.dumpIfSet dflags dump_me (showSDoc dflags (ppr pass <+> extra_info)) doc
dumpPassResult :: DynFlags
-> PrintUnqualified
-> Maybe DumpFlag
-> SDoc
-> SDoc
-> CoreProgram -> [CoreRule]
-> IO ()
dumpPassResult dflags unqual mb_flag hdr extra_info binds rules
= do { forM_ mb_flag $ \flag -> do
let sty = mkDumpStyle unqual
dumpAction dflags sty (dumpOptionsFromFlag flag)
(showSDoc dflags hdr) FormatCore dump_doc
; Err.debugTraceMsg dflags 2 size_doc
}
where
size_doc = sep [text "Result size of" <+> hdr, nest 2 (equals <+> ppr (coreBindsStats binds))]
dump_doc = vcat [ nest 2 extra_info
, size_doc
, blankLine
, pprCoreBindingsWithSize binds
, ppUnless (null rules) pp_rules ]
pp_rules = vcat [ blankLine
, text "------ Local rules for imported ids --------"
, pprRules rules ]
coreDumpFlag :: CoreToDo -> Maybe DumpFlag
coreDumpFlag (CoreDoSimplify {}) = Just Opt_D_verbose_core2core
coreDumpFlag (CoreDoPluginPass {}) = Just Opt_D_verbose_core2core
coreDumpFlag CoreDoFloatInwards = Just Opt_D_verbose_core2core
coreDumpFlag (CoreDoFloatOutwards {}) = Just Opt_D_verbose_core2core
coreDumpFlag CoreLiberateCase = Just Opt_D_verbose_core2core
coreDumpFlag CoreDoStaticArgs = Just Opt_D_verbose_core2core
coreDumpFlag CoreDoCallArity = Just Opt_D_dump_call_arity
coreDumpFlag CoreDoExitify = Just Opt_D_dump_exitify
coreDumpFlag CoreDoDemand = Just Opt_D_dump_stranal
coreDumpFlag CoreDoCpr = Just Opt_D_dump_cpranal
coreDumpFlag CoreDoWorkerWrapper = Just Opt_D_dump_worker_wrapper
coreDumpFlag CoreDoSpecialising = Just Opt_D_dump_spec
coreDumpFlag CoreDoSpecConstr = Just Opt_D_dump_spec
coreDumpFlag CoreCSE = Just Opt_D_dump_cse
coreDumpFlag CoreDesugar = Just Opt_D_dump_ds_preopt
coreDumpFlag CoreDesugarOpt = Just Opt_D_dump_ds
coreDumpFlag CoreTidy = Just Opt_D_dump_simpl
coreDumpFlag CorePrep = Just Opt_D_dump_prep
coreDumpFlag CoreOccurAnal = Just Opt_D_dump_occur_anal
coreDumpFlag CoreDoPrintCore = Nothing
coreDumpFlag (CoreDoRuleCheck {}) = Nothing
coreDumpFlag CoreDoNothing = Nothing
coreDumpFlag (CoreDoPasses {}) = Nothing
lintPassResult :: HscEnv -> CoreToDo -> CoreProgram -> IO ()
lintPassResult hsc_env pass binds
| not (gopt Opt_DoCoreLinting dflags)
= return ()
| otherwise
= do { let (warns, errs) = lintCoreBindings dflags pass (interactiveInScope hsc_env) binds
; Err.showPass dflags ("Core Linted result of " ++ showPpr dflags pass)
; displayLintResults dflags pass warns errs binds }
where
dflags = hsc_dflags hsc_env
displayLintResults :: DynFlags -> CoreToDo
-> Bag Err.MsgDoc -> Bag Err.MsgDoc -> CoreProgram
-> IO ()
displayLintResults dflags pass warns errs binds
| not (isEmptyBag errs)
= do { putLogMsg dflags NoReason Err.SevDump noSrcSpan
$ withPprStyle defaultDumpStyle
(vcat [ lint_banner "errors" (ppr pass), Err.pprMessageBag errs
, text "*** Offending Program ***"
, pprCoreBindings binds
, text "*** End of Offense ***" ])
; Err.ghcExit dflags 1 }
| not (isEmptyBag warns)
, not (hasNoDebugOutput dflags)
, showLintWarnings pass
= putLogMsg dflags NoReason Err.SevInfo noSrcSpan
$ withPprStyle defaultDumpStyle
(lint_banner "warnings" (ppr pass) $$ Err.pprMessageBag (mapBag ($$ blankLine) warns))
| otherwise = return ()
where
lint_banner :: String -> SDoc -> SDoc
lint_banner string pass = text "*** Core Lint" <+> text string
<+> text ": in result of" <+> pass
<+> text "***"
showLintWarnings :: CoreToDo -> Bool
showLintWarnings (CoreDoSimplify _ (SimplMode { sm_phase = InitialPhase })) = False
showLintWarnings _ = True
lintInteractiveExpr :: String -> HscEnv -> CoreExpr -> IO ()
lintInteractiveExpr what hsc_env expr
| not (gopt Opt_DoCoreLinting dflags)
= return ()
| Just err <- lintExpr dflags (interactiveInScope hsc_env) expr
= do { display_lint_err err
; Err.ghcExit dflags 1 }
| otherwise
= return ()
where
dflags = hsc_dflags hsc_env
display_lint_err err
= do { putLogMsg dflags NoReason Err.SevDump
noSrcSpan
$ withPprStyle defaultDumpStyle
(vcat [ lint_banner "errors" (text what)
, err
, text "*** Offending Program ***"
, pprCoreExpr expr
, text "*** End of Offense ***" ])
; Err.ghcExit dflags 1 }
interactiveInScope :: HscEnv -> [Var]
interactiveInScope hsc_env
= tyvars ++ ids
where
ictxt = hsc_IC hsc_env
(cls_insts, _fam_insts) = ic_instances ictxt
te1 = mkTypeEnvWithImplicits (ic_tythings ictxt)
te = extendTypeEnvWithIds te1 (map instanceDFunId cls_insts)
ids = typeEnvIds te
tyvars = tyCoVarsOfTypesList $ map idType ids
lintCoreBindings :: DynFlags -> CoreToDo -> [Var] -> CoreProgram -> (Bag MsgDoc, Bag MsgDoc)
lintCoreBindings dflags pass local_in_scope binds
= initL dflags flags local_in_scope $
addLoc TopLevelBindings $
do { checkL (null dups) (dupVars dups)
; checkL (null ext_dups) (dupExtVars ext_dups)
; lintRecBindings TopLevel all_pairs $ \_ ->
return () }
where
all_pairs = flattenBinds binds
binders = map fst all_pairs
flags = (defaultLintFlags dflags)
{ lf_check_global_ids = check_globals
, lf_check_inline_loop_breakers = check_lbs
, lf_check_static_ptrs = check_static_ptrs }
check_globals = case pass of
CoreTidy -> False
CorePrep -> False
_ -> True
check_lbs = case pass of
CoreDesugar -> False
CoreDesugarOpt -> False
_ -> True
check_static_ptrs | not (xopt LangExt.StaticPointers dflags) = AllowAnywhere
| otherwise = case pass of
CoreDoFloatOutwards _ -> AllowAtTopLevel
CoreTidy -> RejectEverywhere
CorePrep -> AllowAtTopLevel
_ -> AllowAnywhere
(_, dups) = removeDups compare binders
ext_dups = snd (removeDups ord_ext (map Var.varName binders))
ord_ext n1 n2 | Just m1 <- nameModule_maybe n1
, Just m2 <- nameModule_maybe n2
= compare (m1, nameOccName n1) (m2, nameOccName n2)
| otherwise = LT
lintUnfolding :: Bool
-> DynFlags
-> SrcLoc
-> VarSet
-> CoreExpr
-> Maybe MsgDoc
lintUnfolding is_compulsory dflags locn var_set expr
| isEmptyBag errs = Nothing
| otherwise = Just (pprMessageBag errs)
where
vars = nonDetEltsUniqSet var_set
(_warns, errs) = initL dflags (defaultLintFlags dflags) vars $
if is_compulsory
then noLPChecks linter
else linter
linter = addLoc (ImportedUnfolding locn) $
lintCoreExpr expr
lintExpr :: DynFlags
-> [Var]
-> CoreExpr
-> Maybe MsgDoc
lintExpr dflags vars expr
| isEmptyBag errs = Nothing
| otherwise = Just (pprMessageBag errs)
where
(_warns, errs) = initL dflags (defaultLintFlags dflags) vars linter
linter = addLoc TopLevelBindings $
lintCoreExpr expr
lintRecBindings :: TopLevelFlag -> [(Id, CoreExpr)]
-> ([LintedId] -> LintM a) -> LintM (a, [UsageEnv])
lintRecBindings top_lvl pairs thing_inside
= lintIdBndrs top_lvl bndrs $ \ bndrs' ->
do { ues <- zipWithM lint_pair bndrs' rhss
; a <- thing_inside bndrs'
; return (a, ues) }
where
(bndrs, rhss) = unzip pairs
lint_pair bndr' rhs
= addLoc (RhsOf bndr') $
do { (rhs_ty, ue) <- lintRhs bndr' rhs
; lintLetBind top_lvl Recursive bndr' rhs rhs_ty
; return ue }
lintLetBody :: [LintedId] -> CoreExpr -> LintM (LintedType, UsageEnv)
lintLetBody bndrs body
= do { (body_ty, body_ue) <- addLoc (BodyOfLetRec bndrs) (lintCoreExpr body)
; mapM_ (lintJoinBndrType body_ty) bndrs
; return (body_ty, body_ue) }
lintLetBind :: TopLevelFlag -> RecFlag -> LintedId
-> CoreExpr -> LintedType -> LintM ()
lintLetBind top_lvl rec_flag binder rhs rhs_ty
= do { let binder_ty = idType binder
; ensureEqTys binder_ty rhs_ty (mkRhsMsg binder (text "RHS") rhs_ty)
; checkL (not (isCoVar binder) || isCoArg rhs)
(mkLetErr binder rhs)
; checkL ( isJoinId binder
|| not (isUnliftedType binder_ty)
|| (isNonRec rec_flag && exprOkForSpeculation rhs)
|| exprIsTickedString rhs)
(badBndrTyMsg binder (text "unlifted"))
; checkL (not (isStrictId binder)
|| (isNonRec rec_flag && not (isTopLevel top_lvl))
|| exprIsTickedString rhs)
(mkStrictMsg binder)
; checkL (not (isTopLevel top_lvl && binder_ty `eqType` addrPrimTy)
|| exprIsTickedString rhs)
(mkTopNonLitStrMsg binder)
; flags <- getLintFlags
; case isJoinId_maybe binder of
Nothing -> return ()
Just arity -> checkL (isValidJoinPointType arity binder_ty)
(mkInvalidJoinPointMsg binder binder_ty)
; when (lf_check_inline_loop_breakers flags
&& isStableUnfolding (realIdUnfolding binder)
&& isStrongLoopBreaker (idOccInfo binder)
&& isInlinePragma (idInlinePragma binder))
(addWarnL (text "INLINE binder is (non-rule) loop breaker:" <+> ppr binder))
; checkL (typeArity (idType binder) `lengthAtLeast` idArity binder)
(text "idArity" <+> ppr (idArity binder) <+>
text "exceeds typeArity" <+>
ppr (length (typeArity (idType binder))) <> colon <+>
ppr binder)
; case splitStrictSig (idStrictness binder) of
(demands, result_info) | isDeadEndDiv result_info ->
checkL (demands `lengthAtLeast` idArity binder)
(text "idArity" <+> ppr (idArity binder) <+>
text "exceeds arity imposed by the strictness signature" <+>
ppr (idStrictness binder) <> colon <+>
ppr binder)
_ -> return ()
; addLoc (RuleOf binder) $ mapM_ (lintCoreRule binder binder_ty) (idCoreRules binder)
; addLoc (UnfoldingOf binder) $
lintIdUnfolding binder binder_ty (idUnfolding binder)
; return () }
lintRhs :: Id -> CoreExpr -> LintM (LintedType, UsageEnv)
lintRhs bndr rhs
| Just arity <- isJoinId_maybe bndr
= lintJoinLams arity (Just bndr) rhs
| AlwaysTailCalled arity <- tailCallInfo (idOccInfo bndr)
= lintJoinLams arity Nothing rhs
lintRhs _bndr rhs = fmap lf_check_static_ptrs getLintFlags >>= go
where
go :: StaticPtrCheck -> LintM (OutType, UsageEnv)
go AllowAtTopLevel
| (binders0, rhs') <- collectTyBinders rhs
, Just (fun, t, info, e) <- collectMakeStaticArgs rhs'
= markAllJoinsBad $
foldr
lintLambda
(do fun_ty_ue <- lintCoreExpr fun
lintCoreArgs fun_ty_ue [Type t, info, e]
)
binders0
go _ = markAllJoinsBad $ lintCoreExpr rhs
lintJoinLams :: JoinArity -> Maybe Id -> CoreExpr -> LintM (LintedType, UsageEnv)
lintJoinLams join_arity enforce rhs
= go join_arity rhs
where
go 0 expr = lintCoreExpr expr
go n (Lam var body) = lintLambda var $ go (n1) body
go n expr | Just bndr <- enforce
= failWithL $ mkBadJoinArityMsg bndr join_arity n rhs
| otherwise
= markAllJoinsBad $ lintCoreExpr expr
lintIdUnfolding :: Id -> Type -> Unfolding -> LintM ()
lintIdUnfolding bndr bndr_ty uf
| isStableUnfolding uf
, Just rhs <- maybeUnfoldingTemplate uf
= do { ty <- fst <$> (if isCompulsoryUnfolding uf
then noLPChecks $ lintRhs bndr rhs
else lintRhs bndr rhs)
; ensureEqTys bndr_ty ty (mkRhsMsg bndr (text "unfolding") ty) }
lintIdUnfolding _ _ _
= return ()
type LintedType = Type
type LintedKind = Kind
type LintedCoercion = Coercion
type LintedTyCoVar = TyCoVar
type LintedId = Id
lintCastExpr :: CoreExpr -> LintedType -> Coercion -> LintM LintedType
lintCastExpr expr expr_ty co
= do { co' <- lintCoercion co
; let (Pair from_ty to_ty, role) = coercionKindRole co'
; checkValueType to_ty $
text "target of cast" <+> quotes (ppr co')
; lintRole co' Representational role
; ensureEqTys from_ty expr_ty (mkCastErr expr co' from_ty expr_ty)
; return to_ty }
lintCoreExpr :: CoreExpr -> LintM (LintedType, UsageEnv)
lintCoreExpr (Var var)
= lintIdOcc var 0
lintCoreExpr (Lit lit)
= return (literalType lit, zeroUE)
lintCoreExpr (Cast expr co)
= do (expr_ty, ue) <- markAllJoinsBad $ lintCoreExpr expr
to_ty <- lintCastExpr expr expr_ty co
return (to_ty, ue)
lintCoreExpr (Tick tickish expr)
= do case tickish of
Breakpoint _ ids -> forM_ ids $ \id -> do
checkDeadIdOcc id
lookupIdInScope id
_ -> return ()
markAllJoinsBadIf block_joins $ lintCoreExpr expr
where
block_joins = not (tickish `tickishScopesLike` SoftScope)
lintCoreExpr (Let (NonRec tv (Type ty)) body)
| isTyVar tv
=
do { ty' <- lintType ty
; lintTyBndr tv $ \ tv' ->
do { addLoc (RhsOf tv) $ lintTyKind tv' ty'
; extendTvSubstL tv ty' $
addLoc (BodyOfLetRec [tv]) $
lintCoreExpr body } }
lintCoreExpr (Let (NonRec bndr rhs) body)
| isId bndr
= do {
(rhs_ty, let_ue) <- lintRhs bndr rhs
; lintBinder LetBind bndr $ \bndr' ->
do { lintLetBind NotTopLevel NonRecursive bndr' rhs rhs_ty
; addAliasUE bndr let_ue (lintLetBody [bndr'] body) } }
| otherwise
= failWithL (mkLetErr bndr rhs)
lintCoreExpr e@(Let (Rec pairs) body)
= do {
checkL (not (null pairs)) (emptyRec e)
; let (_, dups) = removeDups compare bndrs
; checkL (null dups) (dupVars dups)
; checkL (all isJoinId bndrs || all (not . isJoinId) bndrs) $
mkInconsistentRecMsg bndrs
; ((body_type, body_ue), ues) <-
lintRecBindings NotTopLevel pairs $ \ bndrs' ->
lintLetBody bndrs' body
; return (body_type, body_ue `addUE` scaleUE Many (foldr1 addUE ues)) }
where
bndrs = map fst pairs
lintCoreExpr e@(App _ _)
| Var fun <- fun
, fun `hasKey` runRWKey
, arg_ty1 : arg_ty2 : arg3 : rest <- args
= do { fun_pair1 <- lintCoreArg (idType fun, zeroUE) arg_ty1
; (fun_ty2, ue2) <- lintCoreArg fun_pair1 arg_ty2
; let lintRunRWCont :: CoreArg -> LintM (LintedType, UsageEnv)
lintRunRWCont expr@(Lam _ _) = do
lintJoinLams 1 (Just fun) expr
lintRunRWCont other = markAllJoinsBad $ lintCoreExpr other
; (arg3_ty, ue3) <- lintRunRWCont arg3
; app_ty <- lintValApp arg3 fun_ty2 arg3_ty ue2 ue3
; lintCoreArgs app_ty rest }
| otherwise
= do { pair <- lintCoreFun fun (length args)
; lintCoreArgs pair args }
where
(fun, args) = collectArgs e
lintCoreExpr (Lam var expr)
= markAllJoinsBad $
lintLambda var $ lintCoreExpr expr
lintCoreExpr (Case scrut var alt_ty alts)
= lintCaseExpr scrut var alt_ty alts
lintCoreExpr (Type ty)
= failWithL (text "Type found as expression" <+> ppr ty)
lintCoreExpr (Coercion co)
= do { co' <- addLoc (InCo co) $
lintCoercion co
; return (coercionType co', zeroUE) }
lintIdOcc :: Var -> Int
-> LintM (LintedType, UsageEnv)
lintIdOcc var nargs
= addLoc (OccOf var) $
do { checkL (isNonCoVarId var)
(text "Non term variable" <+> ppr var)
; (bndr, linted_bndr_ty) <- lookupIdInScope var
; let occ_ty = idType var
bndr_ty = idType bndr
; ensureEqTys occ_ty bndr_ty $
mkBndrOccTypeMismatchMsg bndr var bndr_ty occ_ty
; lf <- getLintFlags
; when (nargs /= 0 && lf_check_static_ptrs lf /= AllowAnywhere) $
checkL (idName var /= makeStaticName) $
text "Found makeStatic nested in an expression"
; checkDeadIdOcc var
; checkJoinOcc var nargs
; usage <- varCallSiteUsage var
; return (linted_bndr_ty, usage) }
lintCoreFun :: CoreExpr
-> Int
-> LintM (LintedType, UsageEnv)
lintCoreFun (Var var) nargs
= lintIdOcc var nargs
lintCoreFun (Lam var body) nargs
| nargs /= 0
= lintLambda var $ lintCoreFun body (nargs 1)
lintCoreFun expr nargs
= markAllJoinsBadIf (nargs /= 0) $
lintCoreExpr expr
lintLambda :: Var -> LintM (Type, UsageEnv) -> LintM (Type, UsageEnv)
lintLambda var lintBody =
addLoc (LambdaBodyOf var) $
lintBinder LambdaBind var $ \ var' ->
do { (body_ty, ue) <- lintBody
; ue' <- checkLinearity ue var'
; return (mkLamType var' body_ty, ue') }
checkDeadIdOcc :: Id -> LintM ()
checkDeadIdOcc id
| isDeadOcc (idOccInfo id)
= do { in_case <- inCasePat
; checkL in_case
(text "Occurrence of a dead Id" <+> ppr id) }
| otherwise
= return ()
lintJoinBndrType :: LintedType
-> LintedId
-> LintM ()
lintJoinBndrType body_ty bndr
| Just arity <- isJoinId_maybe bndr
, let bndr_ty = idType bndr
, (bndrs, res) <- splitPiTys bndr_ty
= checkL (length bndrs >= arity
&& body_ty `eqType` mkPiTys (drop arity bndrs) res) $
hang (text "Join point returns different type than body")
2 (vcat [ text "Join bndr:" <+> ppr bndr <+> dcolon <+> ppr (idType bndr)
, text "Join arity:" <+> ppr arity
, text "Body type:" <+> ppr body_ty ])
| otherwise
= return ()
checkJoinOcc :: Id -> JoinArity -> LintM ()
checkJoinOcc var n_args
| Just join_arity_occ <- isJoinId_maybe var
= do { mb_join_arity_bndr <- lookupJoinId var
; case mb_join_arity_bndr of {
Nothing ->
do { join_set <- getValidJoins
; addErrL (text "join set " <+> ppr join_set $$
invalidJoinOcc var) } ;
Just join_arity_bndr ->
do { checkL (join_arity_bndr == join_arity_occ) $
mkJoinBndrOccMismatchMsg var join_arity_bndr join_arity_occ
; checkL (n_args == join_arity_occ) $
mkBadJumpMsg var join_arity_occ n_args } } }
| otherwise
= return ()
checkLinearity :: UsageEnv -> Var -> LintM UsageEnv
checkLinearity body_ue lam_var =
case varMultMaybe lam_var of
Just mult -> do ensureSubUsage lhs mult (err_msg mult)
return $ deleteUE body_ue lam_var
Nothing -> return body_ue
where
lhs = lookupUE body_ue lam_var
err_msg mult = text "Linearity failure in lambda:" <+> ppr lam_var
$$ ppr lhs <+> text "⊈" <+> ppr mult
lintCoreArgs :: (LintedType, UsageEnv) -> [CoreArg] -> LintM (LintedType, UsageEnv)
lintCoreArgs (fun_ty, fun_ue) args = foldM lintCoreArg (fun_ty, fun_ue) args
lintCoreArg :: (LintedType, UsageEnv) -> CoreArg -> LintM (LintedType, UsageEnv)
lintCoreArg (fun_ty, ue) (Type arg_ty)
= do { checkL (not (isCoercionTy arg_ty))
(text "Unnecessary coercion-to-type injection:"
<+> ppr arg_ty)
; arg_ty' <- lintType arg_ty
; res <- lintTyApp fun_ty arg_ty'
; return (res, ue) }
lintCoreArg (fun_ty, fun_ue) arg
= do { (arg_ty, arg_ue) <- markAllJoinsBad $ lintCoreExpr arg
; flags <- getLintFlags
; lintL (not (lf_check_levity_poly flags) || not (isTypeLevPoly arg_ty))
(text "Levity-polymorphic argument:" <+>
(ppr arg <+> dcolon <+> parens (ppr arg_ty <+> dcolon <+> ppr (typeKind arg_ty))))
; checkL (not (isUnliftedType arg_ty) || exprOkForSpeculation arg)
(mkLetAppMsg arg)
; lintValApp arg fun_ty arg_ty fun_ue arg_ue }
lintAltBinders :: UsageEnv
-> Var
-> LintedType
-> LintedType
-> [(Mult, OutVar)]
-> LintM UsageEnv
lintAltBinders rhs_ue _case_bndr scrut_ty con_ty []
= do { ensureEqTys con_ty scrut_ty (mkBadPatMsg con_ty scrut_ty)
; return rhs_ue }
lintAltBinders rhs_ue case_bndr scrut_ty con_ty ((var_w, bndr):bndrs)
| isTyVar bndr
= do { con_ty' <- lintTyApp con_ty (mkTyVarTy bndr)
; lintAltBinders rhs_ue case_bndr scrut_ty con_ty' bndrs }
| otherwise
= do { (con_ty', _) <- lintValApp (Var bndr) con_ty (idType bndr) zeroUE zeroUE
; rhs_ue' <- checkCaseLinearity rhs_ue case_bndr var_w bndr
; lintAltBinders rhs_ue' case_bndr scrut_ty con_ty' bndrs }
checkCaseLinearity :: UsageEnv -> Var -> Mult -> Var -> LintM UsageEnv
checkCaseLinearity ue case_bndr var_w bndr = do
ensureSubUsage lhs rhs err_msg
lintLinearBinder (ppr bndr) (case_bndr_w `mkMultMul` var_w) (varMult bndr)
return $ deleteUE ue bndr
where
lhs = bndr_usage `addUsage` (var_w `scaleUsage` case_bndr_usage)
rhs = case_bndr_w `mkMultMul` var_w
err_msg = (text "Linearity failure in variable:" <+> ppr bndr
$$ ppr lhs <+> text "⊈" <+> ppr rhs
$$ text "Computed by:"
<+> text "LHS:" <+> lhs_formula
<+> text "RHS:" <+> rhs_formula)
lhs_formula = ppr bndr_usage <+> text "+"
<+> parens (ppr case_bndr_usage <+> text "*" <+> ppr var_w)
rhs_formula = ppr case_bndr_w <+> text "*" <+> ppr var_w
case_bndr_w = varMult case_bndr
case_bndr_usage = lookupUE ue case_bndr
bndr_usage = lookupUE ue bndr
lintTyApp :: LintedType -> LintedType -> LintM LintedType
lintTyApp fun_ty arg_ty
| Just (tv,body_ty) <- splitForAllTy_maybe fun_ty
= do { lintTyKind tv arg_ty
; in_scope <- getInScope
; return (substTyWithInScope in_scope [tv] [arg_ty] body_ty) }
| otherwise
= failWithL (mkTyAppMsg fun_ty arg_ty)
lintValApp :: CoreExpr -> LintedType -> LintedType -> UsageEnv -> UsageEnv -> LintM (LintedType, UsageEnv)
lintValApp arg fun_ty arg_ty fun_ue arg_ue
| Just (w, arg_ty', res_ty') <- splitFunTy_maybe fun_ty
= do { ensureEqTys arg_ty' arg_ty err1
; let app_ue = addUE fun_ue (scaleUE w arg_ue)
; return (res_ty', app_ue) }
| otherwise
= failWithL err2
where
err1 = mkAppMsg fun_ty arg_ty arg
err2 = mkNonFunAppMsg fun_ty arg_ty arg
lintTyKind :: OutTyVar -> LintedType -> LintM ()
lintTyKind tyvar arg_ty
= unless (arg_kind `eqType` tyvar_kind) $
addErrL (mkKindErrMsg tyvar arg_ty $$ (text "Linted Arg kind:" <+> ppr arg_kind))
where
tyvar_kind = tyVarKind tyvar
arg_kind = typeKind arg_ty
lintCaseExpr :: CoreExpr -> Id -> Type -> [CoreAlt] -> LintM (LintedType, UsageEnv)
lintCaseExpr scrut var alt_ty alts =
do { let e = Case scrut var alt_ty alts
; (scrut_ty, scrut_ue) <- markAllJoinsBad $ lintCoreExpr scrut
; let scrut_mult = varMult var
; alt_ty <- addLoc (CaseTy scrut) $
lintValueType alt_ty
; var_ty <- addLoc (IdTy var) $
lintValueType (idType var)
; let isLitPat (LitAlt _, _ , _) = True
isLitPat _ = False
; checkL (not $ isFloatingTy scrut_ty && any isLitPat alts)
(ptext (sLit $ "Lint warning: Scrutinising floating-point " ++
"expression with literal pattern in case " ++
"analysis (see #9238).")
$$ text "scrut" <+> ppr scrut)
; case tyConAppTyCon_maybe (idType var) of
Just tycon
| debugIsOn
, isAlgTyCon tycon
, not (isAbstractTyCon tycon)
, null (tyConDataCons tycon)
, not (exprIsDeadEnd scrut)
-> pprTrace "Lint warning: case binder's type has no constructors" (ppr var <+> ppr (idType var))
$ return ()
_otherwise -> return ()
; subst <- getTCvSubst
; ensureEqTys var_ty scrut_ty (mkScrutMsg var var_ty scrut_ty subst)
; lintBinder CaseBind var $ \_ ->
do {
; alt_ues <- mapM (lintCoreAlt var scrut_ty scrut_mult alt_ty) alts
; let case_ue = (scaleUE scrut_mult scrut_ue) `addUE` supUEs alt_ues
; checkCaseAlts e scrut_ty alts
; return (alt_ty, case_ue) } }
checkCaseAlts :: CoreExpr -> LintedType -> [CoreAlt] -> LintM ()
checkCaseAlts e ty alts =
do { checkL (all non_deflt con_alts) (mkNonDefltMsg e)
; checkL (increasing_tag con_alts) (mkNonIncreasingAltsMsg e)
; checkL (isJust maybe_deflt || not is_infinite_ty || null alts)
(nonExhaustiveAltsMsg e) }
where
(con_alts, maybe_deflt) = findDefault alts
increasing_tag (alt1 : rest@( alt2 : _)) = alt1 `ltAlt` alt2 && increasing_tag rest
increasing_tag _ = True
non_deflt (DEFAULT, _, _) = False
non_deflt _ = True
is_infinite_ty = case tyConAppTyCon_maybe ty of
Nothing -> False
Just tycon -> isPrimTyCon tycon
lintAltExpr :: CoreExpr -> LintedType -> LintM UsageEnv
lintAltExpr expr ann_ty
= do { (actual_ty, ue) <- lintCoreExpr expr
; ensureEqTys actual_ty ann_ty (mkCaseAltMsg expr actual_ty ann_ty)
; return ue }
lintCoreAlt :: Var
-> LintedType
-> Mult
-> LintedType
-> CoreAlt
-> LintM UsageEnv
lintCoreAlt _ _ _ alt_ty (DEFAULT, args, rhs) =
do { lintL (null args) (mkDefaultArgsMsg args)
; lintAltExpr rhs alt_ty }
lintCoreAlt _case_bndr scrut_ty _ alt_ty (LitAlt lit, args, rhs)
| litIsLifted lit
= failWithL integerScrutinisedMsg
| otherwise
= do { lintL (null args) (mkDefaultArgsMsg args)
; ensureEqTys lit_ty scrut_ty (mkBadPatMsg lit_ty scrut_ty)
; lintAltExpr rhs alt_ty }
where
lit_ty = literalType lit
lintCoreAlt case_bndr scrut_ty _scrut_mult alt_ty alt@(DataAlt con, args, rhs)
| isNewTyCon (dataConTyCon con)
= zeroUE <$ addErrL (mkNewTyDataConAltMsg scrut_ty alt)
| Just (tycon, tycon_arg_tys) <- splitTyConApp_maybe scrut_ty
= addLoc (CaseAlt alt) $ do
{
lintL (tycon == dataConTyCon con) (mkBadConMsg tycon con)
; let { con_payload_ty = piResultTys (dataConRepType con) tycon_arg_tys
; ex_tvs_n = length (dataConExTyCoVars con)
; multiplicities = replicate ex_tvs_n Many ++
map scaledMult (dataConRepArgTys con) }
; lintBinders CasePatBind args $ \ args' -> do
{
rhs_ue <- lintAltExpr rhs alt_ty
; rhs_ue' <- addLoc (CasePat alt) (lintAltBinders rhs_ue case_bndr scrut_ty con_payload_ty (zipEqual "lintCoreAlt" multiplicities args'))
; return $ deleteUE rhs_ue' case_bndr
}
}
| otherwise
= zeroUE <$ addErrL (mkBadAltMsg scrut_ty alt)
lintLinearBinder :: SDoc -> Mult -> Mult -> LintM ()
lintLinearBinder doc actual_usage described_usage
= ensureSubMult actual_usage described_usage err_msg
where
err_msg = (text "Multiplicity of variable does not agree with its context"
$$ doc
$$ ppr actual_usage
$$ text "Annotation:" <+> ppr described_usage)
lintBinders :: BindingSite -> [Var] -> ([Var] -> LintM a) -> LintM a
lintBinders _ [] linterF = linterF []
lintBinders site (var:vars) linterF = lintBinder site var $ \var' ->
lintBinders site vars $ \ vars' ->
linterF (var':vars')
lintBinder :: BindingSite -> Var -> (Var -> LintM a) -> LintM a
lintBinder site var linterF
| isTyCoVar var = lintTyCoBndr var linterF
| otherwise = lintIdBndr NotTopLevel site var linterF
lintTyBndr :: TyVar -> (LintedTyCoVar -> LintM a) -> LintM a
lintTyBndr = lintTyCoBndr
lintTyCoBndr :: TyCoVar -> (LintedTyCoVar -> LintM a) -> LintM a
lintTyCoBndr tcv thing_inside
= do { subst <- getTCvSubst
; kind' <- lintType (varType tcv)
; let tcv' = uniqAway (getTCvInScope subst) $
setVarType tcv kind'
subst' = extendTCvSubstWithClone subst tcv tcv'
; when (isCoVar tcv) $
lintL (isCoVarType kind')
(text "CoVar with non-coercion type:" <+> pprTyVar tcv)
; updateTCvSubst subst' (thing_inside tcv') }
lintIdBndrs :: forall a. TopLevelFlag -> [Id] -> ([LintedId] -> LintM a) -> LintM a
lintIdBndrs top_lvl ids thing_inside
= go ids thing_inside
where
go :: [Id] -> ([Id] -> LintM a) -> LintM a
go [] thing_inside = thing_inside []
go (id:ids) thing_inside = lintIdBndr top_lvl LetBind id $ \id' ->
go ids $ \ids' ->
thing_inside (id' : ids')
lintIdBndr :: TopLevelFlag -> BindingSite
-> InVar -> (OutVar -> LintM a) -> LintM a
lintIdBndr top_lvl bind_site id thing_inside
= ASSERT2( isId id, ppr id )
do { flags <- getLintFlags
; checkL (not (lf_check_global_ids flags) || isLocalId id)
(text "Non-local Id binder" <+> ppr id)
; checkL (not (isExportedId id) || is_top_lvl)
(mkNonTopExportedMsg id)
; checkL (not (isExternalName (Var.varName id)) || is_top_lvl)
(mkNonTopExternalNameMsg id)
; lintL (isJoinId id || not (lf_check_levity_poly flags)
|| not (isTypeLevPoly id_ty)) $
text "Levity-polymorphic binder:" <+> ppr id <+> dcolon <+>
parens (ppr id_ty <+> dcolon <+> ppr (typeKind id_ty))
; when (isJoinId id) $
checkL (not is_top_lvl && is_let_bind) $
mkBadJoinBindMsg id
; lintL (not (isCoVarType id_ty))
(text "Non-CoVar has coercion type" <+> ppr id <+> dcolon <+> ppr id_ty)
; linted_ty <- addLoc (IdTy id) (lintValueType id_ty)
; addInScopeId id linted_ty $
thing_inside (setIdType id linted_ty) }
where
id_ty = idType id
is_top_lvl = isTopLevel top_lvl
is_let_bind = case bind_site of
LetBind -> True
_ -> False
lintValueType :: Type -> LintM LintedType
lintValueType ty
= addLoc (InType ty) $
do { ty' <- lintType ty
; let sk = typeKind ty'
; lintL (classifiesTypeWithValues sk) $
hang (text "Ill-kinded type:" <+> ppr ty)
2 (text "has kind:" <+> ppr sk)
; return ty' }
checkTyCon :: TyCon -> LintM ()
checkTyCon tc
= checkL (not (isTcTyCon tc)) (text "Found TcTyCon:" <+> ppr tc)
lintType :: Type -> LintM LintedType
lintType (TyVarTy tv)
| not (isTyVar tv)
= failWithL (mkBadTyVarMsg tv)
| otherwise
= do { subst <- getTCvSubst
; case lookupTyVar subst tv of
Just linted_ty -> return linted_ty
Nothing | tv `isInScope` subst
-> return (TyVarTy tv)
| otherwise
-> failWithL $
hang (text "The type variable" <+> pprBndr LetBind tv)
2 (text "is out of scope")
}
lintType ty@(AppTy t1 t2)
| TyConApp {} <- t1
= failWithL $ text "TyConApp to the left of AppTy:" <+> ppr ty
| otherwise
= do { t1' <- lintType t1
; t2' <- lintType t2
; lint_ty_app ty (typeKind t1') [t2']
; return (AppTy t1' t2') }
lintType ty@(TyConApp tc tys)
| isTypeSynonymTyCon tc || isTypeFamilyTyCon tc
= do { report_unsat <- lf_report_unsat_syns <$> getLintFlags
; lintTySynFamApp report_unsat ty tc tys }
| isFunTyCon tc
, tys `lengthIs` 5
= failWithL (hang (text "Saturated application of (->)") 2 (ppr ty))
| otherwise
= do { checkTyCon tc
; tys' <- mapM lintType tys
; lint_ty_app ty (tyConKind tc) tys'
; return (TyConApp tc tys') }
lintType ty@(FunTy af tw t1 t2)
= do { t1' <- lintType t1
; t2' <- lintType t2
; tw' <- lintType tw
; lintArrow (text "type or kind" <+> quotes (ppr ty)) t1' t2' tw'
; return (FunTy af tw' t1' t2') }
lintType ty@(ForAllTy (Bndr tcv vis) body_ty)
| not (isTyCoVar tcv)
= failWithL (text "Non-Tyvar or Non-Covar bound in type:" <+> ppr ty)
| otherwise
= lintTyCoBndr tcv $ \tcv' ->
do { body_ty' <- lintType body_ty
; lintForAllBody tcv' body_ty'
; when (isCoVar tcv) $
lintL (tcv `elemVarSet` tyCoVarsOfType body_ty) $
text "Covar does not occur in the body:" <+> (ppr tcv $$ ppr body_ty)
; return (ForAllTy (Bndr tcv' vis) body_ty') }
lintType ty@(LitTy l)
= do { lintTyLit l; return ty }
lintType (CastTy ty co)
= do { ty' <- lintType ty
; co' <- lintStarCoercion co
; let tyk = typeKind ty'
cok = coercionLKind co'
; ensureEqTys tyk cok (mkCastTyErr ty co tyk cok)
; return (CastTy ty' co') }
lintType (CoercionTy co)
= do { co' <- lintCoercion co
; return (CoercionTy co') }
lintForAllBody :: LintedTyCoVar -> LintedType -> LintM ()
lintForAllBody tcv body_ty
= do { checkValueType body_ty (text "the body of forall:" <+> ppr body_ty)
; let body_kind = typeKind body_ty
; when (isTyVar tcv) $
case occCheckExpand [tcv] body_kind of
Just {} -> return ()
Nothing -> failWithL $
hang (text "Variable escape in forall:")
2 (vcat [ text "tyvar:" <+> ppr tcv
, text "type:" <+> ppr body_ty
, text "kind:" <+> ppr body_kind ])
}
lintTySynFamApp :: Bool -> InType -> TyCon -> [InType] -> LintM LintedType
lintTySynFamApp report_unsat ty tc tys
| report_unsat
, tys `lengthLessThan` tyConArity tc
= failWithL (hang (text "Un-saturated type application") 2 (ppr ty))
| Just (tenv, rhs, tys') <- expandSynTyCon_maybe tc tys
, let expanded_ty = mkAppTys (substTy (mkTvSubstPrs tenv) rhs) tys'
= do {
tys' <- setReportUnsat False (mapM lintType tys)
; when report_unsat $
do { _ <- lintType expanded_ty
; return () }
; lint_ty_app ty (tyConKind tc) tys'
; return (TyConApp tc tys') }
| otherwise
= do { tys' <- mapM lintType tys
; lint_ty_app ty (tyConKind tc) tys'
; return (TyConApp tc tys') }
checkValueType :: LintedType -> SDoc -> LintM ()
checkValueType ty doc
= lintL (classifiesTypeWithValues kind)
(text "Non-*-like kind when *-like expected:" <+> ppr kind $$
text "when checking" <+> doc)
where
kind = typeKind ty
lintArrow :: SDoc -> LintedType -> LintedType -> LintedType -> LintM ()
lintArrow what t1 t2 tw
= do { unless (classifiesTypeWithValues k1) (addErrL (msg (text "argument") k1))
; unless (classifiesTypeWithValues k2) (addErrL (msg (text "result") k2))
; unless (isMultiplicityTy kw) (addErrL (msg (text "multiplicity") kw)) }
where
k1 = typeKind t1
k2 = typeKind t2
kw = typeKind tw
msg ar k
= vcat [ hang (text "Ill-kinded" <+> ar)
2 (text "in" <+> what)
, what <+> text "kind:" <+> ppr k ]
lint_ty_app :: Type -> LintedKind -> [LintedType] -> LintM ()
lint_ty_app ty k tys
= lint_app (text "type" <+> quotes (ppr ty)) k tys
lint_co_app :: Coercion -> LintedKind -> [LintedType] -> LintM ()
lint_co_app ty k tys
= lint_app (text "coercion" <+> quotes (ppr ty)) k tys
lintTyLit :: TyLit -> LintM ()
lintTyLit (NumTyLit n)
| n >= 0 = return ()
| otherwise = failWithL msg
where msg = text "Negative type literal:" <+> integer n
lintTyLit (StrTyLit _) = return ()
lint_app :: SDoc -> LintedKind -> [LintedType] -> LintM ()
lint_app doc kfn arg_tys
= do { in_scope <- getInScope
; _ <- foldlM (go_app in_scope) kfn arg_tys
; return () }
where
fail_msg extra = vcat [ hang (text "Kind application error in") 2 doc
, nest 2 (text "Function kind =" <+> ppr kfn)
, nest 2 (text "Arg types =" <+> ppr arg_tys)
, extra ]
go_app in_scope kfn ta
| Just kfn' <- coreView kfn
= go_app in_scope kfn' ta
go_app _ fun_kind@(FunTy _ _ kfa kfb) ta
= do { let ka = typeKind ta
; unless (ka `eqType` kfa) $
addErrL (fail_msg (text "Fun:" <+> (ppr fun_kind $$ ppr ta <+> dcolon <+> ppr ka)))
; return kfb }
go_app in_scope (ForAllTy (Bndr kv _vis) kfn) ta
= do { let kv_kind = varType kv
ka = typeKind ta
; unless (ka `eqType` kv_kind) $
addErrL (fail_msg (text "Forall:" <+> (ppr kv $$ ppr kv_kind $$
ppr ta <+> dcolon <+> ppr ka)))
; return $ substTy (extendTCvSubst (mkEmptyTCvSubst in_scope) kv ta) kfn }
go_app _ kfn ta
= failWithL (fail_msg (text "Not a fun:" <+> (ppr kfn $$ ppr ta)))
lintCoreRule :: OutVar -> LintedType -> CoreRule -> LintM ()
lintCoreRule _ _ (BuiltinRule {})
= return ()
lintCoreRule fun fun_ty rule@(Rule { ru_name = name, ru_bndrs = bndrs
, ru_args = args, ru_rhs = rhs })
= lintBinders LambdaBind bndrs $ \ _ ->
do { (lhs_ty, _) <- lintCoreArgs (fun_ty, zeroUE) args
; (rhs_ty, _) <- case isJoinId_maybe fun of
Just join_arity
-> do { checkL (args `lengthIs` join_arity) $
mkBadJoinPointRuleMsg fun join_arity rule
; lintCoreExpr rhs }
_ -> markAllJoinsBad $ lintCoreExpr rhs
; ensureEqTys lhs_ty rhs_ty $
(rule_doc <+> vcat [ text "lhs type:" <+> ppr lhs_ty
, text "rhs type:" <+> ppr rhs_ty
, text "fun_ty:" <+> ppr fun_ty ])
; let bad_bndrs = filter is_bad_bndr bndrs
; checkL (null bad_bndrs)
(rule_doc <+> text "unbound" <+> ppr bad_bndrs)
}
where
rule_doc = text "Rule" <+> doubleQuotes (ftext name) <> colon
lhs_fvs = exprsFreeVars args
rhs_fvs = exprFreeVars rhs
is_bad_bndr :: Var -> Bool
is_bad_bndr bndr = not (bndr `elemVarSet` lhs_fvs)
&& bndr `elemVarSet` rhs_fvs
&& isNothing (isReflCoVar_maybe bndr)
lintStarCoercion :: InCoercion -> LintM LintedCoercion
lintStarCoercion g
= do { g' <- lintCoercion g
; let Pair t1 t2 = coercionKind g'
; checkValueType t1 (text "the kind of the left type in" <+> ppr g)
; checkValueType t2 (text "the kind of the right type in" <+> ppr g)
; lintRole g Nominal (coercionRole g)
; return g' }
lintCoercion :: InCoercion -> LintM LintedCoercion
lintCoercion (CoVarCo cv)
| not (isCoVar cv)
= failWithL (hang (text "Bad CoVarCo:" <+> ppr cv)
2 (text "With offending type:" <+> ppr (varType cv)))
| otherwise
= do { subst <- getTCvSubst
; case lookupCoVar subst cv of
Just linted_co -> return linted_co ;
Nothing
| cv `isInScope` subst
-> return (CoVarCo cv)
| otherwise
->
failWithL $
hang (text "The coercion variable" <+> pprBndr LetBind cv)
2 (text "is out of scope")
}
lintCoercion (Refl ty)
= do { ty' <- lintType ty
; return (Refl ty') }
lintCoercion (GRefl r ty MRefl)
= do { ty' <- lintType ty
; return (GRefl r ty' MRefl) }
lintCoercion (GRefl r ty (MCo co))
= do { ty' <- lintType ty
; co' <- lintCoercion co
; let tk = typeKind ty'
tl = coercionLKind co'
; ensureEqTys tk tl $
hang (text "GRefl coercion kind mis-match:" <+> ppr co)
2 (vcat [ppr ty', ppr tk, ppr tl])
; lintRole co' Nominal (coercionRole co')
; return (GRefl r ty' (MCo co')) }
lintCoercion co@(TyConAppCo r tc cos)
| tc `hasKey` funTyConKey
, [_w, _rep1,_rep2,_co1,_co2] <- cos
= failWithL (text "Saturated TyConAppCo (->):" <+> ppr co)
| Just {} <- synTyConDefn_maybe tc
= failWithL (text "Synonym in TyConAppCo:" <+> ppr co)
| otherwise
= do { checkTyCon tc
; cos' <- mapM lintCoercion cos
; let (co_kinds, co_roles) = unzip (map coercionKindRole cos')
; lint_co_app co (tyConKind tc) (map pFst co_kinds)
; lint_co_app co (tyConKind tc) (map pSnd co_kinds)
; zipWithM_ (lintRole co) (tyConRolesX r tc) co_roles
; return (TyConAppCo r tc cos') }
lintCoercion co@(AppCo co1 co2)
| TyConAppCo {} <- co1
= failWithL (text "TyConAppCo to the left of AppCo:" <+> ppr co)
| Just (TyConApp {}, _) <- isReflCo_maybe co1
= failWithL (text "Refl (TyConApp ...) to the left of AppCo:" <+> ppr co)
| otherwise
= do { co1' <- lintCoercion co1
; co2' <- lintCoercion co2
; let (Pair lk1 rk1, r1) = coercionKindRole co1'
(Pair lk2 rk2, r2) = coercionKindRole co2'
; lint_co_app co (typeKind lk1) [lk2]
; lint_co_app co (typeKind rk1) [rk2]
; if r1 == Phantom
then lintL (r2 == Phantom || r2 == Nominal)
(text "Second argument in AppCo cannot be R:" $$
ppr co)
else lintRole co Nominal r2
; return (AppCo co1' co2') }
lintCoercion co@(ForAllCo tcv kind_co body_co)
| not (isTyCoVar tcv)
= failWithL (text "Non tyco binder in ForAllCo:" <+> ppr co)
| otherwise
= do { kind_co' <- lintStarCoercion kind_co
; lintTyCoBndr tcv $ \tcv' ->
do { body_co' <- lintCoercion body_co
; ensureEqTys (varType tcv') (coercionLKind kind_co') $
text "Kind mis-match in ForallCo" <+> ppr co
; let Pair lty rty = coercionKind body_co'
; lintForAllBody tcv' lty
; lintForAllBody tcv' rty
; when (isCoVar tcv) $
lintL (almostDevoidCoVarOfCo tcv body_co) $
text "Covar can only appear in Refl and GRefl: " <+> ppr co
; return (ForAllCo tcv' kind_co' body_co') } }
lintCoercion co@(FunCo r cow co1 co2)
= do { co1' <- lintCoercion co1
; co2' <- lintCoercion co2
; cow' <- lintCoercion cow
; let Pair lt1 rt1 = coercionKind co1
Pair lt2 rt2 = coercionKind co2
Pair ltw rtw = coercionKind cow
; lintArrow (text "coercion" <+> quotes (ppr co)) lt1 lt2 ltw
; lintArrow (text "coercion" <+> quotes (ppr co)) rt1 rt2 rtw
; lintRole co1 r (coercionRole co1)
; lintRole co2 r (coercionRole co2)
; ensureEqTys (typeKind ltw) multiplicityTy (text "coercion" <> quotes (ppr co))
; ensureEqTys (typeKind rtw) multiplicityTy (text "coercion" <> quotes (ppr co))
; let expected_mult_role = case r of
Phantom -> Phantom
_ -> Nominal
; lintRole cow expected_mult_role (coercionRole cow)
; return (FunCo r cow' co1' co2') }
lintCoercion co@(UnivCo prov r ty1 ty2)
= do { ty1' <- lintType ty1
; ty2' <- lintType ty2
; let k1 = typeKind ty1'
k2 = typeKind ty2'
; prov' <- lint_prov k1 k2 prov
; when (r /= Phantom && classifiesTypeWithValues k1
&& classifiesTypeWithValues k2)
(checkTypes ty1 ty2)
; return (UnivCo prov' r ty1' ty2') }
where
report s = hang (text $ "Unsafe coercion: " ++ s)
2 (vcat [ text "From:" <+> ppr ty1
, text " To:" <+> ppr ty2])
isUnBoxed :: PrimRep -> Bool
isUnBoxed = not . isGcPtrRep
checkTypes t1 t2
= do { checkWarnL (not lev_poly1)
(report "left-hand type is levity-polymorphic")
; checkWarnL (not lev_poly2)
(report "right-hand type is levity-polymorphic")
; when (not (lev_poly1 || lev_poly2)) $
do { checkWarnL (reps1 `equalLength` reps2)
(report "between values with different # of reps")
; zipWithM_ validateCoercion reps1 reps2 }}
where
lev_poly1 = isTypeLevPoly t1
lev_poly2 = isTypeLevPoly t2
reps1 = typePrimRep t1
reps2 = typePrimRep t2
validateCoercion :: PrimRep -> PrimRep -> LintM ()
validateCoercion rep1 rep2
= do { platform <- targetPlatform <$> getDynFlags
; checkWarnL (isUnBoxed rep1 == isUnBoxed rep2)
(report "between unboxed and boxed value")
; checkWarnL (TyCon.primRepSizeB platform rep1
== TyCon.primRepSizeB platform rep2)
(report "between unboxed values of different size")
; let fl = liftM2 (==) (TyCon.primRepIsFloat rep1)
(TyCon.primRepIsFloat rep2)
; case fl of
Nothing -> addWarnL (report "between vector types")
Just False -> addWarnL (report "between float and integral values")
_ -> return ()
}
lint_prov k1 k2 (PhantomProv kco)
= do { kco' <- lintStarCoercion kco
; lintRole co Phantom r
; check_kinds kco' k1 k2
; return (PhantomProv kco') }
lint_prov k1 k2 (ProofIrrelProv kco)
= do { lintL (isCoercionTy ty1) (mkBadProofIrrelMsg ty1 co)
; lintL (isCoercionTy ty2) (mkBadProofIrrelMsg ty2 co)
; kco' <- lintStarCoercion kco
; check_kinds kco k1 k2
; return (ProofIrrelProv kco') }
lint_prov _ _ prov@(PluginProv _) = return prov
check_kinds kco k1 k2
= do { let Pair k1' k2' = coercionKind kco
; ensureEqTys k1 k1' (mkBadUnivCoMsg CLeft co)
; ensureEqTys k2 k2' (mkBadUnivCoMsg CRight co) }
lintCoercion (SymCo co)
= do { co' <- lintCoercion co
; return (SymCo co') }
lintCoercion co@(TransCo co1 co2)
= do { co1' <- lintCoercion co1
; co2' <- lintCoercion co2
; let ty1b = coercionRKind co1'
ty2a = coercionLKind co2'
; ensureEqTys ty1b ty2a
(hang (text "Trans coercion mis-match:" <+> ppr co)
2 (vcat [ppr (coercionKind co1'), ppr (coercionKind co2')]))
; lintRole co (coercionRole co1) (coercionRole co2)
; return (TransCo co1' co2') }
lintCoercion the_co@(NthCo r0 n co)
= do { co' <- lintCoercion co
; let (Pair s t, r) = coercionKindRole co'
; case (splitForAllTy_maybe s, splitForAllTy_maybe t) of
{ (Just _, Just _)
| n == 0
, (isForAllTy_ty s && isForAllTy_ty t)
|| (isForAllTy_co s && isForAllTy_co t)
-> do { lintRole the_co Nominal r0
; return (NthCo r0 n co') }
; _ -> case (splitTyConApp_maybe s, splitTyConApp_maybe t) of
{ (Just (tc_s, tys_s), Just (tc_t, tys_t))
| tc_s == tc_t
, isInjectiveTyCon tc_s r
, tys_s `equalLength` tys_t
, tys_s `lengthExceeds` n
-> do { lintRole the_co tr r0
; return (NthCo r0 n co') }
where
tr = nthRole r tc_s n
; _ -> failWithL (hang (text "Bad getNth:")
2 (ppr the_co $$ ppr s $$ ppr t)) }}}
lintCoercion the_co@(LRCo lr co)
= do { co' <- lintCoercion co
; let Pair s t = coercionKind co'
r = coercionRole co'
; lintRole co Nominal r
; case (splitAppTy_maybe s, splitAppTy_maybe t) of
(Just _, Just _) -> return (LRCo lr co')
_ -> failWithL (hang (text "Bad LRCo:")
2 (ppr the_co $$ ppr s $$ ppr t)) }
lintCoercion (InstCo co arg)
= do { co' <- lintCoercion co
; arg' <- lintCoercion arg
; let Pair t1 t2 = coercionKind co'
Pair s1 s2 = coercionKind arg'
; lintRole arg Nominal (coercionRole arg')
; case (splitForAllTy_ty_maybe t1, splitForAllTy_ty_maybe t2) of
{ (Just (tv1,_), Just (tv2,_))
| typeKind s1 `eqType` tyVarKind tv1
, typeKind s2 `eqType` tyVarKind tv2
-> return (InstCo co' arg')
| otherwise
-> failWithL (text "Kind mis-match in inst coercion1" <+> ppr co)
; _ -> case (splitForAllTy_co_maybe t1, splitForAllTy_co_maybe t2) of
{ (Just (cv1, _), Just (cv2, _))
| typeKind s1 `eqType` varType cv1
, typeKind s2 `eqType` varType cv2
, CoercionTy _ <- s1
, CoercionTy _ <- s2
-> return (InstCo co' arg')
| otherwise
-> failWithL (text "Kind mis-match in inst coercion2" <+> ppr co)
; _ -> failWithL (text "Bad argument of inst") }}}
lintCoercion co@(AxiomInstCo con ind cos)
= do { unless (0 <= ind && ind < numBranches (coAxiomBranches con))
(bad_ax (text "index out of range"))
; let CoAxBranch { cab_tvs = ktvs
, cab_cvs = cvs
, cab_roles = roles } = coAxiomNthBranch con ind
; unless (cos `equalLength` (ktvs ++ cvs)) $
bad_ax (text "lengths")
; cos' <- mapM lintCoercion cos
; subst <- getTCvSubst
; let empty_subst = zapTCvSubst subst
; _ <- foldlM check_ki (empty_subst, empty_subst)
(zip3 (ktvs ++ cvs) roles cos')
; let fam_tc = coAxiomTyCon con
; case checkAxInstCo co of
Just bad_branch -> bad_ax $ text "inconsistent with" <+>
pprCoAxBranch fam_tc bad_branch
Nothing -> return ()
; return (AxiomInstCo con ind cos') }
where
bad_ax what = addErrL (hang (text "Bad axiom application" <+> parens what)
2 (ppr co))
check_ki (subst_l, subst_r) (ktv, role, arg')
= do { let Pair s' t' = coercionKind arg'
sk' = typeKind s'
tk' = typeKind t'
; lintRole arg' role (coercionRole arg')
; let ktv_kind_l = substTy subst_l (tyVarKind ktv)
ktv_kind_r = substTy subst_r (tyVarKind ktv)
; unless (sk' `eqType` ktv_kind_l)
(bad_ax (text "check_ki1" <+> vcat [ ppr co, ppr sk', ppr ktv, ppr ktv_kind_l ] ))
; unless (tk' `eqType` ktv_kind_r)
(bad_ax (text "check_ki2" <+> vcat [ ppr co, ppr tk', ppr ktv, ppr ktv_kind_r ] ))
; return (extendTCvSubst subst_l ktv s',
extendTCvSubst subst_r ktv t') }
lintCoercion (KindCo co)
= do { co' <- lintCoercion co
; return (KindCo co') }
lintCoercion (SubCo co')
= do { co' <- lintCoercion co'
; lintRole co' Nominal (coercionRole co')
; return (SubCo co') }
lintCoercion this@(AxiomRuleCo ax cos)
= do { cos' <- mapM lintCoercion cos
; lint_roles 0 (coaxrAsmpRoles ax) cos'
; case coaxrProves ax (map coercionKind cos') of
Nothing -> err "Malformed use of AxiomRuleCo" [ ppr this ]
Just _ -> return (AxiomRuleCo ax cos') }
where
err m xs = failWithL $
hang (text m) 2 $ vcat (text "Rule:" <+> ppr (coaxrName ax) : xs)
lint_roles n (e : es) (co : cos)
| e == coercionRole co = lint_roles (n+1) es cos
| otherwise = err "Argument roles mismatch"
[ text "In argument:" <+> int (n+1)
, text "Expected:" <+> ppr e
, text "Found:" <+> ppr (coercionRole co) ]
lint_roles _ [] [] = return ()
lint_roles n [] rs = err "Too many coercion arguments"
[ text "Expected:" <+> int n
, text "Provided:" <+> int (n + length rs) ]
lint_roles n es [] = err "Not enough coercion arguments"
[ text "Expected:" <+> int (n + length es)
, text "Provided:" <+> int n ]
lintCoercion (HoleCo h)
= do { addErrL $ text "Unfilled coercion hole:" <+> ppr h
; lintCoercion (CoVarCo (coHoleCoVar h)) }
lintAxioms :: DynFlags
-> [CoAxiom Branched]
-> WarnsAndErrs
lintAxioms dflags axioms
= initL dflags (defaultLintFlags dflags) [] $
do { mapM_ lint_axiom axioms
; let axiom_groups = groupWith coAxiomTyCon axioms
; mapM_ lint_axiom_group axiom_groups }
lint_axiom :: CoAxiom Branched -> LintM ()
lint_axiom ax@(CoAxiom { co_ax_tc = tc, co_ax_branches = branches
, co_ax_role = ax_role })
= addLoc (InAxiom ax) $
do { mapM_ (lint_branch tc) branch_list
; extra_checks }
where
branch_list = fromBranches branches
extra_checks
| isNewTyCon tc
= do { CoAxBranch { cab_tvs = tvs
, cab_eta_tvs = eta_tvs
, cab_cvs = cvs
, cab_roles = roles
, cab_lhs = lhs_tys }
<- case branch_list of
[branch] -> return branch
_ -> failWithL (text "multi-branch axiom with newtype")
; let ax_lhs = mkInfForAllTys tvs $
mkTyConApp tc lhs_tys
nt_tvs = takeList tvs (tyConTyVars tc)
nt_lhs = mkInfForAllTys nt_tvs $
mkTyConApp tc (mkTyVarTys nt_tvs)
; lintL (ax_lhs `eqType` nt_lhs)
(text "Newtype axiom LHS does not match newtype definition")
; lintL (null cvs)
(text "Newtype axiom binds coercion variables")
; lintL (null eta_tvs)
(text "Newtype axiom has eta-tvs")
; lintL (ax_role == Representational)
(text "Newtype axiom role not representational")
; lintL (roles `equalLength` tvs)
(text "Newtype axiom roles list is the wrong length." $$
text "roles:" <+> sep (map ppr roles))
; lintL (roles == takeList roles (tyConRoles tc))
(vcat [ text "Newtype axiom roles do not match newtype tycon's."
, text "axiom roles:" <+> sep (map ppr roles)
, text "tycon roles:" <+> sep (map ppr (tyConRoles tc)) ])
}
| isFamilyTyCon tc
= do { if | isTypeFamilyTyCon tc
-> lintL (ax_role == Nominal)
(text "type family axiom is not nominal")
| isDataFamilyTyCon tc
-> lintL (ax_role == Representational)
(text "data family axiom is not representational")
| otherwise
-> addErrL (text "A family TyCon is neither a type family nor a data family:" <+> ppr tc)
; mapM_ (lint_family_branch tc) branch_list }
| otherwise
= addErrL (text "Axiom tycon is neither a newtype nor a family.")
lint_branch :: TyCon -> CoAxBranch -> LintM ()
lint_branch ax_tc (CoAxBranch { cab_tvs = tvs, cab_cvs = cvs
, cab_lhs = lhs_args, cab_rhs = rhs })
= lintBinders LambdaBind (tvs ++ cvs) $ \_ ->
do { let lhs = mkTyConApp ax_tc lhs_args
; lhs' <- lintType lhs
; rhs' <- lintType rhs
; let lhs_kind = typeKind lhs'
rhs_kind = typeKind rhs'
; lintL (lhs_kind `eqType` rhs_kind) $
hang (text "Inhomogeneous axiom")
2 (text "lhs:" <+> ppr lhs <+> dcolon <+> ppr lhs_kind $$
text "rhs:" <+> ppr rhs <+> dcolon <+> ppr rhs_kind) }
lint_family_branch :: TyCon -> CoAxBranch -> LintM ()
lint_family_branch fam_tc br@(CoAxBranch { cab_tvs = tvs
, cab_eta_tvs = eta_tvs
, cab_cvs = cvs
, cab_roles = roles
, cab_lhs = lhs
, cab_incomps = incomps })
= do { lintL (isDataFamilyTyCon fam_tc || null eta_tvs)
(text "Type family axiom has eta-tvs")
; lintL (all (`elemVarSet` tyCoVarsOfTypes lhs) tvs)
(text "Quantified variable in family axiom unused in LHS")
; lintL (all isTyFamFree lhs)
(text "Type family application on LHS of family axiom")
; lintL (all (== Nominal) roles)
(text "Non-nominal role in family axiom" $$
text "roles:" <+> sep (map ppr roles))
; lintL (null cvs)
(text "Coercion variables bound in family axiom")
; forM_ incomps $ \ br' ->
lintL (not (compatible_branches br br')) $
text "Incorrect incompatible branch:" <+> ppr br' }
lint_axiom_group :: NonEmpty (CoAxiom Branched) -> LintM ()
lint_axiom_group (_ :| []) = return ()
lint_axiom_group (ax :| axs)
= do { lintL (isOpenFamilyTyCon tc)
(text "Non-open-family with multiple axioms")
; let all_pairs = [ (ax1, ax2) | ax1 <- all_axs
, ax2 <- all_axs ]
; mapM_ (lint_axiom_pair tc) all_pairs }
where
all_axs = ax : axs
tc = coAxiomTyCon ax
lint_axiom_pair :: TyCon -> (CoAxiom Branched, CoAxiom Branched) -> LintM ()
lint_axiom_pair tc (ax1, ax2)
| Just br1@(CoAxBranch { cab_tvs = tvs1
, cab_lhs = lhs1
, cab_rhs = rhs1 }) <- coAxiomSingleBranch_maybe ax1
, Just br2@(CoAxBranch { cab_tvs = tvs2
, cab_lhs = lhs2
, cab_rhs = rhs2 }) <- coAxiomSingleBranch_maybe ax2
= lintL (compatible_branches br1 br2) $
vcat [ hsep [ text "Axioms", ppr ax1, text "and", ppr ax2
, text "are incompatible" ]
, text "tvs1 =" <+> pprTyVars tvs1
, text "lhs1 =" <+> ppr (mkTyConApp tc lhs1)
, text "rhs1 =" <+> ppr rhs1
, text "tvs2 =" <+> pprTyVars tvs2
, text "lhs2 =" <+> ppr (mkTyConApp tc lhs2)
, text "rhs2 =" <+> ppr rhs2 ]
| otherwise
= addErrL (text "Open type family axiom has more than one branch: either" <+>
ppr ax1 <+> text "or" <+> ppr ax2)
compatible_branches :: CoAxBranch -> CoAxBranch -> Bool
compatible_branches (CoAxBranch { cab_tvs = tvs1
, cab_lhs = lhs1
, cab_rhs = rhs1 })
(CoAxBranch { cab_tvs = tvs2
, cab_lhs = lhs2
, cab_rhs = rhs2 })
=
let in_scope = mkInScopeSet (mkVarSet tvs1)
subst0 = mkEmptyTCvSubst in_scope
(subst, _) = substTyVarBndrs subst0 tvs2
lhs2' = substTys subst lhs2
rhs2' = substTy subst rhs2
in
case tcUnifyTys (const BindMe) lhs1 lhs2' of
Just unifying_subst -> substTy unifying_subst rhs1 `eqType`
substTy unifying_subst rhs2'
Nothing -> True
data LintEnv
= LE { le_flags :: LintFlags
, le_loc :: [LintLocInfo]
, le_subst :: TCvSubst
, le_ids :: VarEnv (Id, LintedType)
, le_joins :: IdSet
, le_dynflags :: DynFlags
, le_ue_aliases :: NameEnv UsageEnv
}
data LintFlags
= LF { lf_check_global_ids :: Bool
, lf_check_inline_loop_breakers :: Bool
, lf_check_static_ptrs :: StaticPtrCheck
, lf_report_unsat_syns :: Bool
, lf_check_linearity :: Bool
, lf_check_levity_poly :: Bool
}
data StaticPtrCheck
= AllowAnywhere
| AllowAtTopLevel
| RejectEverywhere
deriving Eq
defaultLintFlags :: DynFlags -> LintFlags
defaultLintFlags dflags = LF { lf_check_global_ids = False
, lf_check_inline_loop_breakers = True
, lf_check_static_ptrs = AllowAnywhere
, lf_check_linearity = gopt Opt_DoLinearCoreLinting dflags
, lf_report_unsat_syns = True
, lf_check_levity_poly = True
}
newtype LintM a =
LintM { unLintM ::
LintEnv ->
WarnsAndErrs ->
(Maybe a, WarnsAndErrs) }
deriving (Functor)
type WarnsAndErrs = (Bag MsgDoc, Bag MsgDoc)
instance Applicative LintM where
pure x = LintM $ \ _ errs -> (Just x, errs)
(<*>) = ap
instance Monad LintM where
m >>= k = LintM (\ env errs ->
let (res, errs') = unLintM m env errs in
case res of
Just r -> unLintM (k r) env errs'
Nothing -> (Nothing, errs'))
instance MonadFail LintM where
fail err = failWithL (text err)
instance HasDynFlags LintM where
getDynFlags = LintM (\ e errs -> (Just (le_dynflags e), errs))
data LintLocInfo
= RhsOf Id
| OccOf Id
| LambdaBodyOf Id
| RuleOf Id
| UnfoldingOf Id
| BodyOfLetRec [Id]
| CaseAlt CoreAlt
| CasePat CoreAlt
| CaseTy CoreExpr
| IdTy Id
| AnExpr CoreExpr
| ImportedUnfolding SrcLoc
| TopLevelBindings
| InType Type
| InCo Coercion
| InAxiom (CoAxiom Branched)
initL :: DynFlags -> LintFlags -> [Var]
-> LintM a -> WarnsAndErrs
initL dflags flags vars m
= case unLintM m env (emptyBag, emptyBag) of
(Just _, errs) -> errs
(Nothing, errs@(_, e)) | not (isEmptyBag e) -> errs
| otherwise -> pprPanic ("Bug in Lint: a failure occurred " ++
"without reporting an error message") empty
where
(tcvs, ids) = partition isTyCoVar vars
env = LE { le_flags = flags
, le_subst = mkEmptyTCvSubst (mkInScopeSet (mkVarSet tcvs))
, le_ids = mkVarEnv [(id, (id,idType id)) | id <- ids]
, le_joins = emptyVarSet
, le_loc = []
, le_dynflags = dflags
, le_ue_aliases = emptyNameEnv }
setReportUnsat :: Bool -> LintM a -> LintM a
setReportUnsat ru thing_inside
= LintM $ \ env errs ->
let env' = env { le_flags = (le_flags env) { lf_report_unsat_syns = ru } }
in unLintM thing_inside env' errs
noLPChecks :: LintM a -> LintM a
noLPChecks thing_inside
= LintM $ \env errs ->
let env' = env { le_flags = (le_flags env) { lf_check_levity_poly = False } }
in unLintM thing_inside env' errs
getLintFlags :: LintM LintFlags
getLintFlags = LintM $ \ env errs -> (Just (le_flags env), errs)
checkL :: Bool -> MsgDoc -> LintM ()
checkL True _ = return ()
checkL False msg = failWithL msg
lintL :: Bool -> MsgDoc -> LintM ()
lintL = checkL
checkWarnL :: Bool -> MsgDoc -> LintM ()
checkWarnL True _ = return ()
checkWarnL False msg = addWarnL msg
failWithL :: MsgDoc -> LintM a
failWithL msg = LintM $ \ env (warns,errs) ->
(Nothing, (warns, addMsg True env errs msg))
addErrL :: MsgDoc -> LintM ()
addErrL msg = LintM $ \ env (warns,errs) ->
(Just (), (warns, addMsg True env errs msg))
addWarnL :: MsgDoc -> LintM ()
addWarnL msg = LintM $ \ env (warns,errs) ->
(Just (), (addMsg False env warns msg, errs))
addMsg :: Bool -> LintEnv -> Bag MsgDoc -> MsgDoc -> Bag MsgDoc
addMsg is_error env msgs msg
= ASSERT2( notNull loc_msgs, msg )
msgs `snocBag` mk_msg msg
where
loc_msgs :: [(SrcLoc, SDoc)]
loc_msgs = map dumpLoc (le_loc env)
cxt_doc = vcat [ vcat $ reverse $ map snd loc_msgs
, text "Substitution:" <+> ppr (le_subst env) ]
context | is_error = cxt_doc
| otherwise = whenPprDebug cxt_doc
msg_span = case [ span | (loc,_) <- loc_msgs
, let span = srcLocSpan loc
, isGoodSrcSpan span ] of
[] -> noSrcSpan
(s:_) -> s
mk_msg msg = mkLocMessage SevWarning msg_span
(msg $$ context)
addLoc :: LintLocInfo -> LintM a -> LintM a
addLoc extra_loc m
= LintM $ \ env errs ->
unLintM m (env { le_loc = extra_loc : le_loc env }) errs
inCasePat :: LintM Bool
inCasePat = LintM $ \ env errs -> (Just (is_case_pat env), errs)
where
is_case_pat (LE { le_loc = CasePat {} : _ }) = True
is_case_pat _other = False
addInScopeId :: Id -> LintedType -> LintM a -> LintM a
addInScopeId id linted_ty m
= LintM $ \ env@(LE { le_ids = id_set, le_joins = join_set }) errs ->
unLintM m (env { le_ids = extendVarEnv id_set id (id, linted_ty)
, le_joins = add_joins join_set }) errs
where
add_joins join_set
| isJoinId id = extendVarSet join_set id
| otherwise = delVarSet join_set id
getInScopeIds :: LintM (VarEnv (Id,LintedType))
getInScopeIds = LintM (\env errs -> (Just (le_ids env), errs))
extendTvSubstL :: TyVar -> Type -> LintM a -> LintM a
extendTvSubstL tv ty m
= LintM $ \ env errs ->
unLintM m (env { le_subst = Type.extendTvSubst (le_subst env) tv ty }) errs
updateTCvSubst :: TCvSubst -> LintM a -> LintM a
updateTCvSubst subst' m
= LintM $ \ env errs -> unLintM m (env { le_subst = subst' }) errs
markAllJoinsBad :: LintM a -> LintM a
markAllJoinsBad m
= LintM $ \ env errs -> unLintM m (env { le_joins = emptyVarSet }) errs
markAllJoinsBadIf :: Bool -> LintM a -> LintM a
markAllJoinsBadIf True m = markAllJoinsBad m
markAllJoinsBadIf False m = m
getValidJoins :: LintM IdSet
getValidJoins = LintM (\ env errs -> (Just (le_joins env), errs))
getTCvSubst :: LintM TCvSubst
getTCvSubst = LintM (\ env errs -> (Just (le_subst env), errs))
getUEAliases :: LintM (NameEnv UsageEnv)
getUEAliases = LintM (\ env errs -> (Just (le_ue_aliases env), errs))
getInScope :: LintM InScopeSet
getInScope = LintM (\ env errs -> (Just (getTCvInScope $ le_subst env), errs))
lookupIdInScope :: Id -> LintM (Id, LintedType)
lookupIdInScope id_occ
= do { in_scope_ids <- getInScopeIds
; case lookupVarEnv in_scope_ids id_occ of
Just (id_bndr, linted_ty)
-> do { checkL (not (bad_global id_bndr)) global_in_scope
; return (id_bndr, linted_ty) }
Nothing -> do { checkL (not is_local) local_out_of_scope
; return (id_occ, idType id_occ) } }
where
is_local = mustHaveLocalBinding id_occ
local_out_of_scope = text "Out of scope:" <+> pprBndr LetBind id_occ
global_in_scope = hang (text "Occurrence is GlobalId, but binding is LocalId")
2 (pprBndr LetBind id_occ)
bad_global id_bnd = isGlobalId id_occ
&& isLocalId id_bnd
&& not (isWiredIn id_occ)
lookupJoinId :: Id -> LintM (Maybe JoinArity)
lookupJoinId id
= do { join_set <- getValidJoins
; case lookupVarSet join_set id of
Just id' -> return (isJoinId_maybe id')
Nothing -> return Nothing }
addAliasUE :: Id -> UsageEnv -> LintM a -> LintM a
addAliasUE id ue thing_inside = LintM $ \ env errs ->
let new_ue_aliases =
extendNameEnv (le_ue_aliases env) (getName id) ue
in
unLintM thing_inside (env { le_ue_aliases = new_ue_aliases }) errs
varCallSiteUsage :: Id -> LintM UsageEnv
varCallSiteUsage id =
do m <- getUEAliases
return $ case lookupNameEnv m (getName id) of
Nothing -> unitUE id One
Just id_ue -> id_ue
ensureEqTys :: LintedType -> LintedType -> MsgDoc -> LintM ()
ensureEqTys ty1 ty2 msg = lintL (ty1 `eqType` ty2) msg
ensureSubUsage :: Usage -> Mult -> SDoc -> LintM ()
ensureSubUsage Bottom _ _ = return ()
ensureSubUsage Zero described_mult err_msg = ensureSubMult Many described_mult err_msg
ensureSubUsage (MUsage m) described_mult err_msg = ensureSubMult m described_mult err_msg
ensureSubMult :: Mult -> Mult -> SDoc -> LintM ()
ensureSubMult actual_usage described_usage err_msg = do
flags <- getLintFlags
when (lf_check_linearity flags) $ case actual_usage' `submult` described_usage' of
Submult -> return ()
Unknown -> case isMultMul actual_usage' of
Just (m1, m2) -> ensureSubMult m1 described_usage' err_msg >>
ensureSubMult m2 described_usage' err_msg
Nothing -> when (not (actual_usage' `eqType` described_usage')) (addErrL err_msg)
where actual_usage' = normalize actual_usage
described_usage' = normalize described_usage
normalize :: Mult -> Mult
normalize m = case isMultMul m of
Just (m1, m2) -> mkMultMul (normalize m1) (normalize m2)
Nothing -> m
lintRole :: Outputable thing
=> thing
-> Role
-> Role
-> LintM ()
lintRole co r1 r2
= lintL (r1 == r2)
(text "Role incompatibility: expected" <+> ppr r1 <> comma <+>
text "got" <+> ppr r2 $$
text "in" <+> ppr co)
dumpLoc :: LintLocInfo -> (SrcLoc, SDoc)
dumpLoc (RhsOf v)
= (getSrcLoc v, text "In the RHS of" <+> pp_binders [v])
dumpLoc (OccOf v)
= (getSrcLoc v, text "In an occurrence of" <+> pp_binder v)
dumpLoc (LambdaBodyOf b)
= (getSrcLoc b, text "In the body of lambda with binder" <+> pp_binder b)
dumpLoc (RuleOf b)
= (getSrcLoc b, text "In a rule attached to" <+> pp_binder b)
dumpLoc (UnfoldingOf b)
= (getSrcLoc b, text "In the unfolding of" <+> pp_binder b)
dumpLoc (BodyOfLetRec [])
= (noSrcLoc, text "In body of a letrec with no binders")
dumpLoc (BodyOfLetRec bs@(_:_))
= ( getSrcLoc (head bs), text "In the body of letrec with binders" <+> pp_binders bs)
dumpLoc (AnExpr e)
= (noSrcLoc, text "In the expression:" <+> ppr e)
dumpLoc (CaseAlt (con, args, _))
= (noSrcLoc, text "In a case alternative:" <+> parens (ppr con <+> pp_binders args))
dumpLoc (CasePat (con, args, _))
= (noSrcLoc, text "In the pattern of a case alternative:" <+> parens (ppr con <+> pp_binders args))
dumpLoc (CaseTy scrut)
= (noSrcLoc, hang (text "In the result-type of a case with scrutinee:")
2 (ppr scrut))
dumpLoc (IdTy b)
= (getSrcLoc b, text "In the type of a binder:" <+> ppr b)
dumpLoc (ImportedUnfolding locn)
= (locn, text "In an imported unfolding")
dumpLoc TopLevelBindings
= (noSrcLoc, Outputable.empty)
dumpLoc (InType ty)
= (noSrcLoc, text "In the type" <+> quotes (ppr ty))
dumpLoc (InCo co)
= (noSrcLoc, text "In the coercion" <+> quotes (ppr co))
dumpLoc (InAxiom ax)
= (getSrcLoc ax_name, text "In the coercion axiom" <+> ppr ax_name <+> dcolon <+> pp_ax)
where
CoAxiom { co_ax_name = ax_name
, co_ax_tc = tc
, co_ax_role = ax_role
, co_ax_branches = branches } = ax
branch_list = fromBranches branches
pp_ax
| [branch] <- branch_list
= pp_branch branch
| otherwise
= braces $ vcat (map pp_branch branch_list)
pp_branch (CoAxBranch { cab_tvs = tvs
, cab_cvs = cvs
, cab_lhs = lhs_tys
, cab_rhs = rhs_ty })
= sep [ brackets (pprWithCommas pprTyVar (tvs ++ cvs)) <> dot
, ppr (mkTyConApp tc lhs_tys)
, text "~_" <> pp_role ax_role
, ppr rhs_ty ]
pp_role Nominal = text "N"
pp_role Representational = text "R"
pp_role Phantom = text "P"
pp_binders :: [Var] -> SDoc
pp_binders bs = sep (punctuate comma (map pp_binder bs))
pp_binder :: Var -> SDoc
pp_binder b | isId b = hsep [ppr b, dcolon, ppr (idType b)]
| otherwise = hsep [ppr b, dcolon, ppr (tyVarKind b)]
mkDefaultArgsMsg :: [Var] -> MsgDoc
mkDefaultArgsMsg args
= hang (text "DEFAULT case with binders")
4 (ppr args)
mkCaseAltMsg :: CoreExpr -> Type -> Type -> MsgDoc
mkCaseAltMsg e ty1 ty2
= hang (text "Type of case alternatives not the same as the annotation on case:")
4 (vcat [ text "Actual type:" <+> ppr ty1,
text "Annotation on case:" <+> ppr ty2,
text "Alt Rhs:" <+> ppr e ])
mkScrutMsg :: Id -> Type -> Type -> TCvSubst -> MsgDoc
mkScrutMsg var var_ty scrut_ty subst
= vcat [text "Result binder in case doesn't match scrutinee:" <+> ppr var,
text "Result binder type:" <+> ppr var_ty,
text "Scrutinee type:" <+> ppr scrut_ty,
hsep [text "Current TCv subst", ppr subst]]
mkNonDefltMsg, mkNonIncreasingAltsMsg :: CoreExpr -> MsgDoc
mkNonDefltMsg e
= hang (text "Case expression with DEFAULT not at the beginning") 4 (ppr e)
mkNonIncreasingAltsMsg e
= hang (text "Case expression with badly-ordered alternatives") 4 (ppr e)
nonExhaustiveAltsMsg :: CoreExpr -> MsgDoc
nonExhaustiveAltsMsg e
= hang (text "Case expression with non-exhaustive alternatives") 4 (ppr e)
mkBadConMsg :: TyCon -> DataCon -> MsgDoc
mkBadConMsg tycon datacon
= vcat [
text "In a case alternative, data constructor isn't in scrutinee type:",
text "Scrutinee type constructor:" <+> ppr tycon,
text "Data con:" <+> ppr datacon
]
mkBadPatMsg :: Type -> Type -> MsgDoc
mkBadPatMsg con_result_ty scrut_ty
= vcat [
text "In a case alternative, pattern result type doesn't match scrutinee type:",
text "Pattern result type:" <+> ppr con_result_ty,
text "Scrutinee type:" <+> ppr scrut_ty
]
integerScrutinisedMsg :: MsgDoc
integerScrutinisedMsg
= text "In a LitAlt, the literal is lifted (probably Integer)"
mkBadAltMsg :: Type -> CoreAlt -> MsgDoc
mkBadAltMsg scrut_ty alt
= vcat [ text "Data alternative when scrutinee is not a tycon application",
text "Scrutinee type:" <+> ppr scrut_ty,
text "Alternative:" <+> pprCoreAlt alt ]
mkNewTyDataConAltMsg :: Type -> CoreAlt -> MsgDoc
mkNewTyDataConAltMsg scrut_ty alt
= vcat [ text "Data alternative for newtype datacon",
text "Scrutinee type:" <+> ppr scrut_ty,
text "Alternative:" <+> pprCoreAlt alt ]
mkAppMsg :: Type -> Type -> CoreExpr -> MsgDoc
mkAppMsg fun_ty arg_ty arg
= vcat [text "Argument value doesn't match argument type:",
hang (text "Fun type:") 4 (ppr fun_ty),
hang (text "Arg type:") 4 (ppr arg_ty),
hang (text "Arg:") 4 (ppr arg)]
mkNonFunAppMsg :: Type -> Type -> CoreExpr -> MsgDoc
mkNonFunAppMsg fun_ty arg_ty arg
= vcat [text "Non-function type in function position",
hang (text "Fun type:") 4 (ppr fun_ty),
hang (text "Arg type:") 4 (ppr arg_ty),
hang (text "Arg:") 4 (ppr arg)]
mkLetErr :: TyVar -> CoreExpr -> MsgDoc
mkLetErr bndr rhs
= vcat [text "Bad `let' binding:",
hang (text "Variable:")
4 (ppr bndr <+> dcolon <+> ppr (varType bndr)),
hang (text "Rhs:")
4 (ppr rhs)]
mkTyAppMsg :: Type -> Type -> MsgDoc
mkTyAppMsg ty arg_ty
= vcat [text "Illegal type application:",
hang (text "Exp type:")
4 (ppr ty <+> dcolon <+> ppr (typeKind ty)),
hang (text "Arg type:")
4 (ppr arg_ty <+> dcolon <+> ppr (typeKind arg_ty))]
emptyRec :: CoreExpr -> MsgDoc
emptyRec e = hang (text "Empty Rec binding:") 2 (ppr e)
mkRhsMsg :: Id -> SDoc -> Type -> MsgDoc
mkRhsMsg binder what ty
= vcat
[hsep [text "The type of this binder doesn't match the type of its" <+> what <> colon,
ppr binder],
hsep [text "Binder's type:", ppr (idType binder)],
hsep [text "Rhs type:", ppr ty]]
mkLetAppMsg :: CoreExpr -> MsgDoc
mkLetAppMsg e
= hang (text "This argument does not satisfy the let/app invariant:")
2 (ppr e)
badBndrTyMsg :: Id -> SDoc -> MsgDoc
badBndrTyMsg binder what
= vcat [ text "The type of this binder is" <+> what <> colon <+> ppr binder
, text "Binder's type:" <+> ppr (idType binder) ]
mkStrictMsg :: Id -> MsgDoc
mkStrictMsg binder
= vcat [hsep [text "Recursive or top-level binder has strict demand info:",
ppr binder],
hsep [text "Binder's demand info:", ppr (idDemandInfo binder)]
]
mkNonTopExportedMsg :: Id -> MsgDoc
mkNonTopExportedMsg binder
= hsep [text "Non-top-level binder is marked as exported:", ppr binder]
mkNonTopExternalNameMsg :: Id -> MsgDoc
mkNonTopExternalNameMsg binder
= hsep [text "Non-top-level binder has an external name:", ppr binder]
mkTopNonLitStrMsg :: Id -> MsgDoc
mkTopNonLitStrMsg binder
= hsep [text "Top-level Addr# binder has a non-literal rhs:", ppr binder]
mkKindErrMsg :: TyVar -> Type -> MsgDoc
mkKindErrMsg tyvar arg_ty
= vcat [text "Kinds don't match in type application:",
hang (text "Type variable:")
4 (ppr tyvar <+> dcolon <+> ppr (tyVarKind tyvar)),
hang (text "Arg type:")
4 (ppr arg_ty <+> dcolon <+> ppr (typeKind arg_ty))]
mkCastErr :: CoreExpr -> Coercion -> Type -> Type -> MsgDoc
mkCastErr expr = mk_cast_err "expression" "type" (ppr expr)
mkCastTyErr :: Type -> Coercion -> Kind -> Kind -> MsgDoc
mkCastTyErr ty = mk_cast_err "type" "kind" (ppr ty)
mk_cast_err :: String
-> String
-> SDoc
-> Coercion -> Type -> Type -> MsgDoc
mk_cast_err thing_str co_str pp_thing co from_ty thing_ty
= vcat [from_msg <+> text "of Cast differs from" <+> co_msg
<+> text "of" <+> enclosed_msg,
from_msg <> colon <+> ppr from_ty,
text (capitalise co_str) <+> text "of" <+> enclosed_msg <> colon
<+> ppr thing_ty,
text "Actual" <+> enclosed_msg <> colon <+> pp_thing,
text "Coercion used in cast:" <+> ppr co
]
where
co_msg, from_msg, enclosed_msg :: SDoc
co_msg = text co_str
from_msg = text "From-" <> co_msg
enclosed_msg = text "enclosed" <+> text thing_str
mkBadUnivCoMsg :: LeftOrRight -> Coercion -> SDoc
mkBadUnivCoMsg lr co
= text "Kind mismatch on the" <+> pprLeftOrRight lr <+>
text "side of a UnivCo:" <+> ppr co
mkBadProofIrrelMsg :: Type -> Coercion -> SDoc
mkBadProofIrrelMsg ty co
= hang (text "Found a non-coercion in a proof-irrelevance UnivCo:")
2 (vcat [ text "type:" <+> ppr ty
, text "co:" <+> ppr co ])
mkBadTyVarMsg :: Var -> SDoc
mkBadTyVarMsg tv
= text "Non-tyvar used in TyVarTy:"
<+> ppr tv <+> dcolon <+> ppr (varType tv)
mkBadJoinBindMsg :: Var -> SDoc
mkBadJoinBindMsg var
= vcat [ text "Bad join point binding:" <+> ppr var
, text "Join points can be bound only by a non-top-level let" ]
mkInvalidJoinPointMsg :: Var -> Type -> SDoc
mkInvalidJoinPointMsg var ty
= hang (text "Join point has invalid type:")
2 (ppr var <+> dcolon <+> ppr ty)
mkBadJoinArityMsg :: Var -> Int -> Int -> CoreExpr -> SDoc
mkBadJoinArityMsg var ar n rhs
= vcat [ text "Join point has too few lambdas",
text "Join var:" <+> ppr var,
text "Join arity:" <+> ppr ar,
text "Number of lambdas:" <+> ppr (ar n),
text "Rhs = " <+> ppr rhs
]
invalidJoinOcc :: Var -> SDoc
invalidJoinOcc var
= vcat [ text "Invalid occurrence of a join variable:" <+> ppr var
, text "The binder is either not a join point, or not valid here" ]
mkBadJumpMsg :: Var -> Int -> Int -> SDoc
mkBadJumpMsg var ar nargs
= vcat [ text "Join point invoked with wrong number of arguments",
text "Join var:" <+> ppr var,
text "Join arity:" <+> ppr ar,
text "Number of arguments:" <+> int nargs ]
mkInconsistentRecMsg :: [Var] -> SDoc
mkInconsistentRecMsg bndrs
= vcat [ text "Recursive let binders mix values and join points",
text "Binders:" <+> hsep (map ppr_with_details bndrs) ]
where
ppr_with_details bndr = ppr bndr <> ppr (idDetails bndr)
mkJoinBndrOccMismatchMsg :: Var -> JoinArity -> JoinArity -> SDoc
mkJoinBndrOccMismatchMsg bndr join_arity_bndr join_arity_occ
= vcat [ text "Mismatch in join point arity between binder and occurrence"
, text "Var:" <+> ppr bndr
, text "Arity at binding site:" <+> ppr join_arity_bndr
, text "Arity at occurrence: " <+> ppr join_arity_occ ]
mkBndrOccTypeMismatchMsg :: Var -> Var -> LintedType -> LintedType -> SDoc
mkBndrOccTypeMismatchMsg bndr var bndr_ty var_ty
= vcat [ text "Mismatch in type between binder and occurrence"
, text "Binder:" <+> ppr bndr <+> dcolon <+> ppr bndr_ty
, text "Occurrence:" <+> ppr var <+> dcolon <+> ppr var_ty
, text " Before subst:" <+> ppr (idType var) ]
mkBadJoinPointRuleMsg :: JoinId -> JoinArity -> CoreRule -> SDoc
mkBadJoinPointRuleMsg bndr join_arity rule
= vcat [ text "Join point has rule with wrong number of arguments"
, text "Var:" <+> ppr bndr
, text "Join arity:" <+> ppr join_arity
, text "Rule:" <+> ppr rule ]
pprLeftOrRight :: LeftOrRight -> MsgDoc
pprLeftOrRight CLeft = text "left"
pprLeftOrRight CRight = text "right"
dupVars :: [NonEmpty Var] -> MsgDoc
dupVars vars
= hang (text "Duplicate variables brought into scope")
2 (ppr (map toList vars))
dupExtVars :: [NonEmpty Name] -> MsgDoc
dupExtVars vars
= hang (text "Duplicate top-level variables with the same qualified name")
2 (ppr (map toList vars))
lintAnnots :: SDoc -> (ModGuts -> CoreM ModGuts) -> ModGuts -> CoreM ModGuts
lintAnnots pname pass guts = do
dflags <- getDynFlags
when (gopt Opt_DoAnnotationLinting dflags) $
liftIO $ Err.showPass dflags "Annotation linting - first run"
nguts <- pass guts
when (gopt Opt_DoAnnotationLinting dflags) $ do
liftIO $ Err.showPass dflags "Annotation linting - second run"
nguts' <- withoutAnnots pass guts
liftIO $ Err.showPass dflags "Annotation linting - comparison"
let binds = flattenBinds $ mg_binds nguts
binds' = flattenBinds $ mg_binds nguts'
(diffs,_) = diffBinds True (mkRnEnv2 emptyInScopeSet) binds binds'
when (not (null diffs)) $ GHC.Core.Opt.Monad.putMsg $ vcat
[ lint_banner "warning" pname
, text "Core changes with annotations:"
, withPprStyle defaultDumpStyle $ nest 2 $ vcat diffs
]
return nguts
withoutAnnots :: (ModGuts -> CoreM ModGuts) -> ModGuts -> CoreM ModGuts
withoutAnnots pass guts = do
dflags <- getDynFlags
let removeFlag env = env{ hsc_dflags = dflags{ debugLevel = 0} }
withoutFlag corem =
liftIO =<< runCoreM <$> fmap removeFlag getHscEnv <*> getRuleBase <*>
getUniqMask <*> getModule <*>
getVisibleOrphanMods <*>
getPrintUnqualified <*> getSrcSpanM <*>
pure corem
let nukeTicks = stripTicksE (not . tickishIsCode)
nukeAnnotsBind :: CoreBind -> CoreBind
nukeAnnotsBind bind = case bind of
Rec bs -> Rec $ map (\(b,e) -> (b, nukeTicks e)) bs
NonRec b e -> NonRec b $ nukeTicks e
nukeAnnotsMod mg@ModGuts{mg_binds=binds}
= mg{mg_binds = map nukeAnnotsBind binds}
fmap fst $ withoutFlag $ pass (nukeAnnotsMod guts)