def
Lean.Meta.Grind.Arith.Linear.DiseqCnstr.applyEq?
(a : Int)
(x : Var)
(c₁ : EqCnstr)
(b : Int)
(c₂ : DiseqCnstr)
:
Given an equation c₁
containing the monomial a*x
, and a disequality constraint c₂
containing the monomial b*x
, eliminate x
by applying substitution.
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
Lean.Meta.Grind.Arith.Linear.IneqCnstr.applyEq
(a : Nat)
(x : Var)
(c₁ : EqCnstr)
(b : Int)
(c₂ : IneqCnstr)
:
Given an equation c₁
containing the monomial a*x
, and an inequality constraint c₂
containing the monomial b*x
, eliminate x
by applying substitution.
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
@[export lean_process_linarith_eq]
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[export lean_process_linarith_diseq]
Equations
- One or more equations did not get rendered due to their size.