- natStructId : Nat
Instances For
@[reducible, inline]
Equations
Instances For
@[reducible, inline]
abbrev
Lean.Meta.Grind.Arith.Linear.OfNatModuleM.run
{α : Type}
(natStructId : Nat)
(x : OfNatModuleM α)
:
GoalM α
Equations
- Lean.Meta.Grind.Arith.Linear.OfNatModuleM.run natStructId x = x { natStructId := natStructId }
Instances For
@[reducible, inline]
Equations
- Lean.Meta.Grind.Arith.Linear.getNatStructId = do let __do_lift ← read pure __do_lift.natStructId
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
@[inline]
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.getTermNatStructId? e = do let __do_lift ← Lean.Meta.Grind.Arith.Linear.get' pure (Lean.PersistentHashMap.find? __do_lift.exprToNatStructId { expr := e })
Instances For
Returns some natStructId
if a
and b
are elements of the same NatModule
structure.
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.