Documentation
Lean
.
Meta
.
Tactic
.
Grind
.
Order
.
Assert
Search
return to top
source
Imports
Init.Grind.Order
Init.Grind.Propagator
Lean.Meta.Tactic.Grind.PropagatorAttr
Lean.Meta.Tactic.Grind.Order.OrderM
Lean.Meta.Tactic.Grind.Order.Proof
Lean.Meta.Tactic.Grind.Order.Util
Imported by
Lean
.
Meta
.
Grind
.
Order
.
propagateEqTrue
Lean
.
Meta
.
Grind
.
Order
.
propagateEqFalse
Lean
.
Meta
.
Grind
.
Order
.
processNewEq
source
def
Lean
.
Meta
.
Grind
.
Order
.
propagateEqTrue
(
c
:
Cnstr
NodeId
)
(
e
:
Expr
)
(
u
v
:
NodeId
)
(
k
k'
:
Weight
)
:
OrderM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
Grind
.
Order
.
propagateEqFalse
(
c
:
Cnstr
NodeId
)
(
e
:
Expr
)
(
u
v
:
NodeId
)
(
k
k'
:
Weight
)
:
OrderM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For
source
def
Lean
.
Meta
.
Grind
.
Order
.
processNewEq
(
a
b
:
Expr
)
:
GoalM
Unit
Equations
One or more equations did not get rendered due to their size.
Instances For