@[inline]
Equations
Instances For
@[always_inline]
instance
Lean.Meta.Grind.Arith.Linear.instMonadGetStructOfMonadLift
(m n : Type → Type)
[MonadLift m n]
[MonadGetStruct m]
:
Equations
@[reducible, inline]
We don't want to keep carrying the StructId
around.
Equations
Instances For
@[reducible, inline]
abbrev
Lean.Meta.Grind.Arith.Linear.LinearM.run
{α : Type}
(structId : Nat)
(x : LinearM α)
:
GoalM α
Equations
- Lean.Meta.Grind.Arith.Linear.LinearM.run structId x = x { structId := structId }
Instances For
@[reducible, inline]
Equations
- Lean.Meta.Grind.Arith.Linear.getStructId = do let __do_lift ← read pure __do_lift.structId
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.getRingCore? (some ringId) = Lean.Meta.Grind.Arith.CommRing.RingM.run ringId do let __do_lift ← Lean.Meta.Grind.Arith.CommRing.getRing pure (some __do_lift)
- Lean.Meta.Grind.Arith.Linear.getRingCore? ringId? = pure none
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.throwNotRing = Lean.throwError (Lean.toMessageData "`grind linarith` internal error, structure is not a ring")
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.throwNotCommRing = Lean.throwError (Lean.toMessageData "`grind linarith` internal error, structure is not a commutative ring")
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.getRing? = do let __do_lift ← Lean.Meta.Grind.Arith.Linear.getStruct liftM (Lean.Meta.Grind.Arith.Linear.getRingCore? __do_lift.ringId?)
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.