@[reducible, inline]
Equations
Instances For
@[reducible, inline]
abbrev
Lean.Meta.Grind.Arith.CommRing.SemiringM.run
{α : Type}
(semiringId : Nat)
(x : SemiringM α)
:
GoalM α
Equations
- Lean.Meta.Grind.Arith.CommRing.SemiringM.run semiringId x = x { semiringId := semiringId }
Instances For
@[reducible, inline]
Equations
- Lean.Meta.Grind.Arith.CommRing.getSemiringId = do let __do_lift ← read pure __do_lift.semiringId
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.Grind.Arith.CommRing.getTermSemiringId? e = do let __do_lift ← Lean.Meta.Grind.Arith.CommRing.get' pure (Lean.PersistentHashMap.find? __do_lift.exprToSemiringId { expr := e })
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Similar to mkVar
but for Semiring
s
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Grind.Ring.OfSemiring.Expr.denoteAsRingExpr e = do let __do_lift ← Lean.Grind.Ring.OfSemiring.Expr.denoteAsRingExpr.go✝ e liftM (Lean.Meta.Grind.shareCommon __do_lift)