Equations
- Lean.Meta.Grind.Arith.Linear.isAddInst struct inst = Lean.Meta.Grind.isSameExpr struct.addFn.appArg! inst
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isZeroInst struct inst = Lean.Meta.Grind.isSameExpr struct.zero.appArg! inst
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isHMulInst struct inst = Lean.Meta.Grind.isSameExpr struct.hmulFn.appArg! inst
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isHMulNatInst struct inst = Lean.Meta.Grind.isSameExpr struct.hmulNatFn.appArg! inst
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isHSMulInst struct inst = match struct.hsmulFn? with | some smulFn => Lean.Meta.Grind.isSameExpr smulFn.appArg! inst | x => false
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isHSMulNatInst struct inst = match struct.hsmulNatFn? with | some smulFn => Lean.Meta.Grind.isSameExpr smulFn.appArg! inst | x => false
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isSubInst struct inst = Lean.Meta.Grind.isSameExpr struct.subFn.appArg! inst
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.isNegInst struct inst = Lean.Meta.Grind.isSameExpr struct.negFn.appArg! inst
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Converts a Lean IntModule
expression e
into a LinExpr
If skipVar
is true
, then the result is none
if e
is not an interpreted IntModule
term.
We use skipVar := false
when processing inequalities, and skipVar := true
for equalities and disequalities
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.reify?.toVar e = do let __do_lift ← Lean.Meta.Grind.Arith.Linear.mkVar e pure (Lean.Grind.Linarith.Expr.var __do_lift)
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Lean.Meta.Grind.Arith.Linear.reify?.isOfNatZero e = do let __do_lift ← Lean.Meta.Grind.Arith.Linear.getStruct Lean.Meta.withDefault (liftM (Lean.Meta.isDefEq e __do_lift.ofNatZero))