Helper function for removing dependency on
GoalM
. InRingM
andSemiringM
, this is justsharedCommon (← canon e)
When printing counterexamples, we are atMetaM
, and this is just the identity function.Helper function for removing dependency on
GoalM
. During search we want to track the instances synthesized bygrind
, and this isGrind.synthInstance
.
Instances
@[always_inline]
instance
Lean.Meta.Grind.Arith.CommRing.instMonadCanonOfMonadLift
(m n : Type → Type)
[MonadLift m n]
[MonadCanon m]
:
Equations
- One or more equations did not get rendered due to their size.
def
Lean.Meta.Grind.Arith.CommRing.MonadCanon.synthInstance
{m : Type → Type}
[Monad m]
[MonadError m]
[MonadCanon m]
(type : Expr)
:
m Expr
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[always_inline]
instance
Lean.Meta.Grind.Arith.CommRing.instMonadCommRingOfMonadLift
(m n : Type → Type)
[MonadLift m n]
[MonadCommRing m]
:
Equations
- One or more equations did not get rendered due to their size.
@[always_inline]
instance
Lean.Meta.Grind.Arith.CommRing.instMonadRingOfMonadOfMonadCommRing
(m : Type → Type)
[Monad m]
[MonadCommRing m]
:
Equations
- One or more equations did not get rendered due to their size.