{-# LANGUAGE CPP #-}
{-# LANGUAGE DeriveFunctor #-}

module TcCanonical(
     canonicalize,
     unifyDerived,
     makeSuperClasses, maybeSym,
     StopOrContinue(..), stopWith, continueWith,
     solveCallStack    -- For TcSimplify
  ) where

#include "HsVersions.h"

import GhcPrelude

import Constraint
import Predicate
import TcOrigin
import TcUnify( swapOverTyVars, metaTyVarUpdateOK )
import TcType
import Type
import TcFlatten
import TcSMonad
import TcEvidence
import TcEvTerm
import Class
import TyCon
import TyCoRep   -- cleverly decomposes types, good for completeness checking
import Coercion
import CoreSyn
import Id( idType, mkTemplateLocals )
import FamInstEnv ( FamInstEnvs )
import FamInst ( tcTopNormaliseNewTypeTF_maybe )
import Var
import VarEnv( mkInScopeSet )
import VarSet( delVarSetList )
import Outputable
import DynFlags( DynFlags )
import NameSet
import RdrName
import GHC.Hs.Types( HsIPName(..) )

import Pair
import Util
import Bag
import MonadUtils
import Control.Monad
import Data.Maybe ( isJust )
import Data.List  ( zip4 )
import BasicTypes

import Data.Bifunctor ( bimap )
import Data.Foldable ( traverse_ )

{-
************************************************************************
*                                                                      *
*                      The Canonicaliser                               *
*                                                                      *
************************************************************************

Note [Canonicalization]
~~~~~~~~~~~~~~~~~~~~~~~

Canonicalization converts a simple constraint to a canonical form. It is
unary (i.e. treats individual constraints one at a time).

Constraints originating from user-written code come into being as
CNonCanonicals (except for CHoleCans, arising from holes). We know nothing
about these constraints. So, first:

     Classify CNonCanoncal constraints, depending on whether they
     are equalities, class predicates, or other.

Then proceed depending on the shape of the constraint. Generally speaking,
each constraint gets flattened and then decomposed into one of several forms
(see type Ct in TcRnTypes).

When an already-canonicalized constraint gets kicked out of the inert set,
it must be recanonicalized. But we know a bit about its shape from the
last time through, so we can skip the classification step.

-}

-- Top-level canonicalization
-- ~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~

canonicalize :: Ct -> TcS (StopOrContinue Ct)
canonicalize :: Ct -> TcS (StopOrContinue Ct)
canonicalize (CNonCanonical { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev })
  = {-# SCC "canNC" #-}
    case PredType -> Pred
classifyPredType PredType
pred of
      ClassPred Class
cls [PredType]
tys     -> do String -> SDoc -> TcS ()
traceTcS String
"canEvNC:cls" (Class -> SDoc
forall a. Outputable a => a -> SDoc
ppr Class
cls SDoc -> SDoc -> SDoc
<+> [PredType] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [PredType]
tys)
                                  CtEvidence -> Class -> [PredType] -> TcS (StopOrContinue Ct)
canClassNC CtEvidence
ev Class
cls [PredType]
tys
      EqPred EqRel
eq_rel PredType
ty1 PredType
ty2 -> do String -> SDoc -> TcS ()
traceTcS String
"canEvNC:eq" (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty1 SDoc -> SDoc -> SDoc
$$ PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty2)
                                  CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqNC    CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ty2
      IrredPred {}          -> do String -> SDoc -> TcS ()
traceTcS String
"canEvNC:irred" (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
pred)
                                  CtEvidence -> TcS (StopOrContinue Ct)
canIrred CtEvidence
ev
      ForAllPred [TyCoVarBinder]
_ [PredType]
_ PredType
pred   -> do String -> SDoc -> TcS ()
traceTcS String
"canEvNC:forall" (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
pred)
                                  CtEvidence -> Bool -> TcS (StopOrContinue Ct)
canForAll CtEvidence
ev (PredType -> Bool
isClassPred PredType
pred)
  where
    pred :: PredType
pred = CtEvidence -> PredType
ctEvPred CtEvidence
ev

canonicalize (CQuantCan (QCI { qci_ev :: QCInst -> CtEvidence
qci_ev = CtEvidence
ev, qci_pend_sc :: QCInst -> Bool
qci_pend_sc = Bool
pend_sc }))
  = CtEvidence -> Bool -> TcS (StopOrContinue Ct)
canForAll CtEvidence
ev Bool
pend_sc

canonicalize (CIrredCan { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev })
  | EqPred EqRel
eq_rel PredType
ty1 PredType
ty2 <- PredType -> Pred
classifyPredType (CtEvidence -> PredType
ctEvPred CtEvidence
ev)
  = -- For insolubles (all of which are equalities, do /not/ flatten the arguments
    -- In #14350 doing so led entire-unnecessary and ridiculously large
    -- type function expansion.  Instead, canEqNC just applies
    -- the substitution to the predicate, and may do decomposition;
    --    e.g. a ~ [a], where [G] a ~ [Int], can decompose
    CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqNC CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ty2

  | Bool
otherwise
  = CtEvidence -> TcS (StopOrContinue Ct)
canIrred CtEvidence
ev

canonicalize (CDictCan { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev, cc_class :: Ct -> Class
cc_class  = Class
cls
                       , cc_tyargs :: Ct -> [PredType]
cc_tyargs = [PredType]
xis, cc_pend_sc :: Ct -> Bool
cc_pend_sc = Bool
pend_sc })
  = {-# SCC "canClass" #-}
    CtEvidence
-> Class -> [PredType] -> Bool -> TcS (StopOrContinue Ct)
canClass CtEvidence
ev Class
cls [PredType]
xis Bool
pend_sc

canonicalize (CTyEqCan { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev
                       , cc_tyvar :: Ct -> TcTyVar
cc_tyvar  = TcTyVar
tv
                       , cc_rhs :: Ct -> PredType
cc_rhs    = PredType
xi
                       , cc_eq_rel :: Ct -> EqRel
cc_eq_rel = EqRel
eq_rel })
  = {-# SCC "canEqLeafTyVarEq" #-}
    CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqNC CtEvidence
ev EqRel
eq_rel (TcTyVar -> PredType
mkTyVarTy TcTyVar
tv) PredType
xi
      -- NB: Don't use canEqTyVar because that expects flattened types,
      -- and tv and xi may not be flat w.r.t. an updated inert set

canonicalize (CFunEqCan { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev
                        , cc_fun :: Ct -> TyCon
cc_fun    = TyCon
fn
                        , cc_tyargs :: Ct -> [PredType]
cc_tyargs = [PredType]
xis1
                        , cc_fsk :: Ct -> TcTyVar
cc_fsk    = TcTyVar
fsk })
  = {-# SCC "canEqLeafFunEq" #-}
    CtEvidence
-> TyCon -> [PredType] -> TcTyVar -> TcS (StopOrContinue Ct)
canCFunEqCan CtEvidence
ev TyCon
fn [PredType]
xis1 TcTyVar
fsk

canonicalize (CHoleCan { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev, cc_hole :: Ct -> Hole
cc_hole = Hole
hole })
  = CtEvidence -> Hole -> TcS (StopOrContinue Ct)
canHole CtEvidence
ev Hole
hole

{-
************************************************************************
*                                                                      *
*                      Class Canonicalization
*                                                                      *
************************************************************************
-}

canClassNC :: CtEvidence -> Class -> [Type] -> TcS (StopOrContinue Ct)
-- "NC" means "non-canonical"; that is, we have got here
-- from a NonCanonical constraint, not from a CDictCan
-- Precondition: EvVar is class evidence
canClassNC :: CtEvidence -> Class -> [PredType] -> TcS (StopOrContinue Ct)
canClassNC CtEvidence
ev Class
cls [PredType]
tys
  | CtEvidence -> Bool
isGiven CtEvidence
ev  -- See Note [Eagerly expand given superclasses]
  = do { [Ct]
sc_cts <- CtEvidence
-> [TcTyVar] -> [PredType] -> Class -> [PredType] -> TcS [Ct]
mkStrictSuperClasses CtEvidence
ev [] [] Class
cls [PredType]
tys
       ; [Ct] -> TcS ()
emitWork [Ct]
sc_cts
       ; CtEvidence
-> Class -> [PredType] -> Bool -> TcS (StopOrContinue Ct)
canClass CtEvidence
ev Class
cls [PredType]
tys Bool
False }

  | CtEvidence -> Bool
isWanted CtEvidence
ev
  , Just FastString
ip_name <- Class -> [PredType] -> Maybe FastString
isCallStackPred Class
cls [PredType]
tys
  , OccurrenceOf Name
func <- CtLoc -> CtOrigin
ctLocOrigin CtLoc
loc
  -- If we're given a CallStack constraint that arose from a function
  -- call, we need to push the current call-site onto the stack instead
  -- of solving it directly from a given.
  -- See Note [Overview of implicit CallStacks] in TcEvidence
  -- and Note [Solving CallStack constraints] in TcSMonad
  = do { -- First we emit a new constraint that will capture the
         -- given CallStack.
       ; let new_loc :: CtLoc
new_loc = CtLoc -> CtOrigin -> CtLoc
setCtLocOrigin CtLoc
loc (HsIPName -> CtOrigin
IPOccOrigin (FastString -> HsIPName
HsIPName FastString
ip_name))
                            -- We change the origin to IPOccOrigin so
                            -- this rule does not fire again.
                            -- See Note [Overview of implicit CallStacks]

       ; CtEvidence
new_ev <- CtLoc -> PredType -> TcS CtEvidence
newWantedEvVarNC CtLoc
new_loc PredType
pred

         -- Then we solve the wanted by pushing the call-site
         -- onto the newly emitted CallStack
       ; let ev_cs :: EvCallStack
ev_cs = Name -> RealSrcSpan -> EvExpr -> EvCallStack
EvCsPushCall Name
func (CtLoc -> RealSrcSpan
ctLocSpan CtLoc
loc) (CtEvidence -> EvExpr
ctEvExpr CtEvidence
new_ev)
       ; CtEvidence -> EvCallStack -> TcS ()
solveCallStack CtEvidence
ev EvCallStack
ev_cs

       ; CtEvidence
-> Class -> [PredType] -> Bool -> TcS (StopOrContinue Ct)
canClass CtEvidence
new_ev Class
cls [PredType]
tys Bool
False }

  | Bool
otherwise
  = CtEvidence
-> Class -> [PredType] -> Bool -> TcS (StopOrContinue Ct)
canClass CtEvidence
ev Class
cls [PredType]
tys (Class -> Bool
has_scs Class
cls)

  where
    has_scs :: Class -> Bool
has_scs Class
cls = Bool -> Bool
not ([PredType] -> Bool
forall (t :: * -> *) a. Foldable t => t a -> Bool
null (Class -> [PredType]
classSCTheta Class
cls))
    loc :: CtLoc
loc  = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev
    pred :: PredType
pred = CtEvidence -> PredType
ctEvPred CtEvidence
ev

solveCallStack :: CtEvidence -> EvCallStack -> TcS ()
-- Also called from TcSimplify when defaulting call stacks
solveCallStack :: CtEvidence -> EvCallStack -> TcS ()
solveCallStack CtEvidence
ev EvCallStack
ev_cs = do
  -- We're given ev_cs :: CallStack, but the evidence term should be a
  -- dictionary, so we have to coerce ev_cs to a dictionary for
  -- `IP ip CallStack`. See Note [Overview of implicit CallStacks]
  EvExpr
cs_tm <- EvCallStack -> TcS EvExpr
forall (m :: * -> *).
(MonadThings m, HasModule m, HasDynFlags m) =>
EvCallStack -> m EvExpr
evCallStack EvCallStack
ev_cs
  let ev_tm :: EvTerm
ev_tm = EvExpr -> TcCoercion -> EvTerm
mkEvCast EvExpr
cs_tm (PredType -> TcCoercion
wrapIP (CtEvidence -> PredType
ctEvPred CtEvidence
ev))
  CtEvidence -> EvTerm -> TcS ()
setEvBindIfWanted CtEvidence
ev EvTerm
ev_tm

canClass :: CtEvidence
         -> Class -> [Type]
         -> Bool            -- True <=> un-explored superclasses
         -> TcS (StopOrContinue Ct)
-- Precondition: EvVar is class evidence

canClass :: CtEvidence
-> Class -> [PredType] -> Bool -> TcS (StopOrContinue Ct)
canClass CtEvidence
ev Class
cls [PredType]
tys Bool
pend_sc
  =   -- all classes do *nominal* matching
    ASSERT2( ctEvRole ev == Nominal, ppr ev $$ ppr cls $$ ppr tys )
    do { ([PredType]
xis, [TcCoercion]
cos, TcCoercion
_kind_co) <- CtEvidence
-> TyCon
-> [PredType]
-> TcS ([PredType], [TcCoercion], TcCoercion)
flattenArgsNom CtEvidence
ev TyCon
cls_tc [PredType]
tys
       ; MASSERT( isTcReflCo _kind_co )
       ; let co :: TcCoercion
co = Role -> TyCon -> [TcCoercion] -> TcCoercion
mkTcTyConAppCo Role
Nominal TyCon
cls_tc [TcCoercion]
cos
             xi :: PredType
xi = Class -> [PredType] -> PredType
mkClassPred Class
cls [PredType]
xis
             mk_ct :: CtEvidence -> Ct
mk_ct CtEvidence
new_ev = CDictCan :: CtEvidence -> Class -> [PredType] -> Bool -> Ct
CDictCan { cc_ev :: CtEvidence
cc_ev = CtEvidence
new_ev
                                     , cc_tyargs :: [PredType]
cc_tyargs = [PredType]
xis
                                     , cc_class :: Class
cc_class = Class
cls
                                     , cc_pend_sc :: Bool
cc_pend_sc = Bool
pend_sc }
       ; StopOrContinue CtEvidence
mb <- CtEvidence
-> PredType -> TcCoercion -> TcS (StopOrContinue CtEvidence)
rewriteEvidence CtEvidence
ev PredType
xi TcCoercion
co
       ; String -> SDoc -> TcS ()
traceTcS String
"canClass" ([SDoc] -> SDoc
vcat [ CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev
                                   , PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
xi, StopOrContinue CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr StopOrContinue CtEvidence
mb ])
       ; StopOrContinue Ct -> TcS (StopOrContinue Ct)
forall (m :: * -> *) a. Monad m => a -> m a
return ((CtEvidence -> Ct)
-> StopOrContinue CtEvidence -> StopOrContinue Ct
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap CtEvidence -> Ct
mk_ct StopOrContinue CtEvidence
mb) }
  where
    cls_tc :: TyCon
cls_tc = Class -> TyCon
classTyCon Class
cls

{- Note [The superclass story]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
We need to add superclass constraints for two reasons:

* For givens [G], they give us a route to proof.  E.g.
    f :: Ord a => a -> Bool
    f x = x == x
  We get a Wanted (Eq a), which can only be solved from the superclass
  of the Given (Ord a).

* For wanteds [W], and deriveds [WD], [D], they may give useful
  functional dependencies.  E.g.
     class C a b | a -> b where ...
     class C a b => D a b where ...
  Now a [W] constraint (D Int beta) has (C Int beta) as a superclass
  and that might tell us about beta, via C's fundeps.  We can get this
  by generating a [D] (C Int beta) constraint.  It's derived because
  we don't actually have to cough up any evidence for it; it's only there
  to generate fundep equalities.

See Note [Why adding superclasses can help].

For these reasons we want to generate superclass constraints for both
Givens and Wanteds. But:

* (Minor) they are often not needed, so generating them aggressively
  is a waste of time.

* (Major) if we want recursive superclasses, there would be an infinite
  number of them.  Here is a real-life example (#10318);

     class (Frac (Frac a) ~ Frac a,
            Fractional (Frac a),
            IntegralDomain (Frac a))
         => IntegralDomain a where
      type Frac a :: *

  Notice that IntegralDomain has an associated type Frac, and one
  of IntegralDomain's superclasses is another IntegralDomain constraint.

So here's the plan:

1. Eagerly generate superclasses for given (but not wanted)
   constraints; see Note [Eagerly expand given superclasses].
   This is done using mkStrictSuperClasses in canClassNC, when
   we take a non-canonical Given constraint and cannonicalise it.

   However stop if you encounter the same class twice.  That is,
   mkStrictSuperClasses expands eagerly, but has a conservative
   termination condition: see Note [Expanding superclasses] in TcType.

2. Solve the wanteds as usual, but do no further expansion of
   superclasses for canonical CDictCans in solveSimpleGivens or
   solveSimpleWanteds; Note [Danger of adding superclasses during solving]

   However, /do/ continue to eagerly expand superlasses for new /given/
   /non-canonical/ constraints (canClassNC does this).  As #12175
   showed, a type-family application can expand to a class constraint,
   and we want to see its superclasses for just the same reason as
   Note [Eagerly expand given superclasses].

3. If we have any remaining unsolved wanteds
        (see Note [When superclasses help] in Constraint)
   try harder: take both the Givens and Wanteds, and expand
   superclasses again.  See the calls to expandSuperClasses in
   TcSimplify.simpl_loop and solveWanteds.

   This may succeed in generating (a finite number of) extra Givens,
   and extra Deriveds. Both may help the proof.

3a An important wrinkle: only expand Givens from the current level.
   Two reasons:
      - We only want to expand it once, and that is best done at
        the level it is bound, rather than repeatedly at the leaves
        of the implication tree
      - We may be inside a type where we can't create term-level
        evidence anyway, so we can't superclass-expand, say,
        (a ~ b) to get (a ~# b).  This happened in #15290.

4. Go round to (2) again.  This loop (2,3,4) is implemented
   in TcSimplify.simpl_loop.

The cc_pend_sc flag in a CDictCan records whether the superclasses of
this constraint have been expanded.  Specifically, in Step 3 we only
expand superclasses for constraints with cc_pend_sc set to true (i.e.
isPendingScDict holds).

Why do we do this?  Two reasons:

* To avoid repeated work, by repeatedly expanding the superclasses of
  same constraint,

* To terminate the above loop, at least in the -XNoRecursiveSuperClasses
  case.  If there are recursive superclasses we could, in principle,
  expand forever, always encountering new constraints.

When we take a CNonCanonical or CIrredCan, but end up classifying it
as a CDictCan, we set the cc_pend_sc flag to False.

Note [Superclass loops]
~~~~~~~~~~~~~~~~~~~~~~~
Suppose we have
  class C a => D a
  class D a => C a

Then, when we expand superclasses, we'll get back to the self-same
predicate, so we have reached a fixpoint in expansion and there is no
point in fruitlessly expanding further.  This case just falls out from
our strategy.  Consider
  f :: C a => a -> Bool
  f x = x==x
Then canClassNC gets the [G] d1: C a constraint, and eager emits superclasses
G] d2: D a, [G] d3: C a (psc).  (The "psc" means it has its sc_pend flag set.)
When processing d3 we find a match with d1 in the inert set, and we always
keep the inert item (d1) if possible: see Note [Replacement vs keeping] in
TcInteract.  So d3 dies a quick, happy death.

Note [Eagerly expand given superclasses]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
In step (1) of Note [The superclass story], why do we eagerly expand
Given superclasses by one layer?  (By "one layer" we mean expand transitively
until you meet the same class again -- the conservative criterion embodied
in expandSuperClasses.  So a "layer" might be a whole stack of superclasses.)
We do this eagerly for Givens mainly because of some very obscure
cases like this:

   instance Bad a => Eq (T a)

   f :: (Ord (T a)) => blah
   f x = ....needs Eq (T a), Ord (T a)....

Here if we can't satisfy (Eq (T a)) from the givens we'll use the
instance declaration; but then we are stuck with (Bad a).  Sigh.
This is really a case of non-confluent proofs, but to stop our users
complaining we expand one layer in advance.

Note [Instance and Given overlap] in TcInteract.

We also want to do this if we have

   f :: F (T a) => blah

where
   type instance F (T a) = Ord (T a)

So we may need to do a little work on the givens to expose the
class that has the superclasses.  That's why the superclass
expansion for Givens happens in canClassNC.

Note [Why adding superclasses can help]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Examples of how adding superclasses can help:

    --- Example 1
        class C a b | a -> b
    Suppose we want to solve
         [G] C a b
         [W] C a beta
    Then adding [D] beta~b will let us solve it.

    -- Example 2 (similar but using a type-equality superclass)
        class (F a ~ b) => C a b
    And try to sllve:
         [G] C a b
         [W] C a beta
    Follow the superclass rules to add
         [G] F a ~ b
         [D] F a ~ beta
    Now we get [D] beta ~ b, and can solve that.

    -- Example (tcfail138)
      class L a b | a -> b
      class (G a, L a b) => C a b

      instance C a b' => G (Maybe a)
      instance C a b  => C (Maybe a) a
      instance L (Maybe a) a

    When solving the superclasses of the (C (Maybe a) a) instance, we get
      [G] C a b, and hance by superclasses, [G] G a, [G] L a b
      [W] G (Maybe a)
    Use the instance decl to get
      [W] C a beta
    Generate its derived superclass
      [D] L a beta.  Now using fundeps, combine with [G] L a b to get
      [D] beta ~ b
    which is what we want.

Note [Danger of adding superclasses during solving]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Here's a serious, but now out-dated example, from #4497:

   class Num (RealOf t) => Normed t
   type family RealOf x

Assume the generated wanted constraint is:
   [W] RealOf e ~ e
   [W] Normed e

If we were to be adding the superclasses during simplification we'd get:
   [W] RealOf e ~ e
   [W] Normed e
   [D] RealOf e ~ fuv
   [D] Num fuv
==>
   e := fuv, Num fuv, Normed fuv, RealOf fuv ~ fuv

While looks exactly like our original constraint. If we add the
superclass of (Normed fuv) again we'd loop.  By adding superclasses
definitely only once, during canonicalisation, this situation can't
happen.

Mind you, now that Wanteds cannot rewrite Derived, I think this particular
situation can't happen.
  -}

makeSuperClasses :: [Ct] -> TcS [Ct]
-- Returns strict superclasses, transitively, see Note [The superclasses story]
-- See Note [The superclass story]
-- The loop-breaking here follows Note [Expanding superclasses] in TcType
-- Specifically, for an incoming (C t) constraint, we return all of (C t)'s
--    superclasses, up to /and including/ the first repetition of C
--
-- Example:  class D a => C a
--           class C [a] => D a
-- makeSuperClasses (C x) will return (D x, C [x])
--
-- NB: the incoming constraints have had their cc_pend_sc flag already
--     flipped to False, by isPendingScDict, so we are /obliged/ to at
--     least produce the immediate superclasses
makeSuperClasses :: [Ct] -> TcS [Ct]
makeSuperClasses [Ct]
cts = (Ct -> TcS [Ct]) -> [Ct] -> TcS [Ct]
forall (m :: * -> *) a b. Monad m => (a -> m [b]) -> [a] -> m [b]
concatMapM Ct -> TcS [Ct]
go [Ct]
cts
  where
    go :: Ct -> TcS [Ct]
go (CDictCan { cc_ev :: Ct -> CtEvidence
cc_ev = CtEvidence
ev, cc_class :: Ct -> Class
cc_class = Class
cls, cc_tyargs :: Ct -> [PredType]
cc_tyargs = [PredType]
tys })
      = CtEvidence
-> [TcTyVar] -> [PredType] -> Class -> [PredType] -> TcS [Ct]
mkStrictSuperClasses CtEvidence
ev [] [] Class
cls [PredType]
tys
    go (CQuantCan (QCI { qci_pred :: QCInst -> PredType
qci_pred = PredType
pred, qci_ev :: QCInst -> CtEvidence
qci_ev = CtEvidence
ev }))
      = ASSERT2( isClassPred pred, ppr pred )  -- The cts should all have
                                               -- class pred heads
        CtEvidence
-> [TcTyVar] -> [PredType] -> Class -> [PredType] -> TcS [Ct]
mkStrictSuperClasses CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys
      where
        ([TcTyVar]
tvs, [PredType]
theta, Class
cls, [PredType]
tys) = PredType -> ([TcTyVar], [PredType], Class, [PredType])
tcSplitDFunTy (CtEvidence -> PredType
ctEvPred CtEvidence
ev)
    go Ct
ct = String -> SDoc -> TcS [Ct]
forall a. HasCallStack => String -> SDoc -> a
pprPanic String
"makeSuperClasses" (Ct -> SDoc
forall a. Outputable a => a -> SDoc
ppr Ct
ct)

mkStrictSuperClasses
    :: CtEvidence
    -> [TyVar] -> ThetaType  -- These two args are non-empty only when taking
                             -- superclasses of a /quantified/ constraint
    -> Class -> [Type] -> TcS [Ct]
-- Return constraints for the strict superclasses of
--   ev :: forall as. theta => cls tys
mkStrictSuperClasses :: CtEvidence
-> [TcTyVar] -> [PredType] -> Class -> [PredType] -> TcS [Ct]
mkStrictSuperClasses CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys
  = NameSet
-> CtEvidence
-> [TcTyVar]
-> [PredType]
-> Class
-> [PredType]
-> TcS [Ct]
mk_strict_superclasses (Name -> NameSet
unitNameSet (Class -> Name
className Class
cls))
                           CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys

mk_strict_superclasses :: NameSet -> CtEvidence
                       -> [TyVar] -> ThetaType
                       -> Class -> [Type] -> TcS [Ct]
-- Always return the immediate superclasses of (cls tys);
-- and expand their superclasses, provided none of them are in rec_clss
-- nor are repeated
mk_strict_superclasses :: NameSet
-> CtEvidence
-> [TcTyVar]
-> [PredType]
-> Class
-> [PredType]
-> TcS [Ct]
mk_strict_superclasses NameSet
rec_clss CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys
  | CtGiven { ctev_evar :: CtEvidence -> TcTyVar
ctev_evar = TcTyVar
evar, ctev_loc :: CtEvidence -> CtLoc
ctev_loc = CtLoc
loc } <- CtEvidence
ev
  = (TcTyVar -> TcS [Ct]) -> [TcTyVar] -> TcS [Ct]
forall (m :: * -> *) a b. Monad m => (a -> m [b]) -> [a] -> m [b]
concatMapM (TcTyVar -> CtLoc -> TcTyVar -> TcS [Ct]
do_one_given TcTyVar
evar (CtLoc -> CtLoc
mk_given_loc CtLoc
loc)) ([TcTyVar] -> TcS [Ct]) -> [TcTyVar] -> TcS [Ct]
forall a b. (a -> b) -> a -> b
$
    Class -> [TcTyVar]
classSCSelIds Class
cls
  where
    dict_ids :: [TcTyVar]
dict_ids  = [PredType] -> [TcTyVar]
mkTemplateLocals [PredType]
theta
    size :: TypeSize
size      = [PredType] -> TypeSize
sizeTypes [PredType]
tys

    do_one_given :: TcTyVar -> CtLoc -> TcTyVar -> TcS [Ct]
do_one_given TcTyVar
evar CtLoc
given_loc TcTyVar
sel_id
      | HasDebugCallStack => PredType -> Bool
PredType -> Bool
isUnliftedType PredType
sc_pred
      , Bool -> Bool
not ([TcTyVar] -> Bool
forall (t :: * -> *) a. Foldable t => t a -> Bool
null [TcTyVar]
tvs Bool -> Bool -> Bool
&& [PredType] -> Bool
forall (t :: * -> *) a. Foldable t => t a -> Bool
null [PredType]
theta)
      = -- See Note [Equality superclasses in quantified constraints]
        [Ct] -> TcS [Ct]
forall (m :: * -> *) a. Monad m => a -> m a
return []
      | Bool
otherwise
      = do { CtEvidence
given_ev <- CtLoc -> (PredType, EvTerm) -> TcS CtEvidence
newGivenEvVar CtLoc
given_loc ((PredType, EvTerm) -> TcS CtEvidence)
-> (PredType, EvTerm) -> TcS CtEvidence
forall a b. (a -> b) -> a -> b
$
                         (PredType
given_ty, TcTyVar -> TcTyVar -> EvTerm
mk_sc_sel TcTyVar
evar TcTyVar
sel_id)
           ; NameSet
-> CtEvidence -> [TcTyVar] -> [PredType] -> PredType -> TcS [Ct]
mk_superclasses NameSet
rec_clss CtEvidence
given_ev [TcTyVar]
tvs [PredType]
theta PredType
sc_pred }
      where
        sc_pred :: PredType
sc_pred  = PredType -> PredType
funResultTy (HasDebugCallStack => PredType -> [PredType] -> PredType
PredType -> [PredType] -> PredType
piResultTys (TcTyVar -> PredType
idType TcTyVar
sel_id) [PredType]
tys)
        given_ty :: PredType
given_ty = [TcTyVar] -> [PredType] -> PredType -> PredType
mkInfSigmaTy [TcTyVar]
tvs [PredType]
theta PredType
sc_pred

    mk_sc_sel :: TcTyVar -> TcTyVar -> EvTerm
mk_sc_sel TcTyVar
evar TcTyVar
sel_id
      = EvExpr -> EvTerm
EvExpr (EvExpr -> EvTerm) -> EvExpr -> EvTerm
forall a b. (a -> b) -> a -> b
$ [TcTyVar] -> EvExpr -> EvExpr
forall b. [b] -> Expr b -> Expr b
mkLams [TcTyVar]
tvs (EvExpr -> EvExpr) -> EvExpr -> EvExpr
forall a b. (a -> b) -> a -> b
$ [TcTyVar] -> EvExpr -> EvExpr
forall b. [b] -> Expr b -> Expr b
mkLams [TcTyVar]
dict_ids (EvExpr -> EvExpr) -> EvExpr -> EvExpr
forall a b. (a -> b) -> a -> b
$
        TcTyVar -> EvExpr
forall b. TcTyVar -> Expr b
Var TcTyVar
sel_id EvExpr -> [PredType] -> EvExpr
forall b. Expr b -> [PredType] -> Expr b
`mkTyApps` [PredType]
tys EvExpr -> EvExpr -> EvExpr
forall b. Expr b -> Expr b -> Expr b
`App`
        (TcTyVar -> EvExpr
evId TcTyVar
evar EvExpr -> [PredType] -> EvExpr
forall b. Expr b -> [PredType] -> Expr b
`mkTyApps` [TcTyVar] -> [PredType]
mkTyVarTys [TcTyVar]
tvs EvExpr -> [TcTyVar] -> EvExpr
forall b. Expr b -> [TcTyVar] -> Expr b
`mkVarApps` [TcTyVar]
dict_ids)

    mk_given_loc :: CtLoc -> CtLoc
mk_given_loc CtLoc
loc
       | Class -> Bool
isCTupleClass Class
cls
       = CtLoc
loc   -- For tuple predicates, just take them apart, without
               -- adding their (large) size into the chain.  When we
               -- get down to a base predicate, we'll include its size.
               -- #10335

       | GivenOrigin SkolemInfo
skol_info <- CtLoc -> CtOrigin
ctLocOrigin CtLoc
loc
         -- See Note [Solving superclass constraints] in TcInstDcls
         -- for explantation of this transformation for givens
       = case SkolemInfo
skol_info of
            SkolemInfo
InstSkol -> CtLoc
loc { ctl_origin :: CtOrigin
ctl_origin = SkolemInfo -> CtOrigin
GivenOrigin (TypeSize -> SkolemInfo
InstSC TypeSize
size) }
            InstSC TypeSize
n -> CtLoc
loc { ctl_origin :: CtOrigin
ctl_origin = SkolemInfo -> CtOrigin
GivenOrigin (TypeSize -> SkolemInfo
InstSC (TypeSize
n TypeSize -> TypeSize -> TypeSize
forall a. Ord a => a -> a -> a
`max` TypeSize
size)) }
            SkolemInfo
_        -> CtLoc
loc

       | Bool
otherwise  -- Probably doesn't happen, since this function
       = CtLoc
loc        -- is only used for Givens, but does no harm

mk_strict_superclasses NameSet
rec_clss CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys
  | (PredType -> Bool) -> [PredType] -> Bool
forall (t :: * -> *) a. Foldable t => (a -> Bool) -> t a -> Bool
all PredType -> Bool
noFreeVarsOfType [PredType]
tys
  = [Ct] -> TcS [Ct]
forall (m :: * -> *) a. Monad m => a -> m a
return [] -- Wanteds with no variables yield no deriveds.
              -- See Note [Improvement from Ground Wanteds]

  | Bool
otherwise -- Wanted/Derived case, just add Derived superclasses
              -- that can lead to improvement.
  = ASSERT2( null tvs && null theta, ppr tvs $$ ppr theta )
    (PredType -> TcS [Ct]) -> [PredType] -> TcS [Ct]
forall (m :: * -> *) a b. Monad m => (a -> m [b]) -> [a] -> m [b]
concatMapM PredType -> TcS [Ct]
do_one_derived (Class -> [PredType] -> [PredType]
immSuperClasses Class
cls [PredType]
tys)
  where
    loc :: CtLoc
loc = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev

    do_one_derived :: PredType -> TcS [Ct]
do_one_derived PredType
sc_pred
      = do { CtEvidence
sc_ev <- CtLoc -> PredType -> TcS CtEvidence
newDerivedNC CtLoc
loc PredType
sc_pred
           ; NameSet
-> CtEvidence -> [TcTyVar] -> [PredType] -> PredType -> TcS [Ct]
mk_superclasses NameSet
rec_clss CtEvidence
sc_ev [] [] PredType
sc_pred }

mk_superclasses :: NameSet -> CtEvidence
                -> [TyVar] -> ThetaType -> PredType -> TcS [Ct]
-- Return this constraint, plus its superclasses, if any
mk_superclasses :: NameSet
-> CtEvidence -> [TcTyVar] -> [PredType] -> PredType -> TcS [Ct]
mk_superclasses NameSet
rec_clss CtEvidence
ev [TcTyVar]
tvs [PredType]
theta PredType
pred
  | ClassPred Class
cls [PredType]
tys <- PredType -> Pred
classifyPredType PredType
pred
  = NameSet
-> CtEvidence
-> [TcTyVar]
-> [PredType]
-> Class
-> [PredType]
-> TcS [Ct]
mk_superclasses_of NameSet
rec_clss CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys

  | Bool
otherwise   -- Superclass is not a class predicate
  = [Ct] -> TcS [Ct]
forall (m :: * -> *) a. Monad m => a -> m a
return [CtEvidence -> Ct
mkNonCanonical CtEvidence
ev]

mk_superclasses_of :: NameSet -> CtEvidence
                   -> [TyVar] -> ThetaType -> Class -> [Type]
                   -> TcS [Ct]
-- Always return this class constraint,
-- and expand its superclasses
mk_superclasses_of :: NameSet
-> CtEvidence
-> [TcTyVar]
-> [PredType]
-> Class
-> [PredType]
-> TcS [Ct]
mk_superclasses_of NameSet
rec_clss CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys
  | Bool
loop_found = do { String -> SDoc -> TcS ()
traceTcS String
"mk_superclasses_of: loop" (Class -> SDoc
forall a. Outputable a => a -> SDoc
ppr Class
cls SDoc -> SDoc -> SDoc
<+> [PredType] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [PredType]
tys)
                    ; [Ct] -> TcS [Ct]
forall (m :: * -> *) a. Monad m => a -> m a
return [Ct
this_ct] }  -- cc_pend_sc of this_ct = True
  | Bool
otherwise  = do { String -> SDoc -> TcS ()
traceTcS String
"mk_superclasses_of" ([SDoc] -> SDoc
vcat [ Class -> SDoc
forall a. Outputable a => a -> SDoc
ppr Class
cls SDoc -> SDoc -> SDoc
<+> [PredType] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [PredType]
tys
                                                          , Bool -> SDoc
forall a. Outputable a => a -> SDoc
ppr (Class -> Bool
isCTupleClass Class
cls)
                                                          , NameSet -> SDoc
forall a. Outputable a => a -> SDoc
ppr NameSet
rec_clss
                                                          ])
                    ; [Ct]
sc_cts <- NameSet
-> CtEvidence
-> [TcTyVar]
-> [PredType]
-> Class
-> [PredType]
-> TcS [Ct]
mk_strict_superclasses NameSet
rec_clss' CtEvidence
ev [TcTyVar]
tvs [PredType]
theta Class
cls [PredType]
tys
                    ; [Ct] -> TcS [Ct]
forall (m :: * -> *) a. Monad m => a -> m a
return (Ct
this_ct Ct -> [Ct] -> [Ct]
forall a. a -> [a] -> [a]
: [Ct]
sc_cts) }
                                   -- cc_pend_sc of this_ct = False
  where
    cls_nm :: Name
cls_nm     = Class -> Name
className Class
cls
    loop_found :: Bool
loop_found = Bool -> Bool
not (Class -> Bool
isCTupleClass Class
cls) Bool -> Bool -> Bool
&& Name
cls_nm Name -> NameSet -> Bool
`elemNameSet` NameSet
rec_clss
                 -- Tuples never contribute to recursion, and can be nested
    rec_clss' :: NameSet
rec_clss'  = NameSet
rec_clss NameSet -> Name -> NameSet
`extendNameSet` Name
cls_nm

    this_ct :: Ct
this_ct | [TcTyVar] -> Bool
forall (t :: * -> *) a. Foldable t => t a -> Bool
null [TcTyVar]
tvs, [PredType] -> Bool
forall (t :: * -> *) a. Foldable t => t a -> Bool
null [PredType]
theta
            = CDictCan :: CtEvidence -> Class -> [PredType] -> Bool -> Ct
CDictCan { cc_ev :: CtEvidence
cc_ev = CtEvidence
ev, cc_class :: Class
cc_class = Class
cls, cc_tyargs :: [PredType]
cc_tyargs = [PredType]
tys
                       , cc_pend_sc :: Bool
cc_pend_sc = Bool
loop_found }
                 -- NB: If there is a loop, we cut off, so we have not
                 --     added the superclasses, hence cc_pend_sc = True
            | Bool
otherwise
            = QCInst -> Ct
CQuantCan (QCI :: CtEvidence -> [TcTyVar] -> PredType -> Bool -> QCInst
QCI { qci_tvs :: [TcTyVar]
qci_tvs = [TcTyVar]
tvs, qci_pred :: PredType
qci_pred = Class -> [PredType] -> PredType
mkClassPred Class
cls [PredType]
tys
                             , qci_ev :: CtEvidence
qci_ev = CtEvidence
ev
                             , qci_pend_sc :: Bool
qci_pend_sc = Bool
loop_found })


{- Note [Equality superclasses in quantified constraints]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Consider (#15359, #15593, #15625)
  f :: (forall a. theta => a ~ b) => stuff

It's a bit odd to have a local, quantified constraint for `(a~b)`,
but some people want such a thing (see the tickets). And for
Coercible it is definitely useful
  f :: forall m. (forall p q. Coercible p q => Coercible (m p) (m q)))
                 => stuff

Moreover it's not hard to arrange; we just need to look up /equality/
constraints in the quantified-constraint environment, which we do in
TcInteract.doTopReactOther.

There is a wrinkle though, in the case where 'theta' is empty, so
we have
  f :: (forall a. a~b) => stuff

Now, potentially, the superclass machinery kicks in, in
makeSuperClasses, giving us a a second quantified constrait
       (forall a. a ~# b)
BUT this is an unboxed value!  And nothing has prepared us for
dictionary "functions" that are unboxed.  Actually it does just
about work, but the simplier ends up with stuff like
   case (/\a. eq_sel d) of df -> ...(df @Int)...
and fails to simplify that any further.  And it doesn't satisfy
isPredTy any more.

So for now we simply decline to take superclasses in the quantified
case.  Instead we have a special case in TcInteract.doTopReactOther,
which looks for primitive equalities specially in the quantified
constraints.

See also Note [Evidence for quantified constraints] in Predicate.


************************************************************************
*                                                                      *
*                      Irreducibles canonicalization
*                                                                      *
************************************************************************
-}

canIrred :: CtEvidence -> TcS (StopOrContinue Ct)
-- Precondition: ty not a tuple and no other evidence form
canIrred :: CtEvidence -> TcS (StopOrContinue Ct)
canIrred CtEvidence
ev
  = do { let pred :: PredType
pred = CtEvidence -> PredType
ctEvPred CtEvidence
ev
       ; String -> SDoc -> TcS ()
traceTcS String
"can_pred" (String -> SDoc
text String
"IrredPred = " SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
pred)
       ; (PredType
xi,TcCoercion
co) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_FlattenAll CtEvidence
ev PredType
pred -- co :: xi ~ pred
       ; CtEvidence
-> PredType -> TcCoercion -> TcS (StopOrContinue CtEvidence)
rewriteEvidence CtEvidence
ev PredType
xi TcCoercion
co TcS (StopOrContinue CtEvidence)
-> (CtEvidence -> TcS (StopOrContinue Ct))
-> TcS (StopOrContinue Ct)
forall a b.
TcS (StopOrContinue a)
-> (a -> TcS (StopOrContinue b)) -> TcS (StopOrContinue b)
`andWhenContinue` \ CtEvidence
new_ev ->
    do { -- Re-classify, in case flattening has improved its shape
       ; case PredType -> Pred
classifyPredType (CtEvidence -> PredType
ctEvPred CtEvidence
new_ev) of
           ClassPred Class
cls [PredType]
tys     -> CtEvidence -> Class -> [PredType] -> TcS (StopOrContinue Ct)
canClassNC CtEvidence
new_ev Class
cls [PredType]
tys
           EqPred EqRel
eq_rel PredType
ty1 PredType
ty2 -> CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqNC CtEvidence
new_ev EqRel
eq_rel PredType
ty1 PredType
ty2
           Pred
_                     -> Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (Ct -> TcS (StopOrContinue Ct)) -> Ct -> TcS (StopOrContinue Ct)
forall a b. (a -> b) -> a -> b
$
                                    CtEvidence -> Ct
mkIrredCt CtEvidence
new_ev } }

canHole :: CtEvidence -> Hole -> TcS (StopOrContinue Ct)
canHole :: CtEvidence -> Hole -> TcS (StopOrContinue Ct)
canHole CtEvidence
ev Hole
hole
  = do { let pred :: PredType
pred = CtEvidence -> PredType
ctEvPred CtEvidence
ev
       ; (PredType
xi,TcCoercion
co) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_SubstOnly CtEvidence
ev PredType
pred -- co :: xi ~ pred
       ; CtEvidence
-> PredType -> TcCoercion -> TcS (StopOrContinue CtEvidence)
rewriteEvidence CtEvidence
ev PredType
xi TcCoercion
co TcS (StopOrContinue CtEvidence)
-> (CtEvidence -> TcS (StopOrContinue Ct))
-> TcS (StopOrContinue Ct)
forall a b.
TcS (StopOrContinue a)
-> (a -> TcS (StopOrContinue b)) -> TcS (StopOrContinue b)
`andWhenContinue` \ CtEvidence
new_ev ->
    do { (Cts -> Cts) -> TcS ()
updInertIrreds (Cts -> Ct -> Cts
`snocCts` (CHoleCan :: CtEvidence -> Hole -> Ct
CHoleCan { cc_ev :: CtEvidence
cc_ev = CtEvidence
new_ev
                                             , cc_hole :: Hole
cc_hole = Hole
hole }))
       ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
new_ev String
"Emit insoluble hole" } }


{- *********************************************************************
*                                                                      *
*                      Quantified predicates
*                                                                      *
********************************************************************* -}

{- Note [Quantified constraints]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
The -XQuantifiedConstraints extension allows type-class contexts like this:

  data Rose f x = Rose x (f (Rose f x))

  instance (Eq a, forall b. Eq b => Eq (f b))
        => Eq (Rose f a)  where
    (Rose x1 rs1) == (Rose x2 rs2) = x1==x2 && rs1 == rs2

Note the (forall b. Eq b => Eq (f b)) in the instance contexts.
This quantified constraint is needed to solve the
 [W] (Eq (f (Rose f x)))
constraint which arises form the (==) definition.

The wiki page is
  https://gitlab.haskell.org/ghc/ghc/wikis/quantified-constraints
which in turn contains a link to the GHC Proposal where the change
is specified, and a Haskell Symposium paper about it.

We implement two main extensions to the design in the paper:

 1. We allow a variable in the instance head, e.g.
      f :: forall m a. (forall b. m b) => D (m a)
    Notice the 'm' in the head of the quantified constraint, not
    a class.

 2. We suport superclasses to quantified constraints.
    For example (contrived):
      f :: (Ord b, forall b. Ord b => Ord (m b)) => m a -> m a -> Bool
      f x y = x==y
    Here we need (Eq (m a)); but the quantifed constraint deals only
    with Ord.  But we can make it work by using its superclass.

Here are the moving parts
  * Language extension {-# LANGUAGE QuantifiedConstraints #-}
    and add it to ghc-boot-th:GHC.LanguageExtensions.Type.Extension

  * A new form of evidence, EvDFun, that is used to discharge
    such wanted constraints

  * checkValidType gets some changes to accept forall-constraints
    only in the right places.

  * Predicate.Pred gets a new constructor ForAllPred, and
    and classifyPredType analyses a PredType to decompose
    the new forall-constraints

  * TcSMonad.InertCans gets an extra field, inert_insts,
    which holds all the Given forall-constraints.  In effect,
    such Given constraints are like local instance decls.

  * When trying to solve a class constraint, via
    TcInteract.matchInstEnv, use the InstEnv from inert_insts
    so that we include the local Given forall-constraints
    in the lookup.  (See TcSMonad.getInstEnvs.)

  * TcCanonical.canForAll deals with solving a
    forall-constraint.  See
       Note [Solving a Wanted forall-constraint]

  * We augment the kick-out code to kick out an inert
    forall constraint if it can be rewritten by a new
    type equality; see TcSMonad.kick_out_rewritable

Note that a quantified constraint is never /inferred/
(by TcSimplify.simplifyInfer).  A function can only have a
quantified constraint in its type if it is given an explicit
type signature.

Note that we implement
-}

canForAll :: CtEvidence -> Bool -> TcS (StopOrContinue Ct)
-- We have a constraint (forall as. blah => C tys)
canForAll :: CtEvidence -> Bool -> TcS (StopOrContinue Ct)
canForAll CtEvidence
ev Bool
pend_sc
  = do { -- First rewrite it to apply the current substitution
         -- Do not bother with type-family reductions; we can't
         -- do them under a forall anyway (c.f. Flatten.flatten_one
         -- on a forall type)
         let pred :: PredType
pred = CtEvidence -> PredType
ctEvPred CtEvidence
ev
       ; (PredType
xi,TcCoercion
co) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_SubstOnly CtEvidence
ev PredType
pred -- co :: xi ~ pred
       ; CtEvidence
-> PredType -> TcCoercion -> TcS (StopOrContinue CtEvidence)
rewriteEvidence CtEvidence
ev PredType
xi TcCoercion
co TcS (StopOrContinue CtEvidence)
-> (CtEvidence -> TcS (StopOrContinue Ct))
-> TcS (StopOrContinue Ct)
forall a b.
TcS (StopOrContinue a)
-> (a -> TcS (StopOrContinue b)) -> TcS (StopOrContinue b)
`andWhenContinue` \ CtEvidence
new_ev ->

    do { -- Now decompose into its pieces and solve it
         -- (It takes a lot less code to flatten before decomposing.)
       ; case PredType -> Pred
classifyPredType (CtEvidence -> PredType
ctEvPred CtEvidence
new_ev) of
           ForAllPred [TyCoVarBinder]
tv_bndrs [PredType]
theta PredType
pred
              -> CtEvidence
-> [TyCoVarBinder]
-> [PredType]
-> PredType
-> Bool
-> TcS (StopOrContinue Ct)
solveForAll CtEvidence
new_ev [TyCoVarBinder]
tv_bndrs [PredType]
theta PredType
pred Bool
pend_sc
           Pred
_  -> String -> SDoc -> TcS (StopOrContinue Ct)
forall a. HasCallStack => String -> SDoc -> a
pprPanic String
"canForAll" (CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
new_ev)
    } }

solveForAll :: CtEvidence -> [TyVarBinder] -> TcThetaType -> PredType -> Bool
            -> TcS (StopOrContinue Ct)
solveForAll :: CtEvidence
-> [TyCoVarBinder]
-> [PredType]
-> PredType
-> Bool
-> TcS (StopOrContinue Ct)
solveForAll CtEvidence
ev [TyCoVarBinder]
tv_bndrs [PredType]
theta PredType
pred Bool
pend_sc
  | CtWanted { ctev_dest :: CtEvidence -> TcEvDest
ctev_dest = TcEvDest
dest } <- CtEvidence
ev
  = -- See Note [Solving a Wanted forall-constraint]
    do { let skol_info :: SkolemInfo
skol_info = SkolemInfo
QuantCtxtSkol
             empty_subst :: TCvSubst
empty_subst = InScopeSet -> TCvSubst
mkEmptyTCvSubst (InScopeSet -> TCvSubst) -> InScopeSet -> TCvSubst
forall a b. (a -> b) -> a -> b
$ VarSet -> InScopeSet
mkInScopeSet (VarSet -> InScopeSet) -> VarSet -> InScopeSet
forall a b. (a -> b) -> a -> b
$
                           [PredType] -> VarSet
tyCoVarsOfTypes (PredType
predPredType -> [PredType] -> [PredType]
forall a. a -> [a] -> [a]
:[PredType]
theta) VarSet -> [TcTyVar] -> VarSet
`delVarSetList` [TcTyVar]
tvs
       ; (TCvSubst
subst, [TcTyVar]
skol_tvs) <- TCvSubst -> [TcTyVar] -> TcS (TCvSubst, [TcTyVar])
tcInstSkolTyVarsX TCvSubst
empty_subst [TcTyVar]
tvs
       ; [TcTyVar]
given_ev_vars <- (PredType -> TcS TcTyVar) -> [PredType] -> TcS [TcTyVar]
forall (t :: * -> *) (m :: * -> *) a b.
(Traversable t, Monad m) =>
(a -> m b) -> t a -> m (t b)
mapM PredType -> TcS TcTyVar
newEvVar (HasCallStack => TCvSubst -> [PredType] -> [PredType]
TCvSubst -> [PredType] -> [PredType]
substTheta TCvSubst
subst [PredType]
theta)

       ; (TcLevel
lvl, (TcTyVar
w_id, Cts
wanteds))
             <- SDoc -> TcS (TcTyVar, Cts) -> TcS (TcLevel, (TcTyVar, Cts))
forall a. SDoc -> TcS a -> TcS (TcLevel, a)
pushLevelNoWorkList (SkolemInfo -> SDoc
forall a. Outputable a => a -> SDoc
ppr SkolemInfo
skol_info) (TcS (TcTyVar, Cts) -> TcS (TcLevel, (TcTyVar, Cts)))
-> TcS (TcTyVar, Cts) -> TcS (TcLevel, (TcTyVar, Cts))
forall a b. (a -> b) -> a -> b
$
                do { CtEvidence
wanted_ev <- CtLoc -> PredType -> TcS CtEvidence
newWantedEvVarNC CtLoc
loc (PredType -> TcS CtEvidence) -> PredType -> TcS CtEvidence
forall a b. (a -> b) -> a -> b
$
                                  HasCallStack => TCvSubst -> PredType -> PredType
TCvSubst -> PredType -> PredType
substTy TCvSubst
subst PredType
pred
                   ; (TcTyVar, Cts) -> TcS (TcTyVar, Cts)
forall (m :: * -> *) a. Monad m => a -> m a
return ( CtEvidence -> TcTyVar
ctEvEvId CtEvidence
wanted_ev
                            , Ct -> Cts
forall a. a -> Bag a
unitBag (CtEvidence -> Ct
mkNonCanonical CtEvidence
wanted_ev)) }

      ; TcEvBinds
ev_binds <- TcLevel
-> SkolemInfo -> [TcTyVar] -> [TcTyVar] -> Cts -> TcS TcEvBinds
emitImplicationTcS TcLevel
lvl SkolemInfo
skol_info [TcTyVar]
skol_tvs
                                       [TcTyVar]
given_ev_vars Cts
wanteds

      ; TcEvDest -> EvTerm -> TcS ()
setWantedEvTerm TcEvDest
dest (EvTerm -> TcS ()) -> EvTerm -> TcS ()
forall a b. (a -> b) -> a -> b
$
        EvFun :: [TcTyVar] -> [TcTyVar] -> TcEvBinds -> TcTyVar -> EvTerm
EvFun { et_tvs :: [TcTyVar]
et_tvs = [TcTyVar]
skol_tvs, et_given :: [TcTyVar]
et_given = [TcTyVar]
given_ev_vars
              , et_binds :: TcEvBinds
et_binds = TcEvBinds
ev_binds, et_body :: TcTyVar
et_body = TcTyVar
w_id }

      ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Wanted forall-constraint" }

  | CtEvidence -> Bool
isGiven CtEvidence
ev   -- See Note [Solving a Given forall-constraint]
  = do { QCInst -> TcS ()
addInertForAll QCInst
qci
       ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Given forall-constraint" }

  | Bool
otherwise
  = CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Derived forall-constraint"
  where
    loc :: CtLoc
loc = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev
    tvs :: [TcTyVar]
tvs = [TyCoVarBinder] -> [TcTyVar]
forall tv argf. [VarBndr tv argf] -> [tv]
binderVars [TyCoVarBinder]
tv_bndrs
    qci :: QCInst
qci = QCI :: CtEvidence -> [TcTyVar] -> PredType -> Bool -> QCInst
QCI { qci_ev :: CtEvidence
qci_ev = CtEvidence
ev, qci_tvs :: [TcTyVar]
qci_tvs = [TcTyVar]
tvs
              , qci_pred :: PredType
qci_pred = PredType
pred, qci_pend_sc :: Bool
qci_pend_sc = Bool
pend_sc }

{- Note [Solving a Wanted forall-constraint]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Solving a wanted forall (quantified) constraint
  [W] df :: forall ab. (Eq a, Ord b) => C x a b
is delightfully easy.   Just build an implication constraint
    forall ab. (g1::Eq a, g2::Ord b) => [W] d :: C x a
and discharge df thus:
    df = /\ab. \g1 g2. let <binds> in d
where <binds> is filled in by solving the implication constraint.
All the machinery is to hand; there is little to do.

Note [Solving a Given forall-constraint]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
For a Given constraint
  [G] df :: forall ab. (Eq a, Ord b) => C x a b
we just add it to TcS's local InstEnv of known instances,
via addInertForall.  Then, if we look up (C x Int Bool), say,
we'll find a match in the InstEnv.


************************************************************************
*                                                                      *
*        Equalities
*                                                                      *
************************************************************************

Note [Canonicalising equalities]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
In order to canonicalise an equality, we look at the structure of the
two types at hand, looking for similarities. A difficulty is that the
types may look dissimilar before flattening but similar after flattening.
However, we don't just want to jump in and flatten right away, because
this might be wasted effort. So, after looking for similarities and failing,
we flatten and then try again. Of course, we don't want to loop, so we
track whether or not we've already flattened.

It is conceivable to do a better job at tracking whether or not a type
is flattened, but this is left as future work. (Mar '15)


Note [FunTy and decomposing tycon applications]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
When can_eq_nc' attempts to decompose a tycon application we haven't yet zonked.
This means that we may very well have a FunTy containing a type of some unknown
kind. For instance, we may have,

    FunTy (a :: k) Int

Where k is a unification variable. tcRepSplitTyConApp_maybe panics in the event
that it sees such a type as it cannot determine the RuntimeReps which the (->)
is applied to. Consequently, it is vital that we instead use
tcRepSplitTyConApp_maybe', which simply returns Nothing in such a case.

When this happens can_eq_nc' will fail to decompose, zonk, and try again.
Zonking should fill the variable k, meaning that decomposition will succeed the
second time around.
-}

canEqNC :: CtEvidence -> EqRel -> Type -> Type -> TcS (StopOrContinue Ct)
canEqNC :: CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqNC CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ty2
  = do { Either (Pair PredType) PredType
result <- PredType -> PredType -> TcS (Either (Pair PredType) PredType)
zonk_eq_types PredType
ty1 PredType
ty2
       ; case Either (Pair PredType) PredType
result of
           Left (Pair PredType
ty1' PredType
ty2') -> Bool
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc Bool
False CtEvidence
ev EqRel
eq_rel PredType
ty1' PredType
ty1 PredType
ty2' PredType
ty2
           Right PredType
ty              -> CtEvidence -> EqRel -> PredType -> TcS (StopOrContinue Ct)
canEqReflexive CtEvidence
ev EqRel
eq_rel PredType
ty }

can_eq_nc
   :: Bool            -- True => both types are flat
   -> CtEvidence
   -> EqRel
   -> Type -> Type    -- LHS, after and before type-synonym expansion, resp
   -> Type -> Type    -- RHS, after and before type-synonym expansion, resp
   -> TcS (StopOrContinue Ct)
can_eq_nc :: Bool
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc Bool
flat CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ps_ty1 PredType
ty2 PredType
ps_ty2
  = do { String -> SDoc -> TcS ()
traceTcS String
"can_eq_nc" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
         [SDoc] -> SDoc
vcat [ Bool -> SDoc
forall a. Outputable a => a -> SDoc
ppr Bool
flat, CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev, EqRel -> SDoc
forall a. Outputable a => a -> SDoc
ppr EqRel
eq_rel, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty1, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ps_ty1, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty2, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ps_ty2 ]
       ; GlobalRdrEnv
rdr_env <- TcS GlobalRdrEnv
getGlobalRdrEnvTcS
       ; (FamInstEnv, FamInstEnv)
fam_insts <- TcS (FamInstEnv, FamInstEnv)
getFamInstEnvs
       ; Bool
-> GlobalRdrEnv
-> (FamInstEnv, FamInstEnv)
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc' Bool
flat GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
fam_insts CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ps_ty1 PredType
ty2 PredType
ps_ty2 }

can_eq_nc'
   :: Bool           -- True => both input types are flattened
   -> GlobalRdrEnv   -- needed to see which newtypes are in scope
   -> FamInstEnvs    -- needed to unwrap data instances
   -> CtEvidence
   -> EqRel
   -> Type -> Type    -- LHS, after and before type-synonym expansion, resp
   -> Type -> Type    -- RHS, after and before type-synonym expansion, resp
   -> TcS (StopOrContinue Ct)

-- Expand synonyms first; see Note [Type synonyms and canonicalization]
can_eq_nc' :: Bool
-> GlobalRdrEnv
-> (FamInstEnv, FamInstEnv)
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc' Bool
flat GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
envs CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ps_ty1 PredType
ty2 PredType
ps_ty2
  | Just PredType
ty1' <- PredType -> Maybe PredType
tcView PredType
ty1 = Bool
-> GlobalRdrEnv
-> (FamInstEnv, FamInstEnv)
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc' Bool
flat GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
envs CtEvidence
ev EqRel
eq_rel PredType
ty1' PredType
ps_ty1 PredType
ty2  PredType
ps_ty2
  | Just PredType
ty2' <- PredType -> Maybe PredType
tcView PredType
ty2 = Bool
-> GlobalRdrEnv
-> (FamInstEnv, FamInstEnv)
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc' Bool
flat GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
envs CtEvidence
ev EqRel
eq_rel PredType
ty1  PredType
ps_ty1 PredType
ty2' PredType
ps_ty2

-- need to check for reflexivity in the ReprEq case.
-- See Note [Eager reflexivity check]
-- Check only when flat because the zonk_eq_types check in canEqNC takes
-- care of the non-flat case.
can_eq_nc' Bool
True GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
ReprEq PredType
ty1 PredType
_ PredType
ty2 PredType
_
  | PredType
ty1 HasDebugCallStack => PredType -> PredType -> Bool
PredType -> PredType -> Bool
`tcEqType` PredType
ty2
  = CtEvidence -> EqRel -> PredType -> TcS (StopOrContinue Ct)
canEqReflexive CtEvidence
ev EqRel
ReprEq PredType
ty1

-- When working with ReprEq, unwrap newtypes.
-- See Note [Unwrap newtypes first]
can_eq_nc' Bool
_flat GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
envs CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ps_ty1 PredType
ty2 PredType
ps_ty2
  | EqRel
ReprEq <- EqRel
eq_rel
  , Just ((Bag GlobalRdrElt, TcCoercion), PredType)
stuff1 <- (FamInstEnv, FamInstEnv)
-> GlobalRdrEnv
-> PredType
-> Maybe ((Bag GlobalRdrElt, TcCoercion), PredType)
tcTopNormaliseNewTypeTF_maybe (FamInstEnv, FamInstEnv)
envs GlobalRdrEnv
rdr_env PredType
ty1
  = CtEvidence
-> SwapFlag
-> PredType
-> ((Bag GlobalRdrElt, TcCoercion), PredType)
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_newtype_nc CtEvidence
ev SwapFlag
NotSwapped PredType
ty1 ((Bag GlobalRdrElt, TcCoercion), PredType)
stuff1 PredType
ty2 PredType
ps_ty2

  | EqRel
ReprEq <- EqRel
eq_rel
  , Just ((Bag GlobalRdrElt, TcCoercion), PredType)
stuff2 <- (FamInstEnv, FamInstEnv)
-> GlobalRdrEnv
-> PredType
-> Maybe ((Bag GlobalRdrElt, TcCoercion), PredType)
tcTopNormaliseNewTypeTF_maybe (FamInstEnv, FamInstEnv)
envs GlobalRdrEnv
rdr_env PredType
ty2
  = CtEvidence
-> SwapFlag
-> PredType
-> ((Bag GlobalRdrElt, TcCoercion), PredType)
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_newtype_nc CtEvidence
ev SwapFlag
IsSwapped  PredType
ty2 ((Bag GlobalRdrElt, TcCoercion), PredType)
stuff2 PredType
ty1 PredType
ps_ty1

-- Then, get rid of casts
can_eq_nc' Bool
flat GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel (CastTy PredType
ty1 TcCoercion
co1) PredType
_ PredType
ty2 PredType
ps_ty2
  = Bool
-> CtEvidence
-> EqRel
-> SwapFlag
-> PredType
-> TcCoercion
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqCast Bool
flat CtEvidence
ev EqRel
eq_rel SwapFlag
NotSwapped PredType
ty1 TcCoercion
co1 PredType
ty2 PredType
ps_ty2
can_eq_nc' Bool
flat GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ps_ty1 (CastTy PredType
ty2 TcCoercion
co2) PredType
_
  = Bool
-> CtEvidence
-> EqRel
-> SwapFlag
-> PredType
-> TcCoercion
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqCast Bool
flat CtEvidence
ev EqRel
eq_rel SwapFlag
IsSwapped PredType
ty2 TcCoercion
co2 PredType
ty1 PredType
ps_ty1

-- NB: pattern match on True: we want only flat types sent to canEqTyVar.
-- See also Note [No top-level newtypes on RHS of representational equalities]
can_eq_nc' Bool
True GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel (TyVarTy TcTyVar
tv1) PredType
ps_ty1 PredType
ty2 PredType
ps_ty2
  = CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVar CtEvidence
ev EqRel
eq_rel SwapFlag
NotSwapped TcTyVar
tv1 PredType
ps_ty1 PredType
ty2 PredType
ps_ty2
can_eq_nc' Bool
True GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ps_ty1 (TyVarTy TcTyVar
tv2) PredType
ps_ty2
  = CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVar CtEvidence
ev EqRel
eq_rel SwapFlag
IsSwapped TcTyVar
tv2 PredType
ps_ty2 PredType
ty1 PredType
ps_ty1

----------------------
-- Otherwise try to decompose
----------------------

-- Literals
can_eq_nc' Bool
_flat GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel ty1 :: PredType
ty1@(LitTy TyLit
l1) PredType
_ (LitTy TyLit
l2) PredType
_
 | TyLit
l1 TyLit -> TyLit -> Bool
forall a. Eq a => a -> a -> Bool
== TyLit
l2
  = do { CtEvidence -> EvTerm -> TcS ()
setEvBindIfWanted CtEvidence
ev (TcCoercion -> EvTerm
evCoercion (TcCoercion -> EvTerm) -> TcCoercion -> EvTerm
forall a b. (a -> b) -> a -> b
$ Role -> PredType -> TcCoercion
mkReflCo (EqRel -> Role
eqRelRole EqRel
eq_rel) PredType
ty1)
       ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Equal LitTy" }

-- Try to decompose type constructor applications
-- Including FunTy (s -> t)
can_eq_nc' Bool
_flat GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
_ PredType
ty2 PredType
_
    --- See Note [FunTy and decomposing type constructor applications].
  | Just (TyCon
tc1, [PredType]
tys1) <- HasDebugCallStack => PredType -> Maybe (TyCon, [PredType])
PredType -> Maybe (TyCon, [PredType])
repSplitTyConApp_maybe PredType
ty1
  , Just (TyCon
tc2, [PredType]
tys2) <- HasDebugCallStack => PredType -> Maybe (TyCon, [PredType])
PredType -> Maybe (TyCon, [PredType])
repSplitTyConApp_maybe PredType
ty2
  , Bool -> Bool
not (TyCon -> Bool
isTypeFamilyTyCon TyCon
tc1)
  , Bool -> Bool
not (TyCon -> Bool
isTypeFamilyTyCon TyCon
tc2)
  = CtEvidence
-> EqRel
-> TyCon
-> [PredType]
-> TyCon
-> [PredType]
-> TcS (StopOrContinue Ct)
canTyConApp CtEvidence
ev EqRel
eq_rel TyCon
tc1 [PredType]
tys1 TyCon
tc2 [PredType]
tys2

can_eq_nc' Bool
_flat GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel
           s1 :: PredType
s1@(ForAllTy {}) PredType
_ s2 :: PredType
s2@(ForAllTy {}) PredType
_
  = CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
can_eq_nc_forall CtEvidence
ev EqRel
eq_rel PredType
s1 PredType
s2

-- See Note [Canonicalising type applications] about why we require flat types
can_eq_nc' Bool
True GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel (AppTy PredType
t1 PredType
s1) PredType
_ PredType
ty2 PredType
_
  | EqRel
NomEq <- EqRel
eq_rel
  , Just (PredType
t2, PredType
s2) <- PredType -> Maybe (PredType, PredType)
tcSplitAppTy_maybe PredType
ty2
  = CtEvidence
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_app CtEvidence
ev PredType
t1 PredType
s1 PredType
t2 PredType
s2
can_eq_nc' Bool
True GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
_ (AppTy PredType
t2 PredType
s2) PredType
_
  | EqRel
NomEq <- EqRel
eq_rel
  , Just (PredType
t1, PredType
s1) <- PredType -> Maybe (PredType, PredType)
tcSplitAppTy_maybe PredType
ty1
  = CtEvidence
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_app CtEvidence
ev PredType
t1 PredType
s1 PredType
t2 PredType
s2

-- No similarity in type structure detected. Flatten and try again.
can_eq_nc' Bool
False GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
envs CtEvidence
ev EqRel
eq_rel PredType
_ PredType
ps_ty1 PredType
_ PredType
ps_ty2
  = do { (PredType
xi1, TcCoercion
co1) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_FlattenAll CtEvidence
ev PredType
ps_ty1
       ; (PredType
xi2, TcCoercion
co2) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_FlattenAll CtEvidence
ev PredType
ps_ty2
       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
NotSwapped PredType
xi1 PredType
xi2 TcCoercion
co1 TcCoercion
co2
       ; Bool
-> GlobalRdrEnv
-> (FamInstEnv, FamInstEnv)
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc' Bool
True GlobalRdrEnv
rdr_env (FamInstEnv, FamInstEnv)
envs CtEvidence
new_ev EqRel
eq_rel PredType
xi1 PredType
xi1 PredType
xi2 PredType
xi2 }

-- We've flattened and the types don't match. Give up.
can_eq_nc' Bool
True GlobalRdrEnv
_rdr_env (FamInstEnv, FamInstEnv)
_envs CtEvidence
ev EqRel
eq_rel PredType
_ PredType
ps_ty1 PredType
_ PredType
ps_ty2
  = do { String -> SDoc -> TcS ()
traceTcS String
"can_eq_nc' catch-all case" (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ps_ty1 SDoc -> SDoc -> SDoc
$$ PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ps_ty2)
       ; case EqRel
eq_rel of -- See Note [Unsolved equalities]
            EqRel
ReprEq -> Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkIrredCt CtEvidence
ev)
            EqRel
NomEq  -> Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkInsolubleCt CtEvidence
ev) }
          -- No need to call canEqFailure/canEqHardFailure because they
          -- flatten, and the types involved here are already flat

{- Note [Unsolved equalities]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
If we have an unsolved equality like
  (a b ~R# Int)
that is not necessarily insoluble!  Maybe 'a' will turn out to be a newtype.
So we want to make it a potentially-soluble Irred not an insoluble one.
Missing this point is what caused #15431
-}

---------------------------------
can_eq_nc_forall :: CtEvidence -> EqRel
                 -> Type -> Type    -- LHS and RHS
                 -> TcS (StopOrContinue Ct)
-- (forall as. phi1) ~ (forall bs. phi2)
-- Check for length match of as, bs
-- Then build an implication constraint: forall as. phi1 ~ phi2[as/bs]
-- But remember also to unify the kinds of as and bs
--  (this is the 'go' loop), and actually substitute phi2[as |> cos / bs]
-- Remember also that we might have forall z (a:z). blah
--  so we must proceed one binder at a time (#13879)

can_eq_nc_forall :: CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
can_eq_nc_forall CtEvidence
ev EqRel
eq_rel PredType
s1 PredType
s2
 | CtWanted { ctev_loc :: CtEvidence -> CtLoc
ctev_loc = CtLoc
loc, ctev_dest :: CtEvidence -> TcEvDest
ctev_dest = TcEvDest
orig_dest } <- CtEvidence
ev
 = do { let free_tvs :: VarSet
free_tvs       = [PredType] -> VarSet
tyCoVarsOfTypes [PredType
s1,PredType
s2]
            ([TyCoVarBinder]
bndrs1, PredType
phi1) = PredType -> ([TyCoVarBinder], PredType)
tcSplitForAllVarBndrs PredType
s1
            ([TyCoVarBinder]
bndrs2, PredType
phi2) = PredType -> ([TyCoVarBinder], PredType)
tcSplitForAllVarBndrs PredType
s2
      ; if Bool -> Bool
not ([TyCoVarBinder] -> [TyCoVarBinder] -> Bool
forall a b. [a] -> [b] -> Bool
equalLength [TyCoVarBinder]
bndrs1 [TyCoVarBinder]
bndrs2)
        then do { String -> SDoc -> TcS ()
traceTcS String
"Forall failure" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
                     [SDoc] -> SDoc
vcat [ PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
s1, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
s2, [TyCoVarBinder] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [TyCoVarBinder]
bndrs1, [TyCoVarBinder] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [TyCoVarBinder]
bndrs2
                          , [ArgFlag] -> SDoc
forall a. Outputable a => a -> SDoc
ppr ((TyCoVarBinder -> ArgFlag) -> [TyCoVarBinder] -> [ArgFlag]
forall a b. (a -> b) -> [a] -> [b]
map TyCoVarBinder -> ArgFlag
forall tv argf. VarBndr tv argf -> argf
binderArgFlag [TyCoVarBinder]
bndrs1)
                          , [ArgFlag] -> SDoc
forall a. Outputable a => a -> SDoc
ppr ((TyCoVarBinder -> ArgFlag) -> [TyCoVarBinder] -> [ArgFlag]
forall a b. (a -> b) -> [a] -> [b]
map TyCoVarBinder -> ArgFlag
forall tv argf. VarBndr tv argf -> argf
binderArgFlag [TyCoVarBinder]
bndrs2) ]
                ; CtEvidence -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqHardFailure CtEvidence
ev PredType
s1 PredType
s2 }
        else
   do { String -> SDoc -> TcS ()
traceTcS String
"Creating implication for polytype equality" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$ CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev
      ; let empty_subst1 :: TCvSubst
empty_subst1 = InScopeSet -> TCvSubst
mkEmptyTCvSubst (InScopeSet -> TCvSubst) -> InScopeSet -> TCvSubst
forall a b. (a -> b) -> a -> b
$ VarSet -> InScopeSet
mkInScopeSet VarSet
free_tvs
      ; (TCvSubst
subst1, [TcTyVar]
skol_tvs) <- TCvSubst -> [TcTyVar] -> TcS (TCvSubst, [TcTyVar])
tcInstSkolTyVarsX TCvSubst
empty_subst1 ([TcTyVar] -> TcS (TCvSubst, [TcTyVar]))
-> [TcTyVar] -> TcS (TCvSubst, [TcTyVar])
forall a b. (a -> b) -> a -> b
$
                              [TyCoVarBinder] -> [TcTyVar]
forall tv argf. [VarBndr tv argf] -> [tv]
binderVars [TyCoVarBinder]
bndrs1

      ; let skol_info :: SkolemInfo
skol_info = PredType -> SkolemInfo
UnifyForAllSkol PredType
phi1
            phi1' :: PredType
phi1' = HasCallStack => TCvSubst -> PredType -> PredType
TCvSubst -> PredType -> PredType
substTy TCvSubst
subst1 PredType
phi1

            -- Unify the kinds, extend the substitution
            go :: [TcTyVar] -> TCvSubst -> [TyVarBinder]
               -> TcS (TcCoercion, Cts)
            go :: [TcTyVar] -> TCvSubst -> [TyCoVarBinder] -> TcS (TcCoercion, Cts)
go (TcTyVar
skol_tv:[TcTyVar]
skol_tvs) TCvSubst
subst (TyCoVarBinder
bndr2:[TyCoVarBinder]
bndrs2)
              = do { let tv2 :: TcTyVar
tv2 = TyCoVarBinder -> TcTyVar
forall tv argf. VarBndr tv argf -> tv
binderVar TyCoVarBinder
bndr2
                   ; (TcCoercion
kind_co, Cts
wanteds1) <- CtLoc -> Role -> PredType -> PredType -> TcS (TcCoercion, Cts)
unify CtLoc
loc Role
Nominal (TcTyVar -> PredType
tyVarKind TcTyVar
skol_tv)
                                                  (HasCallStack => TCvSubst -> PredType -> PredType
TCvSubst -> PredType -> PredType
substTy TCvSubst
subst (TcTyVar -> PredType
tyVarKind TcTyVar
tv2))
                   ; let subst' :: TCvSubst
subst' = TCvSubst -> TcTyVar -> PredType -> TCvSubst
extendTvSubstAndInScope TCvSubst
subst TcTyVar
tv2
                                       (PredType -> TcCoercion -> PredType
mkCastTy (TcTyVar -> PredType
mkTyVarTy TcTyVar
skol_tv) TcCoercion
kind_co)
                         -- skol_tv is already in the in-scope set, but the
                         -- free vars of kind_co are not; hence "...AndInScope"
                   ; (TcCoercion
co, Cts
wanteds2) <- [TcTyVar] -> TCvSubst -> [TyCoVarBinder] -> TcS (TcCoercion, Cts)
go [TcTyVar]
skol_tvs TCvSubst
subst' [TyCoVarBinder]
bndrs2
                   ; (TcCoercion, Cts) -> TcS (TcCoercion, Cts)
forall (m :: * -> *) a. Monad m => a -> m a
return ( TcTyVar -> TcCoercion -> TcCoercion -> TcCoercion
mkTcForAllCo TcTyVar
skol_tv TcCoercion
kind_co TcCoercion
co
                            , Cts
wanteds1 Cts -> Cts -> Cts
forall a. Bag a -> Bag a -> Bag a
`unionBags` Cts
wanteds2 ) }

            -- Done: unify phi1 ~ phi2
            go [] TCvSubst
subst [TyCoVarBinder]
bndrs2
              = ASSERT( null bndrs2 )
                CtLoc -> Role -> PredType -> PredType -> TcS (TcCoercion, Cts)
unify CtLoc
loc (EqRel -> Role
eqRelRole EqRel
eq_rel) PredType
phi1' (TCvSubst -> PredType -> PredType
substTyUnchecked TCvSubst
subst PredType
phi2)

            go [TcTyVar]
_ TCvSubst
_ [TyCoVarBinder]
_ = String -> TcS (TcCoercion, Cts)
forall a. String -> a
panic String
"cna_eq_nc_forall"  -- case (s:ss) []

            empty_subst2 :: TCvSubst
empty_subst2 = InScopeSet -> TCvSubst
mkEmptyTCvSubst (TCvSubst -> InScopeSet
getTCvInScope TCvSubst
subst1)

      ; (TcLevel
lvl, (TcCoercion
all_co, Cts
wanteds)) <- SDoc -> TcS (TcCoercion, Cts) -> TcS (TcLevel, (TcCoercion, Cts))
forall a. SDoc -> TcS a -> TcS (TcLevel, a)
pushLevelNoWorkList (SkolemInfo -> SDoc
forall a. Outputable a => a -> SDoc
ppr SkolemInfo
skol_info) (TcS (TcCoercion, Cts) -> TcS (TcLevel, (TcCoercion, Cts)))
-> TcS (TcCoercion, Cts) -> TcS (TcLevel, (TcCoercion, Cts))
forall a b. (a -> b) -> a -> b
$
                                    [TcTyVar] -> TCvSubst -> [TyCoVarBinder] -> TcS (TcCoercion, Cts)
go [TcTyVar]
skol_tvs TCvSubst
empty_subst2 [TyCoVarBinder]
bndrs2
      ; TcLevel -> SkolemInfo -> [TcTyVar] -> Cts -> TcS ()
emitTvImplicationTcS TcLevel
lvl SkolemInfo
skol_info [TcTyVar]
skol_tvs Cts
wanteds

      ; TcEvDest -> TcCoercion -> TcS ()
setWantedEq TcEvDest
orig_dest TcCoercion
all_co
      ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Deferred polytype equality" } }

 | Bool
otherwise
 = do { String -> SDoc -> TcS ()
traceTcS String
"Omitting decomposition of given polytype equality" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
        PredType -> PredType -> SDoc
pprEq PredType
s1 PredType
s2    -- See Note [Do not decompose given polytype equalities]
      ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Discard given polytype equality" }

 where
    unify :: CtLoc -> Role -> TcType -> TcType -> TcS (TcCoercion, Cts)
    -- This version returns the wanted constraint rather
    -- than putting it in the work list
    unify :: CtLoc -> Role -> PredType -> PredType -> TcS (TcCoercion, Cts)
unify CtLoc
loc Role
role PredType
ty1 PredType
ty2
      | PredType
ty1 HasDebugCallStack => PredType -> PredType -> Bool
PredType -> PredType -> Bool
`tcEqType` PredType
ty2
      = (TcCoercion, Cts) -> TcS (TcCoercion, Cts)
forall (m :: * -> *) a. Monad m => a -> m a
return (Role -> PredType -> TcCoercion
mkTcReflCo Role
role PredType
ty1, Cts
forall a. Bag a
emptyBag)
      | Bool
otherwise
      = do { (CtEvidence
wanted, TcCoercion
co) <- CtLoc
-> Role -> PredType -> PredType -> TcS (CtEvidence, TcCoercion)
newWantedEq CtLoc
loc Role
role PredType
ty1 PredType
ty2
           ; (TcCoercion, Cts) -> TcS (TcCoercion, Cts)
forall (m :: * -> *) a. Monad m => a -> m a
return (TcCoercion
co, Ct -> Cts
forall a. a -> Bag a
unitBag (CtEvidence -> Ct
mkNonCanonical CtEvidence
wanted)) }

---------------------------------
-- | Compare types for equality, while zonking as necessary. Gives up
-- as soon as it finds that two types are not equal.
-- This is quite handy when some unification has made two
-- types in an inert Wanted to be equal. We can discover the equality without
-- flattening, which is sometimes very expensive (in the case of type functions).
-- In particular, this function makes a ~20% improvement in test case
-- perf/compiler/T5030.
--
-- Returns either the (partially zonked) types in the case of
-- inequality, or the one type in the case of equality. canEqReflexive is
-- a good next step in the 'Right' case. Returning 'Left' is always safe.
--
-- NB: This does *not* look through type synonyms. In fact, it treats type
-- synonyms as rigid constructors. In the future, it might be convenient
-- to look at only those arguments of type synonyms that actually appear
-- in the synonym RHS. But we're not there yet.
zonk_eq_types :: TcType -> TcType -> TcS (Either (Pair TcType) TcType)
zonk_eq_types :: PredType -> PredType -> TcS (Either (Pair PredType) PredType)
zonk_eq_types = PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go
  where
    go :: PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go (TyVarTy TcTyVar
tv1) (TyVarTy TcTyVar
tv2) = TcTyVar -> TcTyVar -> TcS (Either (Pair PredType) PredType)
tyvar_tyvar TcTyVar
tv1 TcTyVar
tv2
    go (TyVarTy TcTyVar
tv1) PredType
ty2           = SwapFlag
-> TcTyVar -> PredType -> TcS (Either (Pair PredType) PredType)
tyvar SwapFlag
NotSwapped TcTyVar
tv1 PredType
ty2
    go PredType
ty1 (TyVarTy TcTyVar
tv2)           = SwapFlag
-> TcTyVar -> PredType -> TcS (Either (Pair PredType) PredType)
tyvar SwapFlag
IsSwapped  TcTyVar
tv2 PredType
ty1

    -- We handle FunTys explicitly here despite the fact that they could also be
    -- treated as an application. Why? Well, for one it's cheaper to just look
    -- at two types (the argument and result types) than four (the argument,
    -- result, and their RuntimeReps). Also, we haven't completely zonked yet,
    -- so we may run into an unzonked type variable while trying to compute the
    -- RuntimeReps of the argument and result types. This can be observed in
    -- testcase tc269.
    go PredType
ty1 PredType
ty2
      | Just (PredType
arg1, PredType
res1) <- Maybe (PredType, PredType)
split1
      , Just (PredType
arg2, PredType
res2) <- Maybe (PredType, PredType)
split2
      = do { Either (Pair PredType) PredType
res_a <- PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go PredType
arg1 PredType
arg2
           ; Either (Pair PredType) PredType
res_b <- PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go PredType
res1 PredType
res2
           ; Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a. Monad m => a -> m a
return (Either (Pair PredType) PredType
 -> TcS (Either (Pair PredType) PredType))
-> Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall a b. (a -> b) -> a -> b
$ (PredType -> PredType -> PredType)
-> Either (Pair PredType) PredType
-> Either (Pair PredType) PredType
-> Either (Pair PredType) PredType
forall a b c.
(a -> b -> c)
-> Either (Pair b) b -> Either (Pair a) a -> Either (Pair c) c
combine_rev PredType -> PredType -> PredType
mkVisFunTy Either (Pair PredType) PredType
res_b Either (Pair PredType) PredType
res_a
           }
      | Maybe (PredType, PredType) -> Bool
forall a. Maybe a -> Bool
isJust Maybe (PredType, PredType)
split1 Bool -> Bool -> Bool
|| Maybe (PredType, PredType) -> Bool
forall a. Maybe a -> Bool
isJust Maybe (PredType, PredType)
split2
      = PredType -> PredType -> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a b.
Monad m =>
a -> a -> m (Either (Pair a) b)
bale_out PredType
ty1 PredType
ty2
      where
        split1 :: Maybe (PredType, PredType)
split1 = PredType -> Maybe (PredType, PredType)
tcSplitFunTy_maybe PredType
ty1
        split2 :: Maybe (PredType, PredType)
split2 = PredType -> Maybe (PredType, PredType)
tcSplitFunTy_maybe PredType
ty2

    go PredType
ty1 PredType
ty2
      | Just (TyCon
tc1, [PredType]
tys1) <- HasDebugCallStack => PredType -> Maybe (TyCon, [PredType])
PredType -> Maybe (TyCon, [PredType])
repSplitTyConApp_maybe PredType
ty1
      , Just (TyCon
tc2, [PredType]
tys2) <- HasDebugCallStack => PredType -> Maybe (TyCon, [PredType])
PredType -> Maybe (TyCon, [PredType])
repSplitTyConApp_maybe PredType
ty2
      = if TyCon
tc1 TyCon -> TyCon -> Bool
forall a. Eq a => a -> a -> Bool
== TyCon
tc2 Bool -> Bool -> Bool
&& [PredType]
tys1 [PredType] -> [PredType] -> Bool
forall a b. [a] -> [b] -> Bool
`equalLength` [PredType]
tys2
          -- Crucial to check for equal-length args, because
          -- we cannot assume that the two args to 'go' have
          -- the same kind.  E.g go (Proxy *      (Maybe Int))
          --                        (Proxy (*->*) Maybe)
          -- We'll call (go (Maybe Int) Maybe)
          -- See #13083
        then TyCon
-> [PredType]
-> [PredType]
-> TcS (Either (Pair PredType) PredType)
tycon TyCon
tc1 [PredType]
tys1 [PredType]
tys2
        else PredType -> PredType -> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a b.
Monad m =>
a -> a -> m (Either (Pair a) b)
bale_out PredType
ty1 PredType
ty2

    go PredType
ty1 PredType
ty2
      | Just (PredType
ty1a, PredType
ty1b) <- PredType -> Maybe (PredType, PredType)
tcRepSplitAppTy_maybe PredType
ty1
      , Just (PredType
ty2a, PredType
ty2b) <- PredType -> Maybe (PredType, PredType)
tcRepSplitAppTy_maybe PredType
ty2
      = do { Either (Pair PredType) PredType
res_a <- PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go PredType
ty1a PredType
ty2a
           ; Either (Pair PredType) PredType
res_b <- PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go PredType
ty1b PredType
ty2b
           ; Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a. Monad m => a -> m a
return (Either (Pair PredType) PredType
 -> TcS (Either (Pair PredType) PredType))
-> Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall a b. (a -> b) -> a -> b
$ (PredType -> PredType -> PredType)
-> Either (Pair PredType) PredType
-> Either (Pair PredType) PredType
-> Either (Pair PredType) PredType
forall a b c.
(a -> b -> c)
-> Either (Pair b) b -> Either (Pair a) a -> Either (Pair c) c
combine_rev PredType -> PredType -> PredType
mkAppTy Either (Pair PredType) PredType
res_b Either (Pair PredType) PredType
res_a }

    go ty1 :: PredType
ty1@(LitTy TyLit
lit1) (LitTy TyLit
lit2)
      | TyLit
lit1 TyLit -> TyLit -> Bool
forall a. Eq a => a -> a -> Bool
== TyLit
lit2
      = Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a. Monad m => a -> m a
return (PredType -> Either (Pair PredType) PredType
forall a b. b -> Either a b
Right PredType
ty1)

    go PredType
ty1 PredType
ty2 = PredType -> PredType -> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a b.
Monad m =>
a -> a -> m (Either (Pair a) b)
bale_out PredType
ty1 PredType
ty2
      -- We don't handle more complex forms here

    bale_out :: a -> a -> m (Either (Pair a) b)
bale_out a
ty1 a
ty2 = Either (Pair a) b -> m (Either (Pair a) b)
forall (m :: * -> *) a. Monad m => a -> m a
return (Either (Pair a) b -> m (Either (Pair a) b))
-> Either (Pair a) b -> m (Either (Pair a) b)
forall a b. (a -> b) -> a -> b
$ Pair a -> Either (Pair a) b
forall a b. a -> Either a b
Left (a -> a -> Pair a
forall a. a -> a -> Pair a
Pair a
ty1 a
ty2)

    tyvar :: SwapFlag -> TcTyVar -> TcType
          -> TcS (Either (Pair TcType) TcType)
      -- Try to do as little as possible, as anything we do here is redundant
      -- with flattening. In particular, no need to zonk kinds. That's why
      -- we don't use the already-defined zonking functions
    tyvar :: SwapFlag
-> TcTyVar -> PredType -> TcS (Either (Pair PredType) PredType)
tyvar SwapFlag
swapped TcTyVar
tv PredType
ty
      = case TcTyVar -> TcTyVarDetails
tcTyVarDetails TcTyVar
tv of
          MetaTv { mtv_ref :: TcTyVarDetails -> IORef MetaDetails
mtv_ref = IORef MetaDetails
ref }
            -> do { MetaDetails
cts <- IORef MetaDetails -> TcS MetaDetails
forall a. TcRef a -> TcS a
readTcRef IORef MetaDetails
ref
                  ; case MetaDetails
cts of
                      MetaDetails
Flexi        -> TcS (Either (Pair PredType) PredType)
forall b. TcS (Either (Pair PredType) b)
give_up
                      Indirect PredType
ty' -> do { TcTyVar -> PredType -> TcS ()
forall a a. (Outputable a, Outputable a) => a -> a -> TcS ()
trace_indirect TcTyVar
tv PredType
ty'
                                         ; SwapFlag
-> (PredType -> PredType -> TcS (Either (Pair PredType) PredType))
-> PredType
-> PredType
-> TcS (Either (Pair PredType) PredType)
forall a b. SwapFlag -> (a -> a -> b) -> a -> a -> b
unSwap SwapFlag
swapped PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go PredType
ty' PredType
ty } }
          TcTyVarDetails
_ -> TcS (Either (Pair PredType) PredType)
forall b. TcS (Either (Pair PredType) b)
give_up
      where
        give_up :: TcS (Either (Pair PredType) b)
give_up = Either (Pair PredType) b -> TcS (Either (Pair PredType) b)
forall (m :: * -> *) a. Monad m => a -> m a
return (Either (Pair PredType) b -> TcS (Either (Pair PredType) b))
-> Either (Pair PredType) b -> TcS (Either (Pair PredType) b)
forall a b. (a -> b) -> a -> b
$ Pair PredType -> Either (Pair PredType) b
forall a b. a -> Either a b
Left (Pair PredType -> Either (Pair PredType) b)
-> Pair PredType -> Either (Pair PredType) b
forall a b. (a -> b) -> a -> b
$ SwapFlag
-> (PredType -> PredType -> Pair PredType)
-> PredType
-> PredType
-> Pair PredType
forall a b. SwapFlag -> (a -> a -> b) -> a -> a -> b
unSwap SwapFlag
swapped PredType -> PredType -> Pair PredType
forall a. a -> a -> Pair a
Pair (TcTyVar -> PredType
mkTyVarTy TcTyVar
tv) PredType
ty

    tyvar_tyvar :: TcTyVar -> TcTyVar -> TcS (Either (Pair PredType) PredType)
tyvar_tyvar TcTyVar
tv1 TcTyVar
tv2
      | TcTyVar
tv1 TcTyVar -> TcTyVar -> Bool
forall a. Eq a => a -> a -> Bool
== TcTyVar
tv2 = Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a. Monad m => a -> m a
return (PredType -> Either (Pair PredType) PredType
forall a b. b -> Either a b
Right (TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1))
      | Bool
otherwise  = do { (PredType
ty1', Bool
progress1) <- TcTyVar -> TcS (PredType, Bool)
quick_zonk TcTyVar
tv1
                        ; (PredType
ty2', Bool
progress2) <- TcTyVar -> TcS (PredType, Bool)
quick_zonk TcTyVar
tv2
                        ; if Bool
progress1 Bool -> Bool -> Bool
|| Bool
progress2
                          then PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go PredType
ty1' PredType
ty2'
                          else Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a. Monad m => a -> m a
return (Either (Pair PredType) PredType
 -> TcS (Either (Pair PredType) PredType))
-> Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall a b. (a -> b) -> a -> b
$ Pair PredType -> Either (Pair PredType) PredType
forall a b. a -> Either a b
Left (PredType -> PredType -> Pair PredType
forall a. a -> a -> Pair a
Pair (TcTyVar -> PredType
TyVarTy TcTyVar
tv1) (TcTyVar -> PredType
TyVarTy TcTyVar
tv2)) }

    trace_indirect :: a -> a -> TcS ()
trace_indirect a
tv a
ty
       = String -> SDoc -> TcS ()
traceTcS String
"Following filled tyvar (zonk_eq_types)"
                  (a -> SDoc
forall a. Outputable a => a -> SDoc
ppr a
tv SDoc -> SDoc -> SDoc
<+> SDoc
equals SDoc -> SDoc -> SDoc
<+> a -> SDoc
forall a. Outputable a => a -> SDoc
ppr a
ty)

    quick_zonk :: TcTyVar -> TcS (PredType, Bool)
quick_zonk TcTyVar
tv = case TcTyVar -> TcTyVarDetails
tcTyVarDetails TcTyVar
tv of
      MetaTv { mtv_ref :: TcTyVarDetails -> IORef MetaDetails
mtv_ref = IORef MetaDetails
ref }
        -> do { MetaDetails
cts <- IORef MetaDetails -> TcS MetaDetails
forall a. TcRef a -> TcS a
readTcRef IORef MetaDetails
ref
              ; case MetaDetails
cts of
                  MetaDetails
Flexi        -> (PredType, Bool) -> TcS (PredType, Bool)
forall (m :: * -> *) a. Monad m => a -> m a
return (TcTyVar -> PredType
TyVarTy TcTyVar
tv, Bool
False)
                  Indirect PredType
ty' -> do { TcTyVar -> PredType -> TcS ()
forall a a. (Outputable a, Outputable a) => a -> a -> TcS ()
trace_indirect TcTyVar
tv PredType
ty'
                                     ; (PredType, Bool) -> TcS (PredType, Bool)
forall (m :: * -> *) a. Monad m => a -> m a
return (PredType
ty', Bool
True) } }
      TcTyVarDetails
_ -> (PredType, Bool) -> TcS (PredType, Bool)
forall (m :: * -> *) a. Monad m => a -> m a
return (TcTyVar -> PredType
TyVarTy TcTyVar
tv, Bool
False)

      -- This happens for type families, too. But recall that failure
      -- here just means to try harder, so it's OK if the type function
      -- isn't injective.
    tycon :: TyCon -> [TcType] -> [TcType]
          -> TcS (Either (Pair TcType) TcType)
    tycon :: TyCon
-> [PredType]
-> [PredType]
-> TcS (Either (Pair PredType) PredType)
tycon TyCon
tc [PredType]
tys1 [PredType]
tys2
      = do { [Either (Pair PredType) PredType]
results <- (PredType -> PredType -> TcS (Either (Pair PredType) PredType))
-> [PredType]
-> [PredType]
-> TcS [Either (Pair PredType) PredType]
forall (m :: * -> *) a b c.
Applicative m =>
(a -> b -> m c) -> [a] -> [b] -> m [c]
zipWithM PredType -> PredType -> TcS (Either (Pair PredType) PredType)
go [PredType]
tys1 [PredType]
tys2
           ; Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall (m :: * -> *) a. Monad m => a -> m a
return (Either (Pair PredType) PredType
 -> TcS (Either (Pair PredType) PredType))
-> Either (Pair PredType) PredType
-> TcS (Either (Pair PredType) PredType)
forall a b. (a -> b) -> a -> b
$ case [Either (Pair PredType) PredType]
-> Either (Pair [PredType]) [PredType]
combine_results [Either (Pair PredType) PredType]
results of
               Left Pair [PredType]
tys  -> Pair PredType -> Either (Pair PredType) PredType
forall a b. a -> Either a b
Left (TyCon -> [PredType] -> PredType
mkTyConApp TyCon
tc ([PredType] -> PredType) -> Pair [PredType] -> Pair PredType
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Pair [PredType]
tys)
               Right [PredType]
tys -> PredType -> Either (Pair PredType) PredType
forall a b. b -> Either a b
Right (TyCon -> [PredType] -> PredType
mkTyConApp TyCon
tc [PredType]
tys) }

    combine_results :: [Either (Pair TcType) TcType]
                    -> Either (Pair [TcType]) [TcType]
    combine_results :: [Either (Pair PredType) PredType]
-> Either (Pair [PredType]) [PredType]
combine_results = (Pair [PredType] -> Pair [PredType])
-> ([PredType] -> [PredType])
-> Either (Pair [PredType]) [PredType]
-> Either (Pair [PredType]) [PredType]
forall (p :: * -> * -> *) a b c d.
Bifunctor p =>
(a -> b) -> (c -> d) -> p a c -> p b d
bimap (([PredType] -> [PredType]) -> Pair [PredType] -> Pair [PredType]
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
fmap [PredType] -> [PredType]
forall a. [a] -> [a]
reverse) [PredType] -> [PredType]
forall a. [a] -> [a]
reverse (Either (Pair [PredType]) [PredType]
 -> Either (Pair [PredType]) [PredType])
-> ([Either (Pair PredType) PredType]
    -> Either (Pair [PredType]) [PredType])
-> [Either (Pair PredType) PredType]
-> Either (Pair [PredType]) [PredType]
forall b c a. (b -> c) -> (a -> b) -> a -> c
.
                      (Either (Pair [PredType]) [PredType]
 -> Either (Pair PredType) PredType
 -> Either (Pair [PredType]) [PredType])
-> Either (Pair [PredType]) [PredType]
-> [Either (Pair PredType) PredType]
-> Either (Pair [PredType]) [PredType]
forall (t :: * -> *) b a.
Foldable t =>
(b -> a -> b) -> b -> t a -> b
foldl' ((PredType -> [PredType] -> [PredType])
-> Either (Pair [PredType]) [PredType]
-> Either (Pair PredType) PredType
-> Either (Pair [PredType]) [PredType]
forall a b c.
(a -> b -> c)
-> Either (Pair b) b -> Either (Pair a) a -> Either (Pair c) c
combine_rev (:)) ([PredType] -> Either (Pair [PredType]) [PredType]
forall a b. b -> Either a b
Right [])

      -- combine (in reverse) a new result onto an already-combined result
    combine_rev :: (a -> b -> c)
                -> Either (Pair b) b
                -> Either (Pair a) a
                -> Either (Pair c) c
    combine_rev :: (a -> b -> c)
-> Either (Pair b) b -> Either (Pair a) a -> Either (Pair c) c
combine_rev a -> b -> c
f (Left Pair b
list) (Left Pair a
elt) = Pair c -> Either (Pair c) c
forall a b. a -> Either a b
Left (a -> b -> c
f (a -> b -> c) -> Pair a -> Pair (b -> c)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Pair a
elt     Pair (b -> c) -> Pair b -> Pair c
forall (f :: * -> *) a b. Applicative f => f (a -> b) -> f a -> f b
<*> Pair b
list)
    combine_rev a -> b -> c
f (Left Pair b
list) (Right a
ty) = Pair c -> Either (Pair c) c
forall a b. a -> Either a b
Left (a -> b -> c
f (a -> b -> c) -> Pair a -> Pair (b -> c)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> a -> Pair a
forall (f :: * -> *) a. Applicative f => a -> f a
pure a
ty Pair (b -> c) -> Pair b -> Pair c
forall (f :: * -> *) a b. Applicative f => f (a -> b) -> f a -> f b
<*> Pair b
list)
    combine_rev a -> b -> c
f (Right b
tys) (Left Pair a
elt) = Pair c -> Either (Pair c) c
forall a b. a -> Either a b
Left (a -> b -> c
f (a -> b -> c) -> Pair a -> Pair (b -> c)
forall (f :: * -> *) a b. Functor f => (a -> b) -> f a -> f b
<$> Pair a
elt     Pair (b -> c) -> Pair b -> Pair c
forall (f :: * -> *) a b. Applicative f => f (a -> b) -> f a -> f b
<*> b -> Pair b
forall (f :: * -> *) a. Applicative f => a -> f a
pure b
tys)
    combine_rev a -> b -> c
f (Right b
tys) (Right a
ty) = c -> Either (Pair c) c
forall a b. b -> Either a b
Right (a -> b -> c
f a
ty b
tys)

{- See Note [Unwrap newtypes first]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Consider
  newtype N m a = MkN (m a)
Then N will get a conservative, Nominal role for its second parameter 'a',
because it appears as an argument to the unknown 'm'. Now consider
  [W] N Maybe a  ~R#  N Maybe b

If we decompose, we'll get
  [W] a ~N# b

But if instead we unwrap we'll get
  [W] Maybe a ~R# Maybe b
which in turn gives us
  [W] a ~R# b
which is easier to satisfy.

Bottom line: unwrap newtypes before decomposing them!
c.f. #9123 comment:52,53 for a compelling example.

Note [Newtypes can blow the stack]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Suppose we have

  newtype X = MkX (Int -> X)
  newtype Y = MkY (Int -> Y)

and now wish to prove

  [W] X ~R Y

This Wanted will loop, expanding out the newtypes ever deeper looking
for a solid match or a solid discrepancy. Indeed, there is something
appropriate to this looping, because X and Y *do* have the same representation,
in the limit -- they're both (Fix ((->) Int)). However, no finitely-sized
coercion will ever witness it. This loop won't actually cause GHC to hang,
though, because we check our depth when unwrapping newtypes.

Note [Eager reflexivity check]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Suppose we have

  newtype X = MkX (Int -> X)

and

  [W] X ~R X

Naively, we would start unwrapping X and end up in a loop. Instead,
we do this eager reflexivity check. This is necessary only for representational
equality because the flattener technology deals with the similar case
(recursive type families) for nominal equality.

Note that this check does not catch all cases, but it will catch the cases
we're most worried about, types like X above that are actually inhabited.

Here's another place where this reflexivity check is key:
Consider trying to prove (f a) ~R (f a). The AppTys in there can't
be decomposed, because representational equality isn't congruent with respect
to AppTy. So, when canonicalising the equality above, we get stuck and
would normally produce a CIrredCan. However, we really do want to
be able to solve (f a) ~R (f a). So, in the representational case only,
we do a reflexivity check.

(This would be sound in the nominal case, but unnecessary, and I [Richard
E.] am worried that it would slow down the common case.)
-}

------------------------
-- | We're able to unwrap a newtype. Update the bits accordingly.
can_eq_newtype_nc :: CtEvidence           -- ^ :: ty1 ~ ty2
                  -> SwapFlag
                  -> TcType                                    -- ^ ty1
                  -> ((Bag GlobalRdrElt, TcCoercion), TcType)  -- ^ :: ty1 ~ ty1'
                  -> TcType               -- ^ ty2
                  -> TcType               -- ^ ty2, with type synonyms
                  -> TcS (StopOrContinue Ct)
can_eq_newtype_nc :: CtEvidence
-> SwapFlag
-> PredType
-> ((Bag GlobalRdrElt, TcCoercion), PredType)
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_newtype_nc CtEvidence
ev SwapFlag
swapped PredType
ty1 ((Bag GlobalRdrElt
gres, TcCoercion
co), PredType
ty1') PredType
ty2 PredType
ps_ty2
  = do { String -> SDoc -> TcS ()
traceTcS String
"can_eq_newtype_nc" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
         [SDoc] -> SDoc
vcat [ CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev, SwapFlag -> SDoc
forall a. Outputable a => a -> SDoc
ppr SwapFlag
swapped, TcCoercion -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcCoercion
co, Bag GlobalRdrElt -> SDoc
forall a. Outputable a => a -> SDoc
ppr Bag GlobalRdrElt
gres, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty1', PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty2 ]

         -- check for blowing our stack:
         -- See Note [Newtypes can blow the stack]
       ; CtLoc -> PredType -> TcS ()
checkReductionDepth (CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev) PredType
ty1

         -- Next, we record uses of newtype constructors, since coercing
         -- through newtypes is tantamount to using their constructors.
       ; [GlobalRdrElt] -> TcS ()
addUsedGREs [GlobalRdrElt]
gre_list
         -- If a newtype constructor was imported, don't warn about not
         -- importing it...
       ; (Name -> TcS ()) -> [Name] -> TcS ()
forall (t :: * -> *) (f :: * -> *) a b.
(Foldable t, Applicative f) =>
(a -> f b) -> t a -> f ()
traverse_ Name -> TcS ()
keepAlive ([Name] -> TcS ()) -> [Name] -> TcS ()
forall a b. (a -> b) -> a -> b
$ (GlobalRdrElt -> Name) -> [GlobalRdrElt] -> [Name]
forall a b. (a -> b) -> [a] -> [b]
map GlobalRdrElt -> Name
gre_name [GlobalRdrElt]
gre_list
         -- ...and similarly, if a newtype constructor was defined in the same
         -- module, don't warn about it being unused.
         -- See Note [Tracking unused binding and imports] in TcRnTypes.

       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
ty1' PredType
ps_ty2
                                     (TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
co) (Role -> PredType -> TcCoercion
mkTcReflCo Role
Representational PredType
ps_ty2)
       ; Bool
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc Bool
False CtEvidence
new_ev EqRel
ReprEq PredType
ty1' PredType
ty1' PredType
ty2 PredType
ps_ty2 }
  where
    gre_list :: [GlobalRdrElt]
gre_list = Bag GlobalRdrElt -> [GlobalRdrElt]
forall a. Bag a -> [a]
bagToList Bag GlobalRdrElt
gres

---------
-- ^ Decompose a type application.
-- All input types must be flat. See Note [Canonicalising type applications]
-- Nominal equality only!
can_eq_app :: CtEvidence       -- :: s1 t1 ~N s2 t2
           -> Xi -> Xi         -- s1 t1
           -> Xi -> Xi         -- s2 t2
           -> TcS (StopOrContinue Ct)

-- AppTys only decompose for nominal equality, so this case just leads
-- to an irreducible constraint; see typecheck/should_compile/T10494
-- See Note [Decomposing equality], note {4}
can_eq_app :: CtEvidence
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_app CtEvidence
ev PredType
s1 PredType
t1 PredType
s2 PredType
t2
  | CtDerived {} <- CtEvidence
ev
  = do { CtLoc -> [Role] -> [PredType] -> [PredType] -> TcS ()
unifyDeriveds CtLoc
loc [Role
Nominal, Role
Nominal] [PredType
s1, PredType
t1] [PredType
s2, PredType
t2]
       ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Decomposed [D] AppTy" }
  | CtWanted { ctev_dest :: CtEvidence -> TcEvDest
ctev_dest = TcEvDest
dest } <- CtEvidence
ev
  = do { TcCoercion
co_s <- CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
loc Role
Nominal PredType
s1 PredType
s2
       ; let arg_loc :: CtLoc
arg_loc
               | PredType -> Bool
isNextArgVisible PredType
s1 = CtLoc
loc
               | Bool
otherwise           = CtLoc -> (CtOrigin -> CtOrigin) -> CtLoc
updateCtLocOrigin CtLoc
loc CtOrigin -> CtOrigin
toInvisibleOrigin
       ; TcCoercion
co_t <- CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
arg_loc Role
Nominal PredType
t1 PredType
t2
       ; let co :: TcCoercion
co = TcCoercion -> TcCoercion -> TcCoercion
mkAppCo TcCoercion
co_s TcCoercion
co_t
       ; TcEvDest -> TcCoercion -> TcS ()
setWantedEq TcEvDest
dest TcCoercion
co
       ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Decomposed [W] AppTy" }

    -- If there is a ForAll/(->) mismatch, the use of the Left coercion
    -- below is ill-typed, potentially leading to a panic in splitTyConApp
    -- Test case: typecheck/should_run/Typeable1
    -- We could also include this mismatch check above (for W and D), but it's slow
    -- and we'll get a better error message not doing it
  | PredType
s1k PredType -> PredType -> Bool
`mismatches` PredType
s2k
  = CtEvidence -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqHardFailure CtEvidence
ev (PredType
s1 PredType -> PredType -> PredType
`mkAppTy` PredType
t1) (PredType
s2 PredType -> PredType -> PredType
`mkAppTy` PredType
t2)

  | CtGiven { ctev_evar :: CtEvidence -> TcTyVar
ctev_evar = TcTyVar
evar } <- CtEvidence
ev
  = do { let co :: TcCoercion
co   = TcTyVar -> TcCoercion
mkTcCoVarCo TcTyVar
evar
             co_s :: TcCoercion
co_s = LeftOrRight -> TcCoercion -> TcCoercion
mkTcLRCo LeftOrRight
CLeft  TcCoercion
co
             co_t :: TcCoercion
co_t = LeftOrRight -> TcCoercion -> TcCoercion
mkTcLRCo LeftOrRight
CRight TcCoercion
co
       ; CtEvidence
evar_s <- CtLoc -> (PredType, EvTerm) -> TcS CtEvidence
newGivenEvVar CtLoc
loc ( CtEvidence -> PredType -> PredType -> PredType
mkTcEqPredLikeEv CtEvidence
ev PredType
s1 PredType
s2
                                     , TcCoercion -> EvTerm
evCoercion TcCoercion
co_s )
       ; CtEvidence
evar_t <- CtLoc -> (PredType, EvTerm) -> TcS CtEvidence
newGivenEvVar CtLoc
loc ( CtEvidence -> PredType -> PredType -> PredType
mkTcEqPredLikeEv CtEvidence
ev PredType
t1 PredType
t2
                                     , TcCoercion -> EvTerm
evCoercion TcCoercion
co_t )
       ; [CtEvidence] -> TcS ()
emitWorkNC [CtEvidence
evar_t]
       ; CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqNC CtEvidence
evar_s EqRel
NomEq PredType
s1 PredType
s2 }

  where
    loc :: CtLoc
loc = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev

    s1k :: PredType
s1k = HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind PredType
s1
    s2k :: PredType
s2k = HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind PredType
s2

    PredType
k1 mismatches :: PredType -> PredType -> Bool
`mismatches` PredType
k2
      =  PredType -> Bool
isForAllTy PredType
k1 Bool -> Bool -> Bool
&& Bool -> Bool
not (PredType -> Bool
isForAllTy PredType
k2)
      Bool -> Bool -> Bool
|| Bool -> Bool
not (PredType -> Bool
isForAllTy PredType
k1) Bool -> Bool -> Bool
&& PredType -> Bool
isForAllTy PredType
k2

-----------------------
-- | Break apart an equality over a casted type
-- looking like   (ty1 |> co1) ~ ty2   (modulo a swap-flag)
canEqCast :: Bool         -- are both types flat?
          -> CtEvidence
          -> EqRel
          -> SwapFlag
          -> TcType -> Coercion   -- LHS (res. RHS), ty1 |> co1
          -> TcType -> TcType     -- RHS (res. LHS), ty2 both normal and pretty
          -> TcS (StopOrContinue Ct)
canEqCast :: Bool
-> CtEvidence
-> EqRel
-> SwapFlag
-> PredType
-> TcCoercion
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqCast Bool
flat CtEvidence
ev EqRel
eq_rel SwapFlag
swapped PredType
ty1 TcCoercion
co1 PredType
ty2 PredType
ps_ty2
  = do { String -> SDoc -> TcS ()
traceTcS String
"Decomposing cast" ([SDoc] -> SDoc
vcat [ CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev
                                           , PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty1 SDoc -> SDoc -> SDoc
<+> String -> SDoc
text String
"|>" SDoc -> SDoc -> SDoc
<+> TcCoercion -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcCoercion
co1
                                           , PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ps_ty2 ])
       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
ty1 PredType
ps_ty2
                                     (Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflRightCo Role
role PredType
ty1 TcCoercion
co1)
                                     (Role -> PredType -> TcCoercion
mkTcReflCo Role
role PredType
ps_ty2)
       ; Bool
-> CtEvidence
-> EqRel
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
can_eq_nc Bool
flat CtEvidence
new_ev EqRel
eq_rel PredType
ty1 PredType
ty1 PredType
ty2 PredType
ps_ty2 }
  where
    role :: Role
role = EqRel -> Role
eqRelRole EqRel
eq_rel

------------------------
canTyConApp :: CtEvidence -> EqRel
            -> TyCon -> [TcType]
            -> TyCon -> [TcType]
            -> TcS (StopOrContinue Ct)
-- See Note [Decomposing TyConApps]
canTyConApp :: CtEvidence
-> EqRel
-> TyCon
-> [PredType]
-> TyCon
-> [PredType]
-> TcS (StopOrContinue Ct)
canTyConApp CtEvidence
ev EqRel
eq_rel TyCon
tc1 [PredType]
tys1 TyCon
tc2 [PredType]
tys2
  | TyCon
tc1 TyCon -> TyCon -> Bool
forall a. Eq a => a -> a -> Bool
== TyCon
tc2
  , [PredType]
tys1 [PredType] -> [PredType] -> Bool
forall a b. [a] -> [b] -> Bool
`equalLength` [PredType]
tys2
  = do { InertSet
inerts <- TcS InertSet
getTcSInerts
       ; if InertSet -> Bool
can_decompose InertSet
inerts
         then do { String -> SDoc -> TcS ()
traceTcS String
"canTyConApp"
                       (CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev SDoc -> SDoc -> SDoc
$$ EqRel -> SDoc
forall a. Outputable a => a -> SDoc
ppr EqRel
eq_rel SDoc -> SDoc -> SDoc
$$ TyCon -> SDoc
forall a. Outputable a => a -> SDoc
ppr TyCon
tc1 SDoc -> SDoc -> SDoc
$$ [PredType] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [PredType]
tys1 SDoc -> SDoc -> SDoc
$$ [PredType] -> SDoc
forall a. Outputable a => a -> SDoc
ppr [PredType]
tys2)
                 ; CtEvidence -> EqRel -> TyCon -> [PredType] -> [PredType] -> TcS ()
canDecomposableTyConAppOK CtEvidence
ev EqRel
eq_rel TyCon
tc1 [PredType]
tys1 [PredType]
tys2
                 ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Decomposed TyConApp" }
         else CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqFailure CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ty2 }

  -- See Note [Skolem abstract data] (at tyConSkolem)
  | TyCon -> Bool
tyConSkolem TyCon
tc1 Bool -> Bool -> Bool
|| TyCon -> Bool
tyConSkolem TyCon
tc2
  = do { String -> SDoc -> TcS ()
traceTcS String
"canTyConApp: skolem abstract" (TyCon -> SDoc
forall a. Outputable a => a -> SDoc
ppr TyCon
tc1 SDoc -> SDoc -> SDoc
$$ TyCon -> SDoc
forall a. Outputable a => a -> SDoc
ppr TyCon
tc2)
       ; Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkIrredCt CtEvidence
ev) }

  -- Fail straight away for better error messages
  -- See Note [Use canEqFailure in canDecomposableTyConApp]
  | EqRel
eq_rel EqRel -> EqRel -> Bool
forall a. Eq a => a -> a -> Bool
== EqRel
ReprEq Bool -> Bool -> Bool
&& Bool -> Bool
not (TyCon -> Role -> Bool
isGenerativeTyCon TyCon
tc1 Role
Representational Bool -> Bool -> Bool
&&
                             TyCon -> Role -> Bool
isGenerativeTyCon TyCon
tc2 Role
Representational)
  = CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqFailure CtEvidence
ev EqRel
eq_rel PredType
ty1 PredType
ty2
  | Bool
otherwise
  = CtEvidence -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqHardFailure CtEvidence
ev PredType
ty1 PredType
ty2
  where
    ty1 :: PredType
ty1 = TyCon -> [PredType] -> PredType
mkTyConApp TyCon
tc1 [PredType]
tys1
    ty2 :: PredType
ty2 = TyCon -> [PredType] -> PredType
mkTyConApp TyCon
tc2 [PredType]
tys2

    loc :: CtLoc
loc  = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev
    pred :: PredType
pred = CtEvidence -> PredType
ctEvPred CtEvidence
ev

     -- See Note [Decomposing equality]
    can_decompose :: InertSet -> Bool
can_decompose InertSet
inerts
      =  TyCon -> Role -> Bool
isInjectiveTyCon TyCon
tc1 (EqRel -> Role
eqRelRole EqRel
eq_rel)
      Bool -> Bool -> Bool
|| (CtEvidence -> CtFlavour
ctEvFlavour CtEvidence
ev CtFlavour -> CtFlavour -> Bool
forall a. Eq a => a -> a -> Bool
/= CtFlavour
Given Bool -> Bool -> Bool
&& Cts -> Bool
forall a. Bag a -> Bool
isEmptyBag (CtLoc -> PredType -> InertSet -> Cts
matchableGivens CtLoc
loc PredType
pred InertSet
inerts))

{-
Note [Use canEqFailure in canDecomposableTyConApp]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
We must use canEqFailure, not canEqHardFailure here, because there is
the possibility of success if working with a representational equality.
Here is one case:

  type family TF a where TF Char = Bool
  data family DF a
  newtype instance DF Bool = MkDF Int

Suppose we are canonicalising (Int ~R DF (TF a)), where we don't yet
know `a`. This is *not* a hard failure, because we might soon learn
that `a` is, in fact, Char, and then the equality succeeds.

Here is another case:

  [G] Age ~R Int

where Age's constructor is not in scope. We don't want to report
an "inaccessible code" error in the context of this Given!

For example, see typecheck/should_compile/T10493, repeated here:

  import Data.Ord (Down)  -- no constructor

  foo :: Coercible (Down Int) Int => Down Int -> Int
  foo = coerce

That should compile, but only because we use canEqFailure and not
canEqHardFailure.

Note [Decomposing equality]
~~~~~~~~~~~~~~~~~~~~~~~~~~~
If we have a constraint (of any flavour and role) that looks like
T tys1 ~ T tys2, what can we conclude about tys1 and tys2? The answer,
of course, is "it depends". This Note spells it all out.

In this Note, "decomposition" refers to taking the constraint
  [fl] (T tys1 ~X T tys2)
(for some flavour fl and some role X) and replacing it with
  [fls'] (tys1 ~Xs' tys2)
where that notation indicates a list of new constraints, where the
new constraints may have different flavours and different roles.

The key property to consider is injectivity. When decomposing a Given the
decomposition is sound if and only if T is injective in all of its type
arguments. When decomposing a Wanted, the decomposition is sound (assuming the
correct roles in the produced equality constraints), but it may be a guess --
that is, an unforced decision by the constraint solver. Decomposing Wanteds
over injective TyCons does not entail guessing. But sometimes we want to
decompose a Wanted even when the TyCon involved is not injective! (See below.)

So, in broad strokes, we want this rule:

(*) Decompose a constraint (T tys1 ~X T tys2) if and only if T is injective
at role X.

Pursuing the details requires exploring three axes:
* Flavour: Given vs. Derived vs. Wanted
* Role: Nominal vs. Representational
* TyCon species: datatype vs. newtype vs. data family vs. type family vs. type variable

(So a type variable isn't a TyCon, but it's convenient to put the AppTy case
in the same table.)

Right away, we can say that Derived behaves just as Wanted for the purposes
of decomposition. The difference between Derived and Wanted is the handling of
evidence. Since decomposition in these cases isn't a matter of soundness but of
guessing, we want the same behavior regardless of evidence.

Here is a table (discussion following) detailing where decomposition of
   (T s1 ... sn) ~r (T t1 .. tn)
is allowed.  The first four lines (Data types ... type family) refer
to TyConApps with various TyCons T; the last line is for AppTy, where
there is presumably a type variable at the head, so it's actually
   (s s1 ... sn) ~r (t t1 .. tn)

NOMINAL               GIVEN                       WANTED

Datatype               YES                         YES
Newtype                YES                         YES
Data family            YES                         YES
Type family            YES, in injective args{1}   YES, in injective args{1}
Type variable          YES                         YES

REPRESENTATIONAL      GIVEN                       WANTED

Datatype               YES                         YES
Newtype                NO{2}                      MAYBE{2}
Data family            NO{3}                      MAYBE{3}
Type family             NO                          NO
Type variable          NO{4}                       NO{4}

{1}: Type families can be injective in some, but not all, of their arguments,
so we want to do partial decomposition. This is quite different than the way
other decomposition is done, where the decomposed equalities replace the original
one. We thus proceed much like we do with superclasses: emitting new Givens
when "decomposing" a partially-injective type family Given and new Deriveds
when "decomposing" a partially-injective type family Wanted. (As of the time of
writing, 13 June 2015, the implementation of injective type families has not
been merged, but it should be soon. Please delete this parenthetical if the
implementation is indeed merged.)

{2}: See Note [Decomposing newtypes at representational role]

{3}: Because of the possibility of newtype instances, we must treat
data families like newtypes. See also Note [Decomposing newtypes at
representational role]. See #10534 and test case
typecheck/should_fail/T10534.

{4}: Because type variables can stand in for newtypes, we conservatively do not
decompose AppTys over representational equality.

In the implementation of can_eq_nc and friends, we don't directly pattern
match using lines like in the tables above, as those tables don't cover
all cases (what about PrimTyCon? tuples?). Instead we just ask about injectivity,
boiling the tables above down to rule (*). The exceptions to rule (*) are for
injective type families, which are handled separately from other decompositions,
and the MAYBE entries above.

Note [Decomposing newtypes at representational role]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
This note discusses the 'newtype' line in the REPRESENTATIONAL table
in Note [Decomposing equality]. (At nominal role, newtypes are fully
decomposable.)

Here is a representative example of why representational equality over
newtypes is tricky:

  newtype Nt a = Mk Bool         -- NB: a is not used in the RHS,
  type role Nt representational  -- but the user gives it an R role anyway

If we have [W] Nt alpha ~R Nt beta, we *don't* want to decompose to
[W] alpha ~R beta, because it's possible that alpha and beta aren't
representationally equal. Here's another example.

  newtype Nt a = MkNt (Id a)
  type family Id a where Id a = a

  [W] Nt Int ~R Nt Age

Because of its use of a type family, Nt's parameter will get inferred to have
a nominal role. Thus, decomposing the wanted will yield [W] Int ~N Age, which
is unsatisfiable. Unwrapping, though, leads to a solution.

Conclusion:
 * Unwrap newtypes before attempting to decompose them.
   This is done in can_eq_nc'.

It all comes from the fact that newtypes aren't necessarily injective
w.r.t. representational equality.

Furthermore, as explained in Note [NthCo and newtypes] in TyCoRep, we can't use
NthCo on representational coercions over newtypes. NthCo comes into play
only when decomposing givens.

Conclusion:
 * Do not decompose [G] N s ~R N t

Is it sensible to decompose *Wanted* constraints over newtypes?  Yes!
It's the only way we could ever prove (IO Int ~R IO Age), recalling
that IO is a newtype.

However we must be careful.  Consider

  type role Nt representational

  [G] Nt a ~R Nt b       (1)
  [W] NT alpha ~R Nt b   (2)
  [W] alpha ~ a          (3)

If we focus on (3) first, we'll substitute in (2), and now it's
identical to the given (1), so we succeed.  But if we focus on (2)
first, and decompose it, we'll get (alpha ~R b), which is not soluble.
This is exactly like the question of overlapping Givens for class
constraints: see Note [Instance and Given overlap] in TcInteract.

Conclusion:
  * Decompose [W] N s ~R N t  iff there no given constraint that could
    later solve it.

-}

canDecomposableTyConAppOK :: CtEvidence -> EqRel
                          -> TyCon -> [TcType] -> [TcType]
                          -> TcS ()
-- Precondition: tys1 and tys2 are the same length, hence "OK"
canDecomposableTyConAppOK :: CtEvidence -> EqRel -> TyCon -> [PredType] -> [PredType] -> TcS ()
canDecomposableTyConAppOK CtEvidence
ev EqRel
eq_rel TyCon
tc [PredType]
tys1 [PredType]
tys2
  = ASSERT( tys1 `equalLength` tys2 )
    case CtEvidence
ev of
     CtDerived {}
        -> CtLoc -> [Role] -> [PredType] -> [PredType] -> TcS ()
unifyDeriveds CtLoc
loc [Role]
tc_roles [PredType]
tys1 [PredType]
tys2

     CtWanted { ctev_dest :: CtEvidence -> TcEvDest
ctev_dest = TcEvDest
dest }
                   -- new_locs and tc_roles are both infinite, so
                   -- we are guaranteed that cos has the same length
                   -- as tys1 and tys2
        -> do { [TcCoercion]
cos <- (CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion)
-> [CtLoc]
-> [Role]
-> [PredType]
-> [PredType]
-> TcS [TcCoercion]
forall (m :: * -> *) a b c d e.
Monad m =>
(a -> b -> c -> d -> m e) -> [a] -> [b] -> [c] -> [d] -> m [e]
zipWith4M CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted [CtLoc]
new_locs [Role]
tc_roles [PredType]
tys1 [PredType]
tys2
              ; TcEvDest -> TcCoercion -> TcS ()
setWantedEq TcEvDest
dest (HasDebugCallStack => Role -> TyCon -> [TcCoercion] -> TcCoercion
Role -> TyCon -> [TcCoercion] -> TcCoercion
mkTyConAppCo Role
role TyCon
tc [TcCoercion]
cos) }

     CtGiven { ctev_evar :: CtEvidence -> TcTyVar
ctev_evar = TcTyVar
evar }
        -> do { let ev_co :: TcCoercion
ev_co = TcTyVar -> TcCoercion
mkCoVarCo TcTyVar
evar
              ; [CtEvidence]
given_evs <- CtLoc -> [(PredType, EvTerm)] -> TcS [CtEvidence]
newGivenEvVars CtLoc
loc ([(PredType, EvTerm)] -> TcS [CtEvidence])
-> [(PredType, EvTerm)] -> TcS [CtEvidence]
forall a b. (a -> b) -> a -> b
$
                             [ ( Role -> PredType -> PredType -> PredType
mkPrimEqPredRole Role
r PredType
ty1 PredType
ty2
                               , TcCoercion -> EvTerm
evCoercion (TcCoercion -> EvTerm) -> TcCoercion -> EvTerm
forall a b. (a -> b) -> a -> b
$ HasDebugCallStack => Role -> Int -> TcCoercion -> TcCoercion
Role -> Int -> TcCoercion -> TcCoercion
mkNthCo Role
r Int
i TcCoercion
ev_co )
                             | (Role
r, PredType
ty1, PredType
ty2, Int
i) <- [Role]
-> [PredType]
-> [PredType]
-> [Int]
-> [(Role, PredType, PredType, Int)]
forall a b c d. [a] -> [b] -> [c] -> [d] -> [(a, b, c, d)]
zip4 [Role]
tc_roles [PredType]
tys1 [PredType]
tys2 [Int
0..]
                             , Role
r Role -> Role -> Bool
forall a. Eq a => a -> a -> Bool
/= Role
Phantom
                             , Bool -> Bool
not (PredType -> Bool
isCoercionTy PredType
ty1) Bool -> Bool -> Bool
&& Bool -> Bool
not (PredType -> Bool
isCoercionTy PredType
ty2) ]
              ; [CtEvidence] -> TcS ()
emitWorkNC [CtEvidence]
given_evs }
  where
    loc :: CtLoc
loc        = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev
    role :: Role
role       = EqRel -> Role
eqRelRole EqRel
eq_rel

      -- infinite, as tyConRolesX returns an infinite tail of Nominal
    tc_roles :: [Role]
tc_roles   = Role -> TyCon -> [Role]
tyConRolesX Role
role TyCon
tc

      -- Add nuances to the location during decomposition:
      --  * if the argument is a kind argument, remember this, so that error
      --    messages say "kind", not "type". This is determined based on whether
      --    the corresponding tyConBinder is named (that is, dependent)
      --  * if the argument is invisible, note this as well, again by
      --    looking at the corresponding binder
      -- For oversaturated tycons, we need the (repeat loc) tail, which doesn't
      -- do either of these changes. (Forgetting to do so led to #16188)
      --
      -- NB: infinite in length
    new_locs :: [CtLoc]
new_locs = [ CtLoc
new_loc
               | TyConBinder
bndr <- TyCon -> [TyConBinder]
tyConBinders TyCon
tc
               , let new_loc0 :: CtLoc
new_loc0 | TyConBinder -> Bool
isNamedTyConBinder TyConBinder
bndr = CtLoc -> CtLoc
toKindLoc CtLoc
loc
                              | Bool
otherwise               = CtLoc
loc
                     new_loc :: CtLoc
new_loc  | TyConBinder -> Bool
forall tv. VarBndr tv TyConBndrVis -> Bool
isVisibleTyConBinder TyConBinder
bndr
                              = CtLoc -> (CtOrigin -> CtOrigin) -> CtLoc
updateCtLocOrigin CtLoc
new_loc0 CtOrigin -> CtOrigin
toInvisibleOrigin
                              | Bool
otherwise
                              = CtLoc
new_loc0 ]
               [CtLoc] -> [CtLoc] -> [CtLoc]
forall a. [a] -> [a] -> [a]
++ CtLoc -> [CtLoc]
forall a. a -> [a]
repeat CtLoc
loc

-- | Call when canonicalizing an equality fails, but if the equality is
-- representational, there is some hope for the future.
-- Examples in Note [Use canEqFailure in canDecomposableTyConApp]
canEqFailure :: CtEvidence -> EqRel
             -> TcType -> TcType -> TcS (StopOrContinue Ct)
canEqFailure :: CtEvidence
-> EqRel -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqFailure CtEvidence
ev EqRel
NomEq PredType
ty1 PredType
ty2
  = CtEvidence -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqHardFailure CtEvidence
ev PredType
ty1 PredType
ty2
canEqFailure CtEvidence
ev EqRel
ReprEq PredType
ty1 PredType
ty2
  = do { (PredType
xi1, TcCoercion
co1) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_FlattenAll CtEvidence
ev PredType
ty1
       ; (PredType
xi2, TcCoercion
co2) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_FlattenAll CtEvidence
ev PredType
ty2
            -- We must flatten the types before putting them in the
            -- inert set, so that we are sure to kick them out when
            -- new equalities become available
       ; String -> SDoc -> TcS ()
traceTcS String
"canEqFailure with ReprEq" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
         [SDoc] -> SDoc
vcat [ CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty1, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
ty2, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
xi1, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
xi2 ]
       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
NotSwapped PredType
xi1 PredType
xi2 TcCoercion
co1 TcCoercion
co2
       ; Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkIrredCt CtEvidence
new_ev) }

-- | Call when canonicalizing an equality fails with utterly no hope.
canEqHardFailure :: CtEvidence
                 -> TcType -> TcType -> TcS (StopOrContinue Ct)
-- See Note [Make sure that insolubles are fully rewritten]
canEqHardFailure :: CtEvidence -> PredType -> PredType -> TcS (StopOrContinue Ct)
canEqHardFailure CtEvidence
ev PredType
ty1 PredType
ty2
  = do { (PredType
s1, TcCoercion
co1) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_SubstOnly CtEvidence
ev PredType
ty1
       ; (PredType
s2, TcCoercion
co2) <- FlattenMode -> CtEvidence -> PredType -> TcS (PredType, TcCoercion)
flatten FlattenMode
FM_SubstOnly CtEvidence
ev PredType
ty2
       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
NotSwapped PredType
s1 PredType
s2 TcCoercion
co1 TcCoercion
co2
       ; Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkInsolubleCt CtEvidence
new_ev) }

{-
Note [Decomposing TyConApps]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~
If we see (T s1 t1 ~ T s2 t2), then we can just decompose to
  (s1 ~ s2, t1 ~ t2)
and push those back into the work list.  But if
  s1 = K k1    s2 = K k2
then we will just decomopose s1~s2, and it might be better to
do so on the spot.  An important special case is where s1=s2,
and we get just Refl.

So canDecomposableTyCon is a fast-path decomposition that uses
unifyWanted etc to short-cut that work.

Note [Canonicalising type applications]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Given (s1 t1) ~ ty2, how should we proceed?
The simple things is to see if ty2 is of form (s2 t2), and
decompose.  By this time s1 and s2 can't be saturated type
function applications, because those have been dealt with
by an earlier equation in can_eq_nc, so it is always sound to
decompose.

However, over-eager decomposition gives bad error messages
for things like
   a b ~ Maybe c
   e f ~ p -> q
Suppose (in the first example) we already know a~Array.  Then if we
decompose the application eagerly, yielding
   a ~ Maybe
   b ~ c
we get an error        "Can't match Array ~ Maybe",
but we'd prefer to get "Can't match Array b ~ Maybe c".

So instead can_eq_wanted_app flattens the LHS and RHS, in the hope of
replacing (a b) by (Array b), before using try_decompose_app to
decompose it.

Note [Make sure that insolubles are fully rewritten]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
When an equality fails, we still want to rewrite the equality
all the way down, so that it accurately reflects
 (a) the mutable reference substitution in force at start of solving
 (b) any ty-binds in force at this point in solving
See Note [Rewrite insolubles] in TcSMonad.
And if we don't do this there is a bad danger that
TcSimplify.applyTyVarDefaulting will find a variable
that has in fact been substituted.

Note [Do not decompose Given polytype equalities]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Consider [G] (forall a. t1 ~ forall a. t2).  Can we decompose this?
No -- what would the evidence look like?  So instead we simply discard
this given evidence.


Note [Combining insoluble constraints]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
As this point we have an insoluble constraint, like Int~Bool.

 * If it is Wanted, delete it from the cache, so that subsequent
   Int~Bool constraints give rise to separate error messages

 * But if it is Derived, DO NOT delete from cache.  A class constraint
   may get kicked out of the inert set, and then have its functional
   dependency Derived constraints generated a second time. In that
   case we don't want to get two (or more) error messages by
   generating two (or more) insoluble fundep constraints from the same
   class constraint.

Note [No top-level newtypes on RHS of representational equalities]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
Suppose we're in this situation:

 work item:  [W] c1 : a ~R b
     inert:  [G] c2 : b ~R Id a

where
  newtype Id a = Id a

We want to make sure canEqTyVar sees [W] a ~R a, after b is flattened
and the Id newtype is unwrapped. This is assured by requiring only flat
types in canEqTyVar *and* having the newtype-unwrapping check above
the tyvar check in can_eq_nc.

Note [Occurs check error]
~~~~~~~~~~~~~~~~~~~~~~~~~
If we have an occurs check error, are we necessarily hosed? Say our
tyvar is tv1 and the type it appears in is xi2. Because xi2 is function
free, then if we're computing w.r.t. nominal equality, then, yes, we're
hosed. Nothing good can come from (a ~ [a]). If we're computing w.r.t.
representational equality, this is a little subtler. Once again, (a ~R [a])
is a bad thing, but (a ~R N a) for a newtype N might be just fine. This
means also that (a ~ b a) might be fine, because `b` might become a newtype.

So, we must check: does tv1 appear in xi2 under any type constructor
that is generative w.r.t. representational equality? That's what
isInsolubleOccursCheck does.

See also #10715, which induced this addition.

Note [canCFunEqCan]
~~~~~~~~~~~~~~~~~~~
Flattening the arguments to a type family can change the kind of the type
family application. As an easy example, consider (Any k) where (k ~ Type)
is in the inert set. The original (Any k :: k) becomes (Any Type :: Type).
The problem here is that the fsk in the CFunEqCan will have the old kind.

The solution is to come up with a new fsk/fmv of the right kind. For
givens, this is easy: just introduce a new fsk and update the flat-cache
with the new one. For wanteds, we want to solve the old one if favor of
the new one, so we use dischargeFmv. This also kicks out constraints
from the inert set; this behavior is correct, as the kind-change may
allow more constraints to be solved.

We use `isTcReflexiveCo`, to ensure that we only use the hetero-kinded case
if we really need to.  Of course `flattenArgsNom` should return `Refl`
whenever possible, but #15577 was an infinite loop because even
though the coercion was homo-kinded, `kind_co` was not `Refl`, so we
made a new (identical) CFunEqCan, and then the entire process repeated.
-}

canCFunEqCan :: CtEvidence
             -> TyCon -> [TcType]   -- LHS
             -> TcTyVar             -- RHS
             -> TcS (StopOrContinue Ct)
-- ^ Canonicalise a CFunEqCan.  We know that
--     the arg types are already flat,
-- and the RHS is a fsk, which we must *not* substitute.
-- So just substitute in the LHS
canCFunEqCan :: CtEvidence
-> TyCon -> [PredType] -> TcTyVar -> TcS (StopOrContinue Ct)
canCFunEqCan CtEvidence
ev TyCon
fn [PredType]
tys TcTyVar
fsk
  = do { ([PredType]
tys', [TcCoercion]
cos, TcCoercion
kind_co) <- CtEvidence
-> TyCon
-> [PredType]
-> TcS ([PredType], [TcCoercion], TcCoercion)
flattenArgsNom CtEvidence
ev TyCon
fn [PredType]
tys
                        -- cos :: tys' ~ tys

       ; let lhs_co :: TcCoercion
lhs_co  = Role -> TyCon -> [TcCoercion] -> TcCoercion
mkTcTyConAppCo Role
Nominal TyCon
fn [TcCoercion]
cos
                        -- :: F tys' ~ F tys
             new_lhs :: PredType
new_lhs = TyCon -> [PredType] -> PredType
mkTyConApp TyCon
fn [PredType]
tys'

             flav :: CtFlavour
flav    = CtEvidence -> CtFlavour
ctEvFlavour CtEvidence
ev
       ; (CtEvidence
ev', TcTyVar
fsk')
           <- if TcCoercion -> Bool
isTcReflexiveCo TcCoercion
kind_co   -- See Note [canCFunEqCan]
              then do { String -> SDoc -> TcS ()
traceTcS String
"canCFunEqCan: refl" (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
new_lhs)
                      ; let fsk_ty :: PredType
fsk_ty = TcTyVar -> PredType
mkTyVarTy TcTyVar
fsk
                      ; CtEvidence
ev' <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
NotSwapped PredType
new_lhs PredType
fsk_ty
                                                 TcCoercion
lhs_co (PredType -> TcCoercion
mkTcNomReflCo PredType
fsk_ty)
                      ; (CtEvidence, TcTyVar) -> TcS (CtEvidence, TcTyVar)
forall (m :: * -> *) a. Monad m => a -> m a
return (CtEvidence
ev', TcTyVar
fsk) }
              else do { String -> SDoc -> TcS ()
traceTcS String
"canCFunEqCan: non-refl" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
                        [SDoc] -> SDoc
vcat [ String -> SDoc
text String
"Kind co:" SDoc -> SDoc -> SDoc
<+> TcCoercion -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcCoercion
kind_co
                             , String -> SDoc
text String
"RHS:" SDoc -> SDoc -> SDoc
<+> TcTyVar -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcTyVar
fsk SDoc -> SDoc -> SDoc
<+> SDoc
dcolon SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr (TcTyVar -> PredType
tyVarKind TcTyVar
fsk)
                             , String -> SDoc
text String
"LHS:" SDoc -> SDoc -> SDoc
<+> SDoc -> Int -> SDoc -> SDoc
hang (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr (TyCon -> [PredType] -> PredType
mkTyConApp TyCon
fn [PredType]
tys))
                                                  Int
2 (SDoc
dcolon SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr (HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind (TyCon -> [PredType] -> PredType
mkTyConApp TyCon
fn [PredType]
tys)))
                             , String -> SDoc
text String
"New LHS" SDoc -> SDoc -> SDoc
<+> SDoc -> Int -> SDoc -> SDoc
hang (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
new_lhs)
                                                     Int
2 (SDoc
dcolon SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr (HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind PredType
new_lhs)) ]
                      ; (CtEvidence
ev', TcCoercion
new_co, TcTyVar
new_fsk)
                          <- CtFlavour
-> CtLoc
-> TyCon
-> [PredType]
-> TcS (CtEvidence, TcCoercion, TcTyVar)
newFlattenSkolem CtFlavour
flav (CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev) TyCon
fn [PredType]
tys'
                      ; let xi :: PredType
xi = TcTyVar -> PredType
mkTyVarTy TcTyVar
new_fsk PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
kind_co
                               -- sym lhs_co :: F tys ~ F tys'
                               -- new_co     :: F tys' ~ new_fsk
                               -- co         :: F tys ~ (new_fsk |> kind_co)
                            co :: TcCoercion
co = TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
lhs_co TcCoercion -> TcCoercion -> TcCoercion
`mkTcTransCo`
                                 Role -> PredType -> TcCoercion -> TcCoercion -> TcCoercion
mkTcCoherenceRightCo Role
Nominal
                                                      (TcTyVar -> PredType
mkTyVarTy TcTyVar
new_fsk)
                                                      TcCoercion
kind_co
                                                      TcCoercion
new_co

                      ; String -> SDoc -> TcS ()
traceTcS String
"Discharging fmv/fsk due to hetero flattening" (CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev)
                      ; CtEvidence -> TcTyVar -> TcCoercion -> PredType -> TcS ()
dischargeFunEq CtEvidence
ev TcTyVar
fsk TcCoercion
co PredType
xi
                      ; (CtEvidence, TcTyVar) -> TcS (CtEvidence, TcTyVar)
forall (m :: * -> *) a. Monad m => a -> m a
return (CtEvidence
ev', TcTyVar
new_fsk) }

       ; TyCon -> [PredType] -> (TcCoercion, PredType, CtFlavour) -> TcS ()
extendFlatCache TyCon
fn [PredType]
tys' (HasDebugCallStack => CtEvidence -> TcCoercion
CtEvidence -> TcCoercion
ctEvCoercion CtEvidence
ev', TcTyVar -> PredType
mkTyVarTy TcTyVar
fsk', CtEvidence -> CtFlavour
ctEvFlavour CtEvidence
ev')
       ; Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CFunEqCan :: CtEvidence -> TyCon -> [PredType] -> TcTyVar -> Ct
CFunEqCan { cc_ev :: CtEvidence
cc_ev = CtEvidence
ev', cc_fun :: TyCon
cc_fun = TyCon
fn
                                 , cc_tyargs :: [PredType]
cc_tyargs = [PredType]
tys', cc_fsk :: TcTyVar
cc_fsk = TcTyVar
fsk' }) }

---------------------
canEqTyVar :: CtEvidence          -- ev :: lhs ~ rhs
           -> EqRel -> SwapFlag
           -> TcTyVar               -- tv1
           -> TcType                -- lhs: pretty lhs, already flat
           -> TcType -> TcType      -- rhs: already flat
           -> TcS (StopOrContinue Ct)
canEqTyVar :: CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVar CtEvidence
ev EqRel
eq_rel SwapFlag
swapped TcTyVar
tv1 PredType
ps_xi1 PredType
xi2 PredType
ps_xi2
  | PredType
k1 HasDebugCallStack => PredType -> PredType -> Bool
PredType -> PredType -> Bool
`tcEqType` PredType
k2
  = CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVarHomo CtEvidence
ev EqRel
eq_rel SwapFlag
swapped TcTyVar
tv1 PredType
ps_xi1 PredType
xi2 PredType
ps_xi2

  -- So the LHS and RHS don't have equal kinds
  -- Note [Flattening] in TcFlatten gives us (F2), which says that
  -- flattening is always homogeneous (doesn't change kinds). But
  -- perhaps by flattening the kinds of the two sides of the equality
  -- at hand makes them equal. So let's try that.
  | Bool
otherwise
  = do { (PredType
flat_k1, TcCoercion
k1_co) <- CtLoc -> CtFlavour -> PredType -> TcS (PredType, TcCoercion)
flattenKind CtLoc
loc CtFlavour
flav PredType
k1  -- k1_co :: flat_k1 ~N kind(xi1)
       ; (PredType
flat_k2, TcCoercion
k2_co) <- CtLoc -> CtFlavour -> PredType -> TcS (PredType, TcCoercion)
flattenKind CtLoc
loc CtFlavour
flav PredType
k2  -- k2_co :: flat_k2 ~N kind(xi2)
       ; String -> SDoc -> TcS ()
traceTcS String
"canEqTyVar tried flattening kinds"
                  ([SDoc] -> SDoc
vcat [ [SDoc] -> SDoc
sep [ SDoc -> SDoc
parens (TcTyVar -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcTyVar
tv1 SDoc -> SDoc -> SDoc
<+> SDoc
dcolon SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
k1)
                              , String -> SDoc
text String
"~"
                              , SDoc -> SDoc
parens (PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
xi2 SDoc -> SDoc -> SDoc
<+> SDoc
dcolon SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
k2) ]
                        , PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
flat_k1
                        , TcCoercion -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcCoercion
k1_co
                        , PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
flat_k2
                        , TcCoercion -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcCoercion
k2_co ])

         -- We know the LHS is a tyvar. So let's dump all the coercions on the RHS
         -- If flat_k1 == flat_k2, let's dump all the coercions on the RHS and
         -- then call canEqTyVarHomo. If they don't equal, just rewriteEqEvidence
         -- (as an optimization, so that we don't have to flatten the kinds again)
         -- and then emit a kind equality in canEqTyVarHetero.
         -- See Note [Equalities with incompatible kinds]

       ; let role :: Role
role = EqRel -> Role
eqRelRole EqRel
eq_rel
       ; if PredType
flat_k1 HasDebugCallStack => PredType -> PredType -> Bool
PredType -> PredType -> Bool
`tcEqType` PredType
flat_k2
         then do { let rhs_kind_co :: TcCoercion
rhs_kind_co = TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
k2_co TcCoercion -> TcCoercion -> TcCoercion
`mkTcTransCo` TcCoercion
k1_co
                         -- :: kind(xi2) ~N kind(xi1)

                       new_rhs :: PredType
new_rhs     = PredType
xi2 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
rhs_kind_co
                       ps_rhs :: PredType
ps_rhs      = PredType
ps_xi2 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
rhs_kind_co
                       rhs_co :: TcCoercion
rhs_co      = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflLeftCo Role
role PredType
xi2 TcCoercion
rhs_kind_co

                 ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
xi1 PredType
new_rhs
                                               (Role -> PredType -> TcCoercion
mkTcReflCo Role
role PredType
xi1) TcCoercion
rhs_co
                       -- NB: rewriteEqEvidence executes a swap, if any, so we're
                       -- NotSwapped now.
                 ; CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVarHomo CtEvidence
new_ev EqRel
eq_rel SwapFlag
NotSwapped TcTyVar
tv1 PredType
ps_xi1 PredType
new_rhs PredType
ps_rhs }
         else
    do { let sym_k1_co :: TcCoercion
sym_k1_co = TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
k1_co  -- :: kind(xi1) ~N flat_k1
             sym_k2_co :: TcCoercion
sym_k2_co = TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
k2_co  -- :: kind(xi2) ~N flat_k2

             new_lhs :: PredType
new_lhs = PredType
xi1 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
sym_k1_co  -- :: flat_k1
             new_rhs :: PredType
new_rhs = PredType
xi2 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
sym_k2_co  -- :: flat_k2
             ps_rhs :: PredType
ps_rhs  = PredType
ps_xi2 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
sym_k2_co

             lhs_co :: TcCoercion
lhs_co = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflLeftCo Role
role PredType
xi1 TcCoercion
sym_k1_co
             rhs_co :: TcCoercion
rhs_co = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflLeftCo Role
role PredType
xi2 TcCoercion
sym_k2_co
               -- lhs_co :: (xi1 |> sym k1_co) ~ xi1
               -- rhs_co :: (xi2 |> sym k2_co) ~ xi2

       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
new_lhs PredType
new_rhs TcCoercion
lhs_co TcCoercion
rhs_co
         -- no longer swapped, due to rewriteEqEvidence
       ; CtEvidence
-> EqRel
-> TcTyVar
-> TcCoercion
-> PredType
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVarHetero CtEvidence
new_ev EqRel
eq_rel TcTyVar
tv1 TcCoercion
sym_k1_co PredType
flat_k1 PredType
ps_xi1
                                        PredType
new_rhs PredType
flat_k2 PredType
ps_rhs } }
  where
    xi1 :: PredType
xi1 = TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1

    k1 :: PredType
k1 = TcTyVar -> PredType
tyVarKind TcTyVar
tv1
    k2 :: PredType
k2 = HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind PredType
xi2

    loc :: CtLoc
loc  = CtEvidence -> CtLoc
ctEvLoc CtEvidence
ev
    flav :: CtFlavour
flav = CtEvidence -> CtFlavour
ctEvFlavour CtEvidence
ev

canEqTyVarHetero :: CtEvidence   -- :: (tv1 |> co1 :: ki1) ~ (xi2 :: ki2)
                 -> EqRel
                 -> TcTyVar -> TcCoercionN -> TcKind  -- tv1 |> co1 :: ki1
                 -> TcType            -- pretty tv1 (*without* the coercion)
                 -> TcType -> TcKind  -- xi2 :: ki2
                 -> TcType            -- pretty xi2
                 -> TcS (StopOrContinue Ct)
canEqTyVarHetero :: CtEvidence
-> EqRel
-> TcTyVar
-> TcCoercion
-> PredType
-> PredType
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVarHetero CtEvidence
ev EqRel
eq_rel TcTyVar
tv1 TcCoercion
co1 PredType
ki1 PredType
ps_tv1 PredType
xi2 PredType
ki2 PredType
ps_xi2
  -- See Note [Equalities with incompatible kinds]
  | CtGiven { ctev_evar :: CtEvidence -> TcTyVar
ctev_evar = TcTyVar
evar } <- CtEvidence
ev
    -- unswapped: tm :: (lhs :: ki1) ~ (rhs :: ki2)
    -- swapped  : tm :: (rhs :: ki2) ~ (lhs :: ki1)
  = do { let kind_co :: TcCoercion
kind_co = TcCoercion -> TcCoercion
mkTcKindCo (TcTyVar -> TcCoercion
mkTcCoVarCo TcTyVar
evar)
       ; CtEvidence
kind_ev <- CtLoc -> (PredType, EvTerm) -> TcS CtEvidence
newGivenEvVar CtLoc
kind_loc (PredType
kind_pty, TcCoercion -> EvTerm
evCoercion TcCoercion
kind_co)
       ; let  -- kind_ev :: (ki1 :: *) ~ (ki2 :: *)   (whether swapped or not)
              -- co1     :: kind(tv1) ~N ki1
              -- homo_co :: ki2 ~N kind(tv1)
             homo_co :: TcCoercion
homo_co = TcCoercion -> TcCoercion
mkTcSymCo (HasDebugCallStack => CtEvidence -> TcCoercion
CtEvidence -> TcCoercion
ctEvCoercion CtEvidence
kind_ev) TcCoercion -> TcCoercion -> TcCoercion
`mkTcTransCo` TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
co1
             rhs' :: PredType
rhs'    = PredType -> TcCoercion -> PredType
mkCastTy PredType
xi2 TcCoercion
homo_co     -- :: kind(tv1)
             ps_rhs' :: PredType
ps_rhs' = PredType -> TcCoercion -> PredType
mkCastTy PredType
ps_xi2 TcCoercion
homo_co  -- :: kind(tv1)
             rhs_co :: TcCoercion
rhs_co  = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflLeftCo Role
role PredType
xi2 TcCoercion
homo_co
               -- rhs_co :: (xi2 |> homo_co :: kind(tv1)) ~ xi2

             lhs' :: PredType
lhs'   = TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1       -- :: kind(tv1)
             lhs_co :: TcCoercion
lhs_co = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflRightCo Role
role PredType
lhs' TcCoercion
co1
               -- lhs_co :: (tv1 :: kind(tv1)) ~ (tv1 |> co1 :: ki1)

       ; String -> SDoc -> TcS ()
traceTcS String
"Hetero equality gives rise to given kind equality"
           (CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
kind_ev SDoc -> SDoc -> SDoc
<+> SDoc
dcolon SDoc -> SDoc -> SDoc
<+> PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
kind_pty)
       ; [CtEvidence] -> TcS ()
emitWorkNC [CtEvidence
kind_ev]
       ; CtEvidence
type_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
NotSwapped PredType
lhs' PredType
rhs' TcCoercion
lhs_co TcCoercion
rhs_co
       ; CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVarHomo CtEvidence
type_ev EqRel
eq_rel SwapFlag
NotSwapped TcTyVar
tv1 PredType
ps_tv1 PredType
rhs' PredType
ps_rhs' }

  -- See Note [Equalities with incompatible kinds]
  | Bool
otherwise   -- Wanted and Derived
                -- NB: all kind equalities are Nominal
  = do { CtLoc -> Role -> PredType -> PredType -> TcS ()
emitNewDerivedEq CtLoc
kind_loc Role
Nominal PredType
ki1 PredType
ki2
             -- kind_ev :: (ki1 :: *) ~ (ki2 :: *)
       ; String -> SDoc -> TcS ()
traceTcS String
"Hetero equality gives rise to derived kind equality" (SDoc -> TcS ()) -> SDoc -> TcS ()
forall a b. (a -> b) -> a -> b
$
           CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev
       ; Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkIrredCt CtEvidence
ev) }

  where
    kind_pty :: PredType
kind_pty = PredType -> PredType -> PredType -> PredType -> PredType
mkHeteroPrimEqPred PredType
liftedTypeKind PredType
liftedTypeKind PredType
ki1 PredType
ki2
    kind_loc :: CtLoc
kind_loc = PredType -> PredType -> CtLoc -> CtLoc
mkKindLoc (TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
co1) PredType
xi2 CtLoc
loc

    loc :: CtLoc
loc  = CtEvidence -> CtLoc
ctev_loc CtEvidence
ev
    role :: Role
role = EqRel -> Role
eqRelRole EqRel
eq_rel

-- guaranteed that tcTypeKind lhs == tcTypeKind rhs
canEqTyVarHomo :: CtEvidence
               -> EqRel -> SwapFlag
               -> TcTyVar                -- lhs: tv1
               -> TcType                 -- pretty lhs, flat
               -> TcType -> TcType       -- rhs, flat
               -> TcS (StopOrContinue Ct)
canEqTyVarHomo :: CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> PredType
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVarHomo CtEvidence
ev EqRel
eq_rel SwapFlag
swapped TcTyVar
tv1 PredType
ps_xi1 PredType
xi2 PredType
_
  | Just (TcTyVar
tv2, TcCoercion
_) <- PredType -> Maybe (TcTyVar, TcCoercion)
tcGetCastedTyVar_maybe PredType
xi2
  , TcTyVar
tv1 TcTyVar -> TcTyVar -> Bool
forall a. Eq a => a -> a -> Bool
== TcTyVar
tv2
  = CtEvidence -> EqRel -> PredType -> TcS (StopOrContinue Ct)
canEqReflexive CtEvidence
ev EqRel
eq_rel (TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1)
    -- we don't need to check co because it must be reflexive

  | Just (TcTyVar
tv2, TcCoercion
co2) <- PredType -> Maybe (TcTyVar, TcCoercion)
tcGetCastedTyVar_maybe PredType
xi2
  , TcTyVar -> TcTyVar -> Bool
swapOverTyVars TcTyVar
tv1 TcTyVar
tv2
  = do { String -> SDoc -> TcS ()
traceTcS String
"canEqTyVar swapOver" (TcTyVar -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcTyVar
tv1 SDoc -> SDoc -> SDoc
$$ TcTyVar -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcTyVar
tv2 SDoc -> SDoc -> SDoc
$$ SwapFlag -> SDoc
forall a. Outputable a => a -> SDoc
ppr SwapFlag
swapped)
         -- FM_Avoid commented out: see Note [Lazy flattening] in TcFlatten
         -- let fmode = FE { fe_ev = ev, fe_mode = FM_Avoid tv1' True }
         -- Flatten the RHS less vigorously, to avoid gratuitous flattening
         -- True <=> xi2 should not itself be a type-function application

       ; let role :: Role
role    = EqRel -> Role
eqRelRole EqRel
eq_rel
             sym_co2 :: TcCoercion
sym_co2 = TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
co2
             ty1 :: PredType
ty1     = TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1
             new_lhs :: PredType
new_lhs = PredType
ty1 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
sym_co2
             lhs_co :: TcCoercion
lhs_co  = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflLeftCo Role
role PredType
ty1 TcCoercion
sym_co2

             new_rhs :: PredType
new_rhs = TcTyVar -> PredType
mkTyVarTy TcTyVar
tv2
             rhs_co :: TcCoercion
rhs_co  = Role -> PredType -> TcCoercion -> TcCoercion
mkTcGReflRightCo Role
role PredType
new_rhs TcCoercion
co2

       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
new_lhs PredType
new_rhs TcCoercion
lhs_co TcCoercion
rhs_co

       ; DynFlags
dflags <- TcS DynFlags
forall (m :: * -> *). HasDynFlags m => m DynFlags
getDynFlags
       ; DynFlags
-> CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVar2 DynFlags
dflags CtEvidence
new_ev EqRel
eq_rel SwapFlag
IsSwapped TcTyVar
tv2 (PredType
ps_xi1 PredType -> TcCoercion -> PredType
`mkCastTy` TcCoercion
sym_co2) }

canEqTyVarHomo CtEvidence
ev EqRel
eq_rel SwapFlag
swapped TcTyVar
tv1 PredType
_ PredType
_ PredType
ps_xi2
  = do { DynFlags
dflags <- TcS DynFlags
forall (m :: * -> *). HasDynFlags m => m DynFlags
getDynFlags
       ; DynFlags
-> CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVar2 DynFlags
dflags CtEvidence
ev EqRel
eq_rel SwapFlag
swapped TcTyVar
tv1 PredType
ps_xi2 }

-- The RHS here is either not a casted tyvar, or it's a tyvar but we want
-- to rewrite the LHS to the RHS (as per swapOverTyVars)
canEqTyVar2 :: DynFlags
            -> CtEvidence   -- lhs ~ rhs (or, if swapped, orhs ~ olhs)
            -> EqRel
            -> SwapFlag
            -> TcTyVar                  -- lhs = tv, flat
            -> TcType                   -- rhs, flat
            -> TcS (StopOrContinue Ct)
-- LHS is an inert type variable,
-- and RHS is fully rewritten, but with type synonyms
-- preserved as much as possible
canEqTyVar2 :: DynFlags
-> CtEvidence
-> EqRel
-> SwapFlag
-> TcTyVar
-> PredType
-> TcS (StopOrContinue Ct)
canEqTyVar2 DynFlags
dflags CtEvidence
ev EqRel
eq_rel SwapFlag
swapped TcTyVar
tv1 PredType
rhs
  | Just PredType
rhs' <- DynFlags -> TcTyVar -> PredType -> Maybe PredType
metaTyVarUpdateOK DynFlags
dflags TcTyVar
tv1 PredType
rhs  -- No occurs check
     -- Must do the occurs check even on tyvar/tyvar
     -- equalities, in case have  x ~ (y :: ..x...)
     -- #12593
  = do { CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
lhs PredType
rhs' TcCoercion
rewrite_co1 TcCoercion
rewrite_co2
       ; Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CTyEqCan :: CtEvidence -> TcTyVar -> PredType -> EqRel -> Ct
CTyEqCan { cc_ev :: CtEvidence
cc_ev = CtEvidence
new_ev, cc_tyvar :: TcTyVar
cc_tyvar = TcTyVar
tv1
                                , cc_rhs :: PredType
cc_rhs = PredType
rhs', cc_eq_rel :: EqRel
cc_eq_rel = EqRel
eq_rel }) }

  | Bool
otherwise  -- For some reason (occurs check, or forall) we can't unify
               -- We must not use it for further rewriting!
  = do { String -> SDoc -> TcS ()
traceTcS String
"canEqTyVar2 can't unify" (TcTyVar -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcTyVar
tv1 SDoc -> SDoc -> SDoc
$$ PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
rhs)
       ; CtEvidence
new_ev <- CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
ev SwapFlag
swapped PredType
lhs PredType
rhs TcCoercion
rewrite_co1 TcCoercion
rewrite_co2
       ; if EqRel -> TcTyVar -> PredType -> Bool
isInsolubleOccursCheck EqRel
eq_rel TcTyVar
tv1 PredType
rhs
         then Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkInsolubleCt CtEvidence
new_ev)
             -- If we have a ~ [a], it is not canonical, and in particular
             -- we don't want to rewrite existing inerts with it, otherwise
             -- we'd risk divergence in the constraint solver

         else Ct -> TcS (StopOrContinue Ct)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence -> Ct
mkIrredCt CtEvidence
new_ev) }
             -- A representational equality with an occurs-check problem isn't
             -- insoluble! For example:
             --   a ~R b a
             -- We might learn that b is the newtype Id.
             -- But, the occurs-check certainly prevents the equality from being
             -- canonical, and we might loop if we were to use it in rewriting.
  where
    role :: Role
role = EqRel -> Role
eqRelRole EqRel
eq_rel

    lhs :: PredType
lhs = TcTyVar -> PredType
mkTyVarTy TcTyVar
tv1

    rewrite_co1 :: TcCoercion
rewrite_co1  = Role -> PredType -> TcCoercion
mkTcReflCo Role
role PredType
lhs
    rewrite_co2 :: TcCoercion
rewrite_co2  = Role -> PredType -> TcCoercion
mkTcReflCo Role
role PredType
rhs

-- | Solve a reflexive equality constraint
canEqReflexive :: CtEvidence    -- ty ~ ty
               -> EqRel
               -> TcType        -- ty
               -> TcS (StopOrContinue Ct)   -- always Stop
canEqReflexive :: CtEvidence -> EqRel -> PredType -> TcS (StopOrContinue Ct)
canEqReflexive CtEvidence
ev EqRel
eq_rel PredType
ty
  = do { CtEvidence -> EvTerm -> TcS ()
setEvBindIfWanted CtEvidence
ev (TcCoercion -> EvTerm
evCoercion (TcCoercion -> EvTerm) -> TcCoercion -> EvTerm
forall a b. (a -> b) -> a -> b
$
                               Role -> PredType -> TcCoercion
mkTcReflCo (EqRel -> Role
eqRelRole EqRel
eq_rel) PredType
ty)
       ; CtEvidence -> String -> TcS (StopOrContinue Ct)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Solved by reflexivity" }

{-
Note [Canonical orientation for tyvar/tyvar equality constraints]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
When we have a ~ b where both 'a' and 'b' are TcTyVars, which way
round should be oriented in the CTyEqCan?  The rules, implemented by
canEqTyVarTyVar, are these

 * If either is a flatten-meta-variables, it goes on the left.

 * Put a meta-tyvar on the left if possible
       alpha[3] ~ r

 * If both are meta-tyvars, put the more touchable one (deepest level
   number) on the left, so there is the best chance of unifying it
        alpha[3] ~ beta[2]

 * If both are meta-tyvars and both at the same level, put a TyVarTv
   on the right if possible
        alpha[2] ~ beta[2](sig-tv)
   That way, when we unify alpha := beta, we don't lose the TyVarTv flag.

 * Put a meta-tv with a System Name on the left if possible so it
   gets eliminated (improves error messages)

 * If one is a flatten-skolem, put it on the left so that it is
   substituted out  Note [Eliminate flat-skols] in TcUinfy
        fsk ~ a

Note [Equalities with incompatible kinds]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
What do we do when we have an equality

  (tv :: k1) ~ (rhs :: k2)

where k1 and k2 differ? This Note explores this treacherous area.

We must proceed differently here depending on whether we have a Wanted
or a Given. Consider this:

 [W] w :: (alpha :: k) ~ (Int :: Type)

where k is a skolem. One possible way forward is this:

 [W] co :: k ~ Type
 [W] w :: (alpha :: k) ~ (Int |> sym co :: k)

The next step will be to unify

  alpha := Int |> sym co

Now, consider what error we'll report if we can't solve the "co"
wanted. Its CtOrigin is the w wanted... which now reads (after zonking)
Int ~ Int. The user thus sees that GHC can't solve Int ~ Int, which
is embarrassing. See #11198 for more tales of destruction.

The reason for this odd behavior is much the same as
Note [Wanteds do not rewrite Wanteds] in Constraint: note that the
new `co` is a Wanted.

The solution is then not to use `co` to "rewrite" -- that is, cast -- `w`, but
instead to keep `w` heterogeneous and irreducible. Given that we're not using
`co`, there is no reason to collect evidence for it, so `co` is born a
Derived, with a CtOrigin of KindEqOrigin. When the Derived is solved (by
unification), the original wanted (`w`) will get kicked out. We thus get

[D] _ :: k ~ Type
[W] w :: (alpha :: k) ~ (Int :: Type)

Note that the Wanted is unchanged and will be irreducible. This all happens
in canEqTyVarHetero.

Note that, if we had [G] co1 :: k ~ Type available, then we never get
to canEqTyVarHetero: canEqTyVar tries flattening the kinds first. If
we have [G] co1 :: k ~ Type, then flattening the kind of alpha would
rewrite k to Type, and we would end up in canEqTyVarHomo.

Successive canonicalizations of the same Wanted may produce
duplicate Deriveds. Similar duplications can happen with fundeps, and there
seems to be no easy way to avoid. I expect this case to be rare.

For Givens, this problem (the Wanteds-rewriting-Wanteds action of
a kind coercion) doesn't bite, so a heterogeneous Given gives
rise to a Given kind equality. No Deriveds here. We thus homogenise
the Given (see the "homo_co" in the Given case in canEqTyVarHetero) and
carry on with a homogeneous equality constraint.

Note [Type synonyms and canonicalization]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
We treat type synonym applications as xi types, that is, they do not
count as type function applications.  However, we do need to be a bit
careful with type synonyms: like type functions they may not be
generative or injective.  However, unlike type functions, they are
parametric, so there is no problem in expanding them whenever we see
them, since we do not need to know anything about their arguments in
order to expand them; this is what justifies not having to treat them
as specially as type function applications.  The thing that causes
some subtleties is that we prefer to leave type synonym applications
*unexpanded* whenever possible, in order to generate better error
messages.

If we encounter an equality constraint with type synonym applications
on both sides, or a type synonym application on one side and some sort
of type application on the other, we simply must expand out the type
synonyms in order to continue decomposing the equality constraint into
primitive equality constraints.  For example, suppose we have

  type F a = [Int]

and we encounter the equality

  F a ~ [b]

In order to continue we must expand F a into [Int], giving us the
equality

  [Int] ~ [b]

which we can then decompose into the more primitive equality
constraint

  Int ~ b.

However, if we encounter an equality constraint with a type synonym
application on one side and a variable on the other side, we should
NOT (necessarily) expand the type synonym, since for the purpose of
good error messages we want to leave type synonyms unexpanded as much
as possible.  Hence the ps_xi1, ps_xi2 argument passed to canEqTyVar.

-}

{-
************************************************************************
*                                                                      *
                  Evidence transformation
*                                                                      *
************************************************************************
-}

data StopOrContinue a
  = ContinueWith a    -- The constraint was not solved, although it may have
                      --   been rewritten

  | Stop CtEvidence   -- The (rewritten) constraint was solved
         SDoc         -- Tells how it was solved
                      -- Any new sub-goals have been put on the work list
  deriving (a -> StopOrContinue b -> StopOrContinue a
(a -> b) -> StopOrContinue a -> StopOrContinue b
(forall a b. (a -> b) -> StopOrContinue a -> StopOrContinue b)
-> (forall a b. a -> StopOrContinue b -> StopOrContinue a)
-> Functor StopOrContinue
forall a b. a -> StopOrContinue b -> StopOrContinue a
forall a b. (a -> b) -> StopOrContinue a -> StopOrContinue b
forall (f :: * -> *).
(forall a b. (a -> b) -> f a -> f b)
-> (forall a b. a -> f b -> f a) -> Functor f
<$ :: a -> StopOrContinue b -> StopOrContinue a
$c<$ :: forall a b. a -> StopOrContinue b -> StopOrContinue a
fmap :: (a -> b) -> StopOrContinue a -> StopOrContinue b
$cfmap :: forall a b. (a -> b) -> StopOrContinue a -> StopOrContinue b
Functor)

instance Outputable a => Outputable (StopOrContinue a) where
  ppr :: StopOrContinue a -> SDoc
ppr (Stop CtEvidence
ev SDoc
s)      = String -> SDoc
text String
"Stop" SDoc -> SDoc -> SDoc
<> SDoc -> SDoc
parens SDoc
s SDoc -> SDoc -> SDoc
<+> CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
ev
  ppr (ContinueWith a
w) = String -> SDoc
text String
"ContinueWith" SDoc -> SDoc -> SDoc
<+> a -> SDoc
forall a. Outputable a => a -> SDoc
ppr a
w

continueWith :: a -> TcS (StopOrContinue a)
continueWith :: a -> TcS (StopOrContinue a)
continueWith = StopOrContinue a -> TcS (StopOrContinue a)
forall (m :: * -> *) a. Monad m => a -> m a
return (StopOrContinue a -> TcS (StopOrContinue a))
-> (a -> StopOrContinue a) -> a -> TcS (StopOrContinue a)
forall b c a. (b -> c) -> (a -> b) -> a -> c
. a -> StopOrContinue a
forall a. a -> StopOrContinue a
ContinueWith

stopWith :: CtEvidence -> String -> TcS (StopOrContinue a)
stopWith :: CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
s = StopOrContinue a -> TcS (StopOrContinue a)
forall (m :: * -> *) a. Monad m => a -> m a
return (CtEvidence -> SDoc -> StopOrContinue a
forall a. CtEvidence -> SDoc -> StopOrContinue a
Stop CtEvidence
ev (String -> SDoc
text String
s))

andWhenContinue :: TcS (StopOrContinue a)
                -> (a -> TcS (StopOrContinue b))
                -> TcS (StopOrContinue b)
andWhenContinue :: TcS (StopOrContinue a)
-> (a -> TcS (StopOrContinue b)) -> TcS (StopOrContinue b)
andWhenContinue TcS (StopOrContinue a)
tcs1 a -> TcS (StopOrContinue b)
tcs2
  = do { StopOrContinue a
r <- TcS (StopOrContinue a)
tcs1
       ; case StopOrContinue a
r of
           Stop CtEvidence
ev SDoc
s       -> StopOrContinue b -> TcS (StopOrContinue b)
forall (m :: * -> *) a. Monad m => a -> m a
return (CtEvidence -> SDoc -> StopOrContinue b
forall a. CtEvidence -> SDoc -> StopOrContinue a
Stop CtEvidence
ev SDoc
s)
           ContinueWith a
ct -> a -> TcS (StopOrContinue b)
tcs2 a
ct }
infixr 0 `andWhenContinue`    -- allow chaining with ($)

rewriteEvidence :: CtEvidence   -- old evidence
                -> TcPredType   -- new predicate
                -> TcCoercion   -- Of type :: new predicate ~ <type of old evidence>
                -> TcS (StopOrContinue CtEvidence)
-- Returns Just new_ev iff either (i)  'co' is reflexivity
--                             or (ii) 'co' is not reflexivity, and 'new_pred' not cached
-- In either case, there is nothing new to do with new_ev
{-
     rewriteEvidence old_ev new_pred co
Main purpose: create new evidence for new_pred;
              unless new_pred is cached already
* Returns a new_ev : new_pred, with same wanted/given/derived flag as old_ev
* If old_ev was wanted, create a binding for old_ev, in terms of new_ev
* If old_ev was given, AND not cached, create a binding for new_ev, in terms of old_ev
* Returns Nothing if new_ev is already cached

        Old evidence    New predicate is               Return new evidence
        flavour                                        of same flavor
        -------------------------------------------------------------------
        Wanted          Already solved or in inert     Nothing
        or Derived      Not                            Just new_evidence

        Given           Already in inert               Nothing
                        Not                            Just new_evidence

Note [Rewriting with Refl]
~~~~~~~~~~~~~~~~~~~~~~~~~~
If the coercion is just reflexivity then you may re-use the same
variable.  But be careful!  Although the coercion is Refl, new_pred
may reflect the result of unification alpha := ty, so new_pred might
not _look_ the same as old_pred, and it's vital to proceed from now on
using new_pred.

qThe flattener preserves type synonyms, so they should appear in new_pred
as well as in old_pred; that is important for good error messages.
 -}


rewriteEvidence :: CtEvidence
-> PredType -> TcCoercion -> TcS (StopOrContinue CtEvidence)
rewriteEvidence old_ev :: CtEvidence
old_ev@(CtDerived {}) PredType
new_pred TcCoercion
_co
  = -- If derived, don't even look at the coercion.
    -- This is very important, DO NOT re-order the equations for
    -- rewriteEvidence to put the isTcReflCo test first!
    -- Why?  Because for *Derived* constraints, c, the coercion, which
    -- was produced by flattening, may contain suspended calls to
    -- (ctEvExpr c), which fails for Derived constraints.
    -- (Getting this wrong caused #7384.)
    CtEvidence -> TcS (StopOrContinue CtEvidence)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence
old_ev { ctev_pred :: PredType
ctev_pred = PredType
new_pred })

rewriteEvidence CtEvidence
old_ev PredType
new_pred TcCoercion
co
  | TcCoercion -> Bool
isTcReflCo TcCoercion
co -- See Note [Rewriting with Refl]
  = CtEvidence -> TcS (StopOrContinue CtEvidence)
forall a. a -> TcS (StopOrContinue a)
continueWith (CtEvidence
old_ev { ctev_pred :: PredType
ctev_pred = PredType
new_pred })

rewriteEvidence ev :: CtEvidence
ev@(CtGiven { ctev_evar :: CtEvidence -> TcTyVar
ctev_evar = TcTyVar
old_evar, ctev_loc :: CtEvidence -> CtLoc
ctev_loc = CtLoc
loc }) PredType
new_pred TcCoercion
co
  = do { CtEvidence
new_ev <- CtLoc -> (PredType, EvTerm) -> TcS CtEvidence
newGivenEvVar CtLoc
loc (PredType
new_pred, EvTerm
new_tm)
       ; CtEvidence -> TcS (StopOrContinue CtEvidence)
forall a. a -> TcS (StopOrContinue a)
continueWith CtEvidence
new_ev }
  where
    -- mkEvCast optimises ReflCo
    new_tm :: EvTerm
new_tm = EvExpr -> TcCoercion -> EvTerm
mkEvCast (TcTyVar -> EvExpr
evId TcTyVar
old_evar) (Role -> Role -> TcCoercion -> TcCoercion
tcDowngradeRole Role
Representational
                                                       (CtEvidence -> Role
ctEvRole CtEvidence
ev)
                                                       (TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
co))

rewriteEvidence ev :: CtEvidence
ev@(CtWanted { ctev_dest :: CtEvidence -> TcEvDest
ctev_dest = TcEvDest
dest
                             , ctev_nosh :: CtEvidence -> ShadowInfo
ctev_nosh = ShadowInfo
si
                             , ctev_loc :: CtEvidence -> CtLoc
ctev_loc = CtLoc
loc }) PredType
new_pred TcCoercion
co
  = do { MaybeNew
mb_new_ev <- ShadowInfo -> CtLoc -> PredType -> TcS MaybeNew
newWanted_SI ShadowInfo
si CtLoc
loc PredType
new_pred
               -- The "_SI" varant ensures that we make a new Wanted
               -- with the same shadow-info as the existing one
               -- with the same shadow-info as the existing one (#16735)
       ; MASSERT( tcCoercionRole co == ctEvRole ev )
       ; TcEvDest -> EvTerm -> TcS ()
setWantedEvTerm TcEvDest
dest
            (EvExpr -> TcCoercion -> EvTerm
mkEvCast (MaybeNew -> EvExpr
getEvExpr MaybeNew
mb_new_ev)
                      (Role -> Role -> TcCoercion -> TcCoercion
tcDowngradeRole Role
Representational (CtEvidence -> Role
ctEvRole CtEvidence
ev) TcCoercion
co))
       ; case MaybeNew
mb_new_ev of
            Fresh  CtEvidence
new_ev -> CtEvidence -> TcS (StopOrContinue CtEvidence)
forall a. a -> TcS (StopOrContinue a)
continueWith CtEvidence
new_ev
            Cached EvExpr
_      -> CtEvidence -> String -> TcS (StopOrContinue CtEvidence)
forall a. CtEvidence -> String -> TcS (StopOrContinue a)
stopWith CtEvidence
ev String
"Cached wanted" }


rewriteEqEvidence :: CtEvidence         -- Old evidence :: olhs ~ orhs (not swapped)
                                        --              or orhs ~ olhs (swapped)
                  -> SwapFlag
                  -> TcType -> TcType   -- New predicate  nlhs ~ nrhs
                                        -- Should be zonked, because we use tcTypeKind on nlhs/nrhs
                  -> TcCoercion         -- lhs_co, of type :: nlhs ~ olhs
                  -> TcCoercion         -- rhs_co, of type :: nrhs ~ orhs
                  -> TcS CtEvidence     -- Of type nlhs ~ nrhs
-- For (rewriteEqEvidence (Given g olhs orhs) False nlhs nrhs lhs_co rhs_co)
-- we generate
-- If not swapped
--      g1 : nlhs ~ nrhs = lhs_co ; g ; sym rhs_co
-- If 'swapped'
--      g1 : nlhs ~ nrhs = lhs_co ; Sym g ; sym rhs_co
--
-- For (Wanted w) we do the dual thing.
-- New  w1 : nlhs ~ nrhs
-- If not swapped
--      w : olhs ~ orhs = sym lhs_co ; w1 ; rhs_co
-- If swapped
--      w : orhs ~ olhs = sym rhs_co ; sym w1 ; lhs_co
--
-- It's all a form of rewwriteEvidence, specialised for equalities
rewriteEqEvidence :: CtEvidence
-> SwapFlag
-> PredType
-> PredType
-> TcCoercion
-> TcCoercion
-> TcS CtEvidence
rewriteEqEvidence CtEvidence
old_ev SwapFlag
swapped PredType
nlhs PredType
nrhs TcCoercion
lhs_co TcCoercion
rhs_co
  | CtDerived {} <- CtEvidence
old_ev  -- Don't force the evidence for a Derived
  = CtEvidence -> TcS CtEvidence
forall (m :: * -> *) a. Monad m => a -> m a
return (CtEvidence
old_ev { ctev_pred :: PredType
ctev_pred = PredType
new_pred })

  | SwapFlag
NotSwapped <- SwapFlag
swapped
  , TcCoercion -> Bool
isTcReflCo TcCoercion
lhs_co      -- See Note [Rewriting with Refl]
  , TcCoercion -> Bool
isTcReflCo TcCoercion
rhs_co
  = CtEvidence -> TcS CtEvidence
forall (m :: * -> *) a. Monad m => a -> m a
return (CtEvidence
old_ev { ctev_pred :: PredType
ctev_pred = PredType
new_pred })

  | CtGiven { ctev_evar :: CtEvidence -> TcTyVar
ctev_evar = TcTyVar
old_evar } <- CtEvidence
old_ev
  = do { let new_tm :: EvTerm
new_tm = TcCoercion -> EvTerm
evCoercion (TcCoercion
lhs_co
                                  TcCoercion -> TcCoercion -> TcCoercion
`mkTcTransCo` SwapFlag -> TcCoercion -> TcCoercion
maybeSym SwapFlag
swapped (TcTyVar -> TcCoercion
mkTcCoVarCo TcTyVar
old_evar)
                                  TcCoercion -> TcCoercion -> TcCoercion
`mkTcTransCo` TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
rhs_co)
       ; CtLoc -> (PredType, EvTerm) -> TcS CtEvidence
newGivenEvVar CtLoc
loc' (PredType
new_pred, EvTerm
new_tm) }

  | CtWanted { ctev_dest :: CtEvidence -> TcEvDest
ctev_dest = TcEvDest
dest, ctev_nosh :: CtEvidence -> ShadowInfo
ctev_nosh = ShadowInfo
si } <- CtEvidence
old_ev
  = do { (CtEvidence
new_ev, TcCoercion
hole_co) <- ShadowInfo
-> CtLoc
-> Role
-> PredType
-> PredType
-> TcS (CtEvidence, TcCoercion)
newWantedEq_SI ShadowInfo
si CtLoc
loc' (CtEvidence -> Role
ctEvRole CtEvidence
old_ev) PredType
nlhs PredType
nrhs
               -- The "_SI" varant ensures that we make a new Wanted
               -- with the same shadow-info as the existing one (#16735)
       ; let co :: TcCoercion
co = SwapFlag -> TcCoercion -> TcCoercion
maybeSym SwapFlag
swapped (TcCoercion -> TcCoercion) -> TcCoercion -> TcCoercion
forall a b. (a -> b) -> a -> b
$
                  TcCoercion -> TcCoercion
mkSymCo TcCoercion
lhs_co
                  TcCoercion -> TcCoercion -> TcCoercion
`mkTransCo` TcCoercion
hole_co
                  TcCoercion -> TcCoercion -> TcCoercion
`mkTransCo` TcCoercion
rhs_co
       ; TcEvDest -> TcCoercion -> TcS ()
setWantedEq TcEvDest
dest TcCoercion
co
       ; String -> SDoc -> TcS ()
traceTcS String
"rewriteEqEvidence" ([SDoc] -> SDoc
vcat [CtEvidence -> SDoc
forall a. Outputable a => a -> SDoc
ppr CtEvidence
old_ev, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
nlhs, PredType -> SDoc
forall a. Outputable a => a -> SDoc
ppr PredType
nrhs, TcCoercion -> SDoc
forall a. Outputable a => a -> SDoc
ppr TcCoercion
co])
       ; CtEvidence -> TcS CtEvidence
forall (m :: * -> *) a. Monad m => a -> m a
return CtEvidence
new_ev }

  | Bool
otherwise
  = String -> TcS CtEvidence
forall a. String -> a
panic String
"rewriteEvidence"
  where
    new_pred :: PredType
new_pred = CtEvidence -> PredType -> PredType -> PredType
mkTcEqPredLikeEv CtEvidence
old_ev PredType
nlhs PredType
nrhs

      -- equality is like a type class. Bumping the depth is necessary because
      -- of recursive newtypes, where "reducing" a newtype can actually make
      -- it bigger. See Note [Newtypes can blow the stack].
    loc :: CtLoc
loc      = CtEvidence -> CtLoc
ctEvLoc CtEvidence
old_ev
    loc' :: CtLoc
loc'     = CtLoc -> CtLoc
bumpCtLocDepth CtLoc
loc

{- Note [unifyWanted and unifyDerived]
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
When decomposing equalities we often create new wanted constraints for
(s ~ t).  But what if s=t?  Then it'd be faster to return Refl right away.
Similar remarks apply for Derived.

Rather than making an equality test (which traverses the structure of the
type, perhaps fruitlessly), unifyWanted traverses the common structure, and
bales out when it finds a difference by creating a new Wanted constraint.
But where it succeeds in finding common structure, it just builds a coercion
to reflect it.
-}

unifyWanted :: CtLoc -> Role
            -> TcType -> TcType -> TcS Coercion
-- Return coercion witnessing the equality of the two types,
-- emitting new work equalities where necessary to achieve that
-- Very good short-cut when the two types are equal, or nearly so
-- See Note [unifyWanted and unifyDerived]
-- The returned coercion's role matches the input parameter
unifyWanted :: CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
loc Role
Phantom PredType
ty1 PredType
ty2
  = do { TcCoercion
kind_co <- CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
loc Role
Nominal (HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind PredType
ty1) (HasDebugCallStack => PredType -> PredType
PredType -> PredType
tcTypeKind PredType
ty2)
       ; TcCoercion -> TcS TcCoercion
forall (m :: * -> *) a. Monad m => a -> m a
return (TcCoercion -> PredType -> PredType -> TcCoercion
mkPhantomCo TcCoercion
kind_co PredType
ty1 PredType
ty2) }

unifyWanted CtLoc
loc Role
role PredType
orig_ty1 PredType
orig_ty2
  = PredType -> PredType -> TcS TcCoercion
go PredType
orig_ty1 PredType
orig_ty2
  where
    go :: PredType -> PredType -> TcS TcCoercion
go PredType
ty1 PredType
ty2 | Just PredType
ty1' <- PredType -> Maybe PredType
tcView PredType
ty1 = PredType -> PredType -> TcS TcCoercion
go PredType
ty1' PredType
ty2
    go PredType
ty1 PredType
ty2 | Just PredType
ty2' <- PredType -> Maybe PredType
tcView PredType
ty2 = PredType -> PredType -> TcS TcCoercion
go PredType
ty1 PredType
ty2'

    go (FunTy AnonArgFlag
_ PredType
s1 PredType
t1) (FunTy AnonArgFlag
_ PredType
s2 PredType
t2)
      = do { TcCoercion
co_s <- CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
loc Role
role PredType
s1 PredType
s2
           ; TcCoercion
co_t <- CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
loc Role
role PredType
t1 PredType
t2
           ; TcCoercion -> TcS TcCoercion
forall (m :: * -> *) a. Monad m => a -> m a
return (Role -> TcCoercion -> TcCoercion -> TcCoercion
mkFunCo Role
role TcCoercion
co_s TcCoercion
co_t) }
    go (TyConApp TyCon
tc1 [PredType]
tys1) (TyConApp TyCon
tc2 [PredType]
tys2)
      | TyCon
tc1 TyCon -> TyCon -> Bool
forall a. Eq a => a -> a -> Bool
== TyCon
tc2, [PredType]
tys1 [PredType] -> [PredType] -> Bool
forall a b. [a] -> [b] -> Bool
`equalLength` [PredType]
tys2
      , TyCon -> Role -> Bool
isInjectiveTyCon TyCon
tc1 Role
role -- don't look under newtypes at Rep equality
      = do { [TcCoercion]
cos <- (Role -> PredType -> PredType -> TcS TcCoercion)
-> [Role] -> [PredType] -> [PredType] -> TcS [TcCoercion]
forall (m :: * -> *) a b c d.
Monad m =>
(a -> b -> c -> m d) -> [a] -> [b] -> [c] -> m [d]
zipWith3M (CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
unifyWanted CtLoc
loc)
                              (Role -> TyCon -> [Role]
tyConRolesX Role
role TyCon
tc1) [PredType]
tys1 [PredType]
tys2
           ; TcCoercion -> TcS TcCoercion
forall (m :: * -> *) a. Monad m => a -> m a
return (HasDebugCallStack => Role -> TyCon -> [TcCoercion] -> TcCoercion
Role -> TyCon -> [TcCoercion] -> TcCoercion
mkTyConAppCo Role
role TyCon
tc1 [TcCoercion]
cos) }

    go ty1 :: PredType
ty1@(TyVarTy TcTyVar
tv) PredType
ty2
      = do { Maybe PredType
mb_ty <- TcTyVar -> TcS (Maybe PredType)
isFilledMetaTyVar_maybe TcTyVar
tv
           ; case Maybe PredType
mb_ty of
                Just PredType
ty1' -> PredType -> PredType -> TcS TcCoercion
go PredType
ty1' PredType
ty2
                Maybe PredType
Nothing   -> PredType -> PredType -> TcS TcCoercion
bale_out PredType
ty1 PredType
ty2}
    go PredType
ty1 ty2 :: PredType
ty2@(TyVarTy TcTyVar
tv)
      = do { Maybe PredType
mb_ty <- TcTyVar -> TcS (Maybe PredType)
isFilledMetaTyVar_maybe TcTyVar
tv
           ; case Maybe PredType
mb_ty of
                Just PredType
ty2' -> PredType -> PredType -> TcS TcCoercion
go PredType
ty1 PredType
ty2'
                Maybe PredType
Nothing   -> PredType -> PredType -> TcS TcCoercion
bale_out PredType
ty1 PredType
ty2 }

    go ty1 :: PredType
ty1@(CoercionTy {}) (CoercionTy {})
      = TcCoercion -> TcS TcCoercion
forall (m :: * -> *) a. Monad m => a -> m a
return (Role -> PredType -> TcCoercion
mkReflCo Role
role PredType
ty1) -- we just don't care about coercions!

    go PredType
ty1 PredType
ty2 = PredType -> PredType -> TcS TcCoercion
bale_out PredType
ty1 PredType
ty2

    bale_out :: PredType -> PredType -> TcS TcCoercion
bale_out PredType
ty1 PredType
ty2
       | PredType
ty1 HasDebugCallStack => PredType -> PredType -> Bool
PredType -> PredType -> Bool
`tcEqType` PredType
ty2 = TcCoercion -> TcS TcCoercion
forall (m :: * -> *) a. Monad m => a -> m a
return (Role -> PredType -> TcCoercion
mkTcReflCo Role
role PredType
ty1)
        -- Check for equality; e.g. a ~ a, or (m a) ~ (m a)
       | Bool
otherwise = CtLoc -> Role -> PredType -> PredType -> TcS TcCoercion
emitNewWantedEq CtLoc
loc Role
role PredType
orig_ty1 PredType
orig_ty2

unifyDeriveds :: CtLoc -> [Role] -> [TcType] -> [TcType] -> TcS ()
-- See Note [unifyWanted and unifyDerived]
unifyDeriveds :: CtLoc -> [Role] -> [PredType] -> [PredType] -> TcS ()
unifyDeriveds CtLoc
loc [Role]
roles [PredType]
tys1 [PredType]
tys2 = (Role -> PredType -> PredType -> TcS ())
-> [Role] -> [PredType] -> [PredType] -> TcS ()
forall (m :: * -> *) a b c d.
Monad m =>
(a -> b -> c -> m d) -> [a] -> [b] -> [c] -> m ()
zipWith3M_ (CtLoc -> Role -> PredType -> PredType -> TcS ()
unify_derived CtLoc
loc) [Role]
roles [PredType]
tys1 [PredType]
tys2

unifyDerived :: CtLoc -> Role -> Pair TcType -> TcS ()
-- See Note [unifyWanted and unifyDerived]
unifyDerived :: CtLoc -> Role -> Pair PredType -> TcS ()
unifyDerived CtLoc
loc Role
role (Pair PredType
ty1 PredType
ty2) = CtLoc -> Role -> PredType -> PredType -> TcS ()
unify_derived CtLoc
loc Role
role PredType
ty1 PredType
ty2

unify_derived :: CtLoc -> Role -> TcType -> TcType -> TcS ()
-- Create new Derived and put it in the work list
-- Should do nothing if the two types are equal
-- See Note [unifyWanted and unifyDerived]
unify_derived :: CtLoc -> Role -> PredType -> PredType -> TcS ()
unify_derived CtLoc
_   Role
Phantom PredType
_        PredType
_        = () -> TcS ()
forall (m :: * -> *) a. Monad m => a -> m a
return ()
unify_derived CtLoc
loc Role
role    PredType
orig_ty1 PredType
orig_ty2
  = PredType -> PredType -> TcS ()
go PredType
orig_ty1 PredType
orig_ty2
  where
    go :: PredType -> PredType -> TcS ()
go PredType
ty1 PredType
ty2 | Just PredType
ty1' <- PredType -> Maybe PredType
tcView PredType
ty1 = PredType -> PredType -> TcS ()
go PredType
ty1' PredType
ty2
    go PredType
ty1 PredType
ty2 | Just PredType
ty2' <- PredType -> Maybe PredType
tcView PredType
ty2 = PredType -> PredType -> TcS ()
go PredType
ty1 PredType
ty2'

    go (FunTy AnonArgFlag
_ PredType
s1 PredType
t1) (FunTy AnonArgFlag
_ PredType
s2 PredType
t2)
      = do { CtLoc -> Role -> PredType -> PredType -> TcS ()
unify_derived CtLoc
loc Role
role PredType
s1 PredType
s2
           ; CtLoc -> Role -> PredType -> PredType -> TcS ()
unify_derived CtLoc
loc Role
role PredType
t1 PredType
t2 }
    go (TyConApp TyCon
tc1 [PredType]
tys1) (TyConApp TyCon
tc2 [PredType]
tys2)
      | TyCon
tc1 TyCon -> TyCon -> Bool
forall a. Eq a => a -> a -> Bool
== TyCon
tc2, [PredType]
tys1 [PredType] -> [PredType] -> Bool
forall a b. [a] -> [b] -> Bool
`equalLength` [PredType]
tys2
      , TyCon -> Role -> Bool
isInjectiveTyCon TyCon
tc1 Role
role
      = CtLoc -> [Role] -> [PredType] -> [PredType] -> TcS ()
unifyDeriveds CtLoc
loc (Role -> TyCon -> [Role]
tyConRolesX Role
role TyCon
tc1) [PredType]
tys1 [PredType]
tys2
    go ty1 :: PredType
ty1@(TyVarTy TcTyVar
tv) PredType
ty2
      = do { Maybe PredType
mb_ty <- TcTyVar -> TcS (Maybe PredType)
isFilledMetaTyVar_maybe TcTyVar
tv
           ; case Maybe PredType
mb_ty of
                Just PredType
ty1' -> PredType -> PredType -> TcS ()
go PredType
ty1' PredType
ty2
                Maybe PredType
Nothing   -> PredType -> PredType -> TcS ()
bale_out PredType
ty1 PredType
ty2 }
    go PredType
ty1 ty2 :: PredType
ty2@(TyVarTy TcTyVar
tv)
      = do { Maybe PredType
mb_ty <- TcTyVar -> TcS (Maybe PredType)
isFilledMetaTyVar_maybe TcTyVar
tv
           ; case Maybe PredType
mb_ty of
                Just PredType
ty2' -> PredType -> PredType -> TcS ()
go PredType
ty1 PredType
ty2'
                Maybe PredType
Nothing   -> PredType -> PredType -> TcS ()
bale_out PredType
ty1 PredType
ty2 }
    go PredType
ty1 PredType
ty2 = PredType -> PredType -> TcS ()
bale_out PredType
ty1 PredType
ty2

    bale_out :: PredType -> PredType -> TcS ()
bale_out PredType
ty1 PredType
ty2
       | PredType
ty1 HasDebugCallStack => PredType -> PredType -> Bool
PredType -> PredType -> Bool
`tcEqType` PredType
ty2 = () -> TcS ()
forall (m :: * -> *) a. Monad m => a -> m a
return ()
        -- Check for equality; e.g. a ~ a, or (m a) ~ (m a)
       | Bool
otherwise = CtLoc -> Role -> PredType -> PredType -> TcS ()
emitNewDerivedEq CtLoc
loc Role
role PredType
orig_ty1 PredType
orig_ty2

maybeSym :: SwapFlag -> TcCoercion -> TcCoercion
maybeSym :: SwapFlag -> TcCoercion -> TcCoercion
maybeSym SwapFlag
IsSwapped  TcCoercion
co = TcCoercion -> TcCoercion
mkTcSymCo TcCoercion
co
maybeSym SwapFlag
NotSwapped TcCoercion
co = TcCoercion
co