Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Auxiliary inductive type for representing constraints and equalities
that should be propagated to core.
Recall that we cannot compute proofs until the short-distance
data-structures have been fully updated when a new edge is inserted.
Thus, we store the information to be propagated into a list.
See field propagate
in State
.
- eqTrue (e : Expr) (u v : NodeId) (k k' : Int) : ToPropagate
- eqFalse (e : Expr) (u v : NodeId) (k k' : Int) : ToPropagate
- eq (u v : NodeId) : ToPropagate
Instances For
State of the constraint offset procedure.
Mapping from
NodeId
to theExpr
represented by the node.Mapping from
Expr
to a node representing it.Mapping from
Expr
representing inequalites to constraints.Mapping from pairs
(u, v)
to a list of offset constraints onu
andv
. We use this mapping to implement exhaustive constraint propagation.For each node with id
u
,sources[u]
contains pairs(v, k)
s.t. there is a path fromv
tou
with weightk
.For each node with id
u
,targets[u]
contains pairs(v, k)
s.t. there is a path fromu
tov
with weightk
.- propagate : List ToPropagate
Truth values and equalities to propagate to core.
Instances For
Equations
- One or more equations did not get rendered due to their size.