3
0
Fork 0
mirror of https://github.com/Z3Prover/z3 synced 2025-04-23 17:15:31 +00:00
Signed-off-by: Nikolaj Bjorner <nbjorner@microsoft.com>
This commit is contained in:
Nikolaj Bjorner 2019-12-17 16:59:33 -08:00
parent f090abce9f
commit 9e4a7ae4b8
6 changed files with 939 additions and 0 deletions

View file

@ -1,6 +1,7 @@
z3_add_component(dd
SOURCES
dd_bdd.cpp
dd_pdd.cpp
COMPONENT_DEPENDENCIES
util
)

642
src/math/dd/dd_pdd.cpp Normal file
View file

@ -0,0 +1,642 @@
/*++
Copyright (c) 2019 Microsoft Corporation
Module Name:
dd_pdd.cpp
Abstract:
Poly DD package
Author:
Nikolaj Bjorner (nbjorner) 2019-12-17
Revision History:
--*/
#include "util/trace.h"
#include "util/stopwatch.h"
#include "math/dd/dd_pdd.h"
namespace dd {
pdd_manager::pdd_manager(unsigned num_vars) {
m_spare_entry = nullptr;
m_max_num_pdd_nodes = 1 << 24; // up to 16M nodes
m_mark_level = 0;
alloc_free_nodes(1024 + num_vars);
m_disable_gc = false;
m_is_new_node = false;
// add dummy nodes for operations, and 0, 1 pdds.
imk_val(rational::zero()); // becomes pdd_zero
imk_val(rational::one()); // becomes pdd_one
for (unsigned i = 2; i <= pdd_no_op + 2; ++i) {
m_nodes.push_back(pdd_node(0,0,0));
m_nodes.back().m_refcount = max_rc;
m_nodes.back().m_index = m_nodes.size()-1;
}
// add variables
for (unsigned i = 0; i < num_vars; ++i) {
reserve_var(i);
}
}
pdd_manager::~pdd_manager() {
if (m_spare_entry) {
m_alloc.deallocate(sizeof(*m_spare_entry), m_spare_entry);
}
for (auto* e : m_op_cache) {
SASSERT(e != m_spare_entry);
m_alloc.deallocate(sizeof(*e), e);
}
}
pdd pdd_manager::add(pdd const& a, pdd const& b) { return pdd(apply(a.root, b.root, pdd_add_op), this); }
pdd pdd_manager::sub(pdd const& a, pdd const& b) { return pdd(apply(a.root, b.root, pdd_sub_op), this); }
pdd pdd_manager::mul(pdd const& a, pdd const& b) { return pdd(apply(a.root, b.root, pdd_mul_op), this); }
pdd pdd_manager::reduce(pdd const& a, pdd const& b) { return pdd(apply(a.root, b.root, pdd_reduce_op), this); }
pdd pdd_manager::mk_val(rational const& r) { return pdd(imk_val(r), this); }
pdd pdd_manager::mul(rational const& r, pdd const& b) { pdd c(mk_val(r)); return pdd(apply(c.root, b.root, pdd_mul_op), this); }
pdd pdd_manager::add(rational const& r, pdd const& b) { pdd c(mk_val(r)); return pdd(apply(c.root, b.root, pdd_add_op), this); }
pdd_manager::PDD pdd_manager::apply(PDD arg1, PDD arg2, pdd_op op) {
bool first = true;
SASSERT(well_formed());
scoped_push _sp(*this);
while (true) {
try {
return apply_rec(arg1, arg2, op);
}
catch (const mem_out &) {
try_gc();
if (!first) throw;
first = false;
}
}
SASSERT(well_formed());
}
bool pdd_manager::check_result(op_entry*& e1, op_entry const* e2, PDD a, PDD b, PDD c) {
if (e1 != e2) {
SASSERT(e2->m_result != null_pdd);
push_entry(e1);
e1 = nullptr;
return true;
}
else {
e1->m_pdd1 = a;
e1->m_pdd2 = b;
e1->m_op = c;
SASSERT(e1->m_result == null_pdd);
return false;
}
}
pdd_manager::PDD pdd_manager::apply_rec(PDD a, PDD b, pdd_op op) {
switch (op) {
case pdd_add_op:
if (is_zero(a)) return b;
if (is_zero(b)) return a;
if (is_val(a) && is_val(b)) return imk_val(val(a) + val(b));
if (level(a) < level(b)) std::swap(a, b);
break;
case pdd_sub_op:
if (a == b) return zero_pdd;
if (is_zero(b)) return a;
if (is_val(a) && is_val(b)) return imk_val(val(a) - val(b));
break;
case pdd_mul_op:
if (is_zero(a) || is_zero(b)) return zero_pdd;
if (is_one(a)) return b;
if (is_one(b)) return a;
if (is_val(a) && is_val(b)) return imk_val(val(a) * val(b));
if (level(a) < level(b)) std::swap(a, b);
break;
case pdd_reduce_op:
if (is_zero(b)) return a;
if (is_val(a)) return a;
if (level(a) < level(b)) return a;
break;
default:
UNREACHABLE();
break;
}
op_entry * e1 = pop_entry(a, b, op);
op_entry const* e2 = m_op_cache.insert_if_not_there(e1);
if (check_result(e1, e2, a, b, op)) {
SASSERT(!m_free_nodes.contains(e2->m_result));
return e2->m_result;
}
PDD r;
unsigned level_a = level(a), level_b = level(b);
unsigned npop = 2;
switch (op) {
case pdd_add_op:
case pdd_sub_op:
if (is_val(a)) {
SASSERT(!is_val(b));
push(apply_rec(a, lo(b), op));
r = make_node(level_b, read(1), hi(b));
npop = 1;
}
else if (is_val(b)) {
SASSERT(!is_val(a));
push(apply_rec(b, lo(a), op));
r = make_node(level_a, read(1), hi(a));
npop = 1;
}
else if (level_a == level_b) {
push(apply_rec(lo(a), lo(b), op));
push(apply_rec(hi(a), hi(b), op));
r = make_node(level_a, read(2), read(1));
}
else if (level_a > level_b) {
push(apply_rec(lo(a), b, op));
r = make_node(level_a, read(1), hi(a));
npop = 1;
}
else {
push(apply_rec(lo(b), a, op));
r = make_node(level_b, read(1), hi(b));
npop = 1;
}
break;
case pdd_mul_op:
if (is_val(a)) {
push(apply_rec(a, lo(b), op));
push(apply_rec(a, hi(b), op));
r = make_node(level_b, read(2), read(1));
}
else if (is_val(b)) {
push(apply_rec(b, lo(a), op));
push(apply_rec(b, hi(a), op));
r = make_node(level_a, read(2), read(1));
}
else if (level_a == level_b) {
// (xa+b)*(xc+d) = x(x*ac + (ad+bc)) + bd
push(apply_rec(hi(a), hi(b), op));
push(apply_rec(hi(a), lo(b), op));
push(apply_rec(lo(a), hi(b), op));
push(apply_rec(lo(a), lo(b), op));
unsigned ac = read(4), ad = read(3), bc = read(2), bd = read(1);
push(apply_rec(ad, bc, pdd_add_op));
r = make_node(level_a, read(1), ac);
r = make_node(level_a, bd, r);
npop = 5;
}
else {
// (xa+b)*c = x(ac) + bc
SASSERT(level_a > level_b);
push(apply_rec(lo(a), b, op));
push(apply_rec(hi(a), b, op));
r = make_node(level_a, read(2), read(1));
}
break;
case pdd_reduce_op:
if (level_a > level_b) {
push(apply_rec(lo(a), b, op));
push(apply_rec(hi(a), b, op));
r = make_node(level_a, read(2), read(1));
}
else {
SASSERT(level_a == level_b);
r = reduce_on_match(a, b);
npop = 0;
}
break;
default:
UNREACHABLE();
}
pop(npop);
e1->m_result = r;
// SASSERT(well_formed());
SASSERT(!m_free_nodes.contains(r));
return r;
}
// q = lt(a)/lt(b), return a - b*q
pdd_manager::PDD pdd_manager::reduce_on_match(PDD a, PDD b) {
SASSERT(level(a) == level(b) && !is_val(a) && !is_val(b));
if (lm_divides(b, a)) {
PDD q = lt_quotient(b, a);
PDD r = apply(q, b, pdd_mul_op);
return apply(a, r, pdd_sub_op);
}
else {
return a;
}
}
// true if leading monomial of p divides leading monomial of q
bool pdd_manager::lm_divides(PDD p, PDD q) const {
while (true) {
if (is_val(p)) return true;
if (is_val(q)) return false;
if (level(p) > level(q)) return false;
if (level(p) == level(q)) {
p = hi(p); q = hi(q);
}
else {
q = hi(q);
}
}
}
// return quotient r, such that lt(q) = lt(p)*r
// assume lm_divides(p, q)
pdd_manager::PDD pdd_manager::lt_quotient(PDD p, PDD q) {
SASSERT(lm_divides(p, q));
if (is_val(p)) {
if (is_val(q)) {
return imk_val(val(q)/val(p));
}
}
else if (level(p) == level(q)) {
p = hi(p);
}
SASSERT(!is_val(q));
return lt_quotient(p, hi(q));
}
//
// p = lcm(lm(a),lm(b))/lm(a), q = lcm(lm(a),lm(b))/lm(b)
// pc = coeff(lt(a)) qc = coeff(lt(b))
// compute a*q*qc - b*p*pc
//
bool pdd_manager::try_spoly(pdd const& a, pdd const& b, pdd& r) {
if (!common_factors(a, b, m_p, m_q, m_pc, m_qc)) return false;
r = spoly(a, b, m_p, m_q, m_pc, m_qc);
return true;
}
pdd pdd_manager::spoly(pdd const& a, pdd const& b, unsigned_vector const& p, unsigned_vector const& q, rational const& pc, rational const& qc) {
pdd r1 = mul(qc, a);
for (unsigned i = p.size(); i-- > 0; ) r1 = mul(mk_var(p[i]), r1);
pdd r2 = mul(qc, b);
for (unsigned i = q.size(); i-- > 0; ) r2 = mul(mk_var(q[i]), r2);
return sub(r1, r2);
}
bool pdd_manager::common_factors(pdd const& a, pdd const& b, unsigned_vector& p, unsigned_vector& q, rational& pc, rational& qc) {
p.reset(); q.reset();
PDD x = a.root, y = b.root;
bool has_common = false;
while (true) {
if (is_val(x) || is_val(y)) {
if (!has_common) return false;
while (!is_val(y)) y = hi(y);
while (!is_val(x)) x = hi(x);
pc = val(x);
qc = val(y);
return true;
}
if (level(x) == level(y)) {
has_common = true;
x = hi(x);
y = hi(y);
}
else if (level(x) > level(y)) {
p.push_back(var(x));
x = hi(x);
}
else {
q.push_back(var(y));
y = hi(y);
}
}
}
void pdd_manager::push(PDD b) {
m_pdd_stack.push_back(b);
}
void pdd_manager::pop(unsigned num_scopes) {
m_pdd_stack.shrink(m_pdd_stack.size() - num_scopes);
}
pdd_manager::PDD pdd_manager::read(unsigned index) {
return m_pdd_stack[m_pdd_stack.size() - index];
}
pdd_manager::op_entry* pdd_manager::pop_entry(PDD l, PDD r, PDD op) {
op_entry* result = nullptr;
if (m_spare_entry) {
result = m_spare_entry;
m_spare_entry = nullptr;
result->m_pdd1 = l;
result->m_pdd2 = r;
result->m_op = op;
}
else {
void * mem = m_alloc.allocate(sizeof(op_entry));
result = new (mem) op_entry(l, r, op);
}
result->m_result = null_pdd;
return result;
}
void pdd_manager::push_entry(op_entry* e) {
SASSERT(!m_spare_entry);
m_spare_entry = e;
}
pdd_manager::PDD pdd_manager::imk_val(rational const& r) {
const_info info;
if (!m_mpq_table.find(r, info)) {
pdd_node n(m_values.size());
info.m_value_index = m_values.size();
info.m_node_index = insert_node(n);
m_mpq_table.insert(r, info);
m_values.push_back(r);
m_nodes[info.m_node_index].m_refcount = max_rc;
}
return info.m_node_index;
}
pdd_manager::PDD pdd_manager::make_node(unsigned lvl, PDD l, PDD h) {
m_is_new_node = false;
if (is_zero(h)) return l;
SASSERT(is_val(l) || level(l) <= lvl);
SASSERT(is_val(h) || level(h) <= lvl);
pdd_node n(lvl, l, h);
return insert_node(n);
}
pdd_manager::PDD pdd_manager::insert_node(pdd_node const& n) {
node_table::entry* e = m_node_table.insert_if_not_there2(n);
if (e->get_data().m_index != 0) {
unsigned result = e->get_data().m_index;
return result;
}
e->get_data().m_refcount = 0;
bool do_gc = m_free_nodes.empty();
if (do_gc && !m_disable_gc) {
gc();
e = m_node_table.insert_if_not_there2(n);
e->get_data().m_refcount = 0;
}
if (do_gc && m_free_nodes.size()*3 < m_nodes.size()) {
if (m_nodes.size() > m_max_num_pdd_nodes) {
throw mem_out();
}
alloc_free_nodes(m_nodes.size()/2);
}
SASSERT(!m_free_nodes.empty());
unsigned result = m_free_nodes.back();
m_free_nodes.pop_back();
e->get_data().m_index = result;
m_nodes[result] = e->get_data();
m_is_new_node = true;
SASSERT(!m_free_nodes.contains(result));
SASSERT(m_nodes[result].m_index == result);
return result;
}
void pdd_manager::try_gc() {
gc();
for (auto* e : m_op_cache) {
m_alloc.deallocate(sizeof(*e), e);
}
m_op_cache.reset();
SASSERT(m_op_cache.empty());
SASSERT(well_formed());
}
void pdd_manager::reserve_var(unsigned i) {
while (m_var2level.size() <= i) {
unsigned v = m_var2level.size();
m_var2pdd.push_back(make_node(v, zero_pdd, one_pdd));
m_nodes[m_var2pdd[v]].m_refcount = max_rc;
m_var2level.push_back(v);
m_level2var.push_back(v);
}
}
pdd pdd_manager::mk_var(unsigned i) {
reserve_var(i);
std::cout << m_var2pdd[i] << "\n";
return pdd(m_var2pdd[i], this);
}
pdd pdd_manager::minus(pdd const &b) {
bool first = true;
while (true) {
try {
return pdd(minus_rec(b.root), this);
}
catch (const mem_out &) {
if (!first) throw;
try_gc();
first = false;
}
}
}
pdd_manager::PDD pdd_manager::minus_rec(PDD b) {
if (is_zero(b)) {
return zero_pdd;
}
if (is_val(b)) {
return imk_val(-val(b));
}
op_entry* e1 = pop_entry(b, b, pdd_minus_op);
op_entry const* e2 = m_op_cache.insert_if_not_there(e1);
if (check_result(e1, e2, b, b, pdd_minus_op))
return e2->m_result;
push(minus_rec(lo(b)));
push(minus_rec(hi(b)));
PDD r = make_node(level(b), read(2), read(1));
pop(2);
e1->m_result = r;
return r;
}
unsigned pdd_manager::pdd_size(pdd const& b) {
init_mark();
set_mark(0);
set_mark(1);
unsigned sz = 0;
m_todo.push_back(b.root);
while (!m_todo.empty()) {
PDD r = m_todo.back();
m_todo.pop_back();
if (!is_marked(r)) {
++sz;
set_mark(r);
if (!is_marked(lo(r))) {
m_todo.push_back(lo(r));
}
if (!is_marked(hi(r))) {
m_todo.push_back(hi(r));
}
}
}
return sz;
}
void pdd_manager::alloc_free_nodes(unsigned n) {
for (unsigned i = 0; i < n; ++i) {
m_free_nodes.push_back(m_nodes.size());
m_nodes.push_back(pdd_node());
m_nodes.back().m_index = m_nodes.size() - 1;
}
m_free_nodes.reverse();
}
void pdd_manager::gc() {
m_free_nodes.reset();
IF_VERBOSE(13, verbose_stream() << "(pdd :gc " << m_nodes.size() << ")\n";);
svector<bool> reachable(m_nodes.size(), false);
for (unsigned i = m_pdd_stack.size(); i-- > 0; ) {
reachable[m_pdd_stack[i]] = true;
m_todo.push_back(m_pdd_stack[i]);
}
for (unsigned i = m_nodes.size(); i-- > 2; ) {
if (m_nodes[i].m_refcount > 0) {
reachable[i] = true;
m_todo.push_back(i);
}
}
while (!m_todo.empty()) {
PDD b = m_todo.back();
m_todo.pop_back();
SASSERT(reachable[b]);
if (is_val(b)) continue;
if (!reachable[lo(b)]) {
reachable[lo(b)] = true;
m_todo.push_back(lo(b));
}
if (!reachable[hi(b)]) {
reachable[hi(b)] = true;
m_todo.push_back(hi(b));
}
}
for (unsigned i = m_nodes.size(); i-- > 2; ) {
if (!reachable[i]) {
m_nodes[i].set_internal();
SASSERT(m_nodes[i].m_refcount == 0);
m_free_nodes.push_back(i);
}
}
// sort free nodes so that adjacent nodes are picked in order of use
std::sort(m_free_nodes.begin(), m_free_nodes.end());
m_free_nodes.reverse();
ptr_vector<op_entry> to_delete, to_keep;
for (auto* e : m_op_cache) {
if (e->m_result != null_pdd) {
to_delete.push_back(e);
}
else {
to_keep.push_back(e);
}
}
m_op_cache.reset();
for (op_entry* e : to_delete) {
m_alloc.deallocate(sizeof(*e), e);
}
for (op_entry* e : to_keep) {
m_op_cache.insert(e);
}
m_node_table.reset();
// re-populate node cache
for (unsigned i = m_nodes.size(); i-- > 2; ) {
if (reachable[i]) {
SASSERT(m_nodes[i].m_index == i);
m_node_table.insert(m_nodes[i]);
}
}
SASSERT(well_formed());
}
void pdd_manager::init_mark() {
m_mark.resize(m_nodes.size());
++m_mark_level;
if (m_mark_level == 0) {
m_mark.fill(0);
++m_mark_level;
}
}
std::ostream& pdd_manager::display(std::ostream& out, pdd const& b) {
init_mark();
m_todo.push_back(b.root);
while (!m_todo.empty()) {
PDD r = m_todo.back();
if (is_marked(r)) {
m_todo.pop_back();
}
else if (is_val(r)) {
set_mark(r);
out << r << " : " << val(r) << "\n";
m_todo.pop_back();
}
else if (!is_marked(lo(r))) {
m_todo.push_back(lo(r));
}
else if (!is_marked(hi(r))) {
m_todo.push_back(hi(r));
}
else {
out << r << " : " << var(r) << " @ " << level(r) << " " << lo(r) << " " << hi(r) << "\n";
set_mark(r);
m_todo.pop_back();
}
}
return out;
}
bool pdd_manager::well_formed() {
bool ok = true;
for (unsigned n : m_free_nodes) {
ok &= (lo(n) == 0 && hi(n) == 0 && m_nodes[n].m_refcount == 0);
if (!ok) {
IF_VERBOSE(0,
verbose_stream() << "free node is not internal " << n << " " << lo(n) << " " << hi(n) << " " << m_nodes[n].m_refcount << "\n";
display(verbose_stream()););
UNREACHABLE();
return false;
}
}
for (pdd_node const& n : m_nodes) {
if (n.is_internal()) continue;
unsigned lvl = n.m_level;
PDD lo = n.m_lo;
PDD hi = n.m_hi;
ok &= is_val(lo) || level(lo) <= lvl;
ok &= is_val(hi) || level(hi) <= lvl;
ok &= is_val(lo) || !m_nodes[lo].is_internal();
ok &= is_val(hi) || !m_nodes[hi].is_internal();
if (!ok) {
IF_VERBOSE(0, display(verbose_stream() << n.m_index << " lo " << lo << " hi " << hi << "\n"););
UNREACHABLE();
return false;
}
}
return ok;
}
std::ostream& pdd_manager::display(std::ostream& out) {
for (unsigned i = 0; i < m_nodes.size(); ++i) {
pdd_node const& n = m_nodes[i];
if (n.is_internal()) continue;
out << i << " : v" << m_level2var[n.m_level] << " " << n.m_lo << " " << n.m_hi << "\n";
}
return out;
}
pdd& pdd::operator=(pdd const& other) { unsigned r1 = root; root = other.root; m->inc_ref(root); m->dec_ref(r1); return *this; }
std::ostream& operator<<(std::ostream& out, pdd const& b) { return b.display(out); }
}

268
src/math/dd/dd_pdd.h Normal file
View file

@ -0,0 +1,268 @@
/*++
Copyright (c) 2019 Microsoft Corporation
Module Name:
dd_pdd
Abstract:
Poly DD package
Internal nodes are of the form x*hi + lo
where
- maxdegree(x, lo) = 0,
Leaf nodes are of the form (0*idx + 0), where idx is an index into m_values.
Author:
Nikolaj Bjorner (nbjorner) 2019-12-17
--*/
#ifndef DD_PDD_H_
#define DD_PDD_H_
#include "util/vector.h"
#include "util/map.h"
#include "util/small_object_allocator.h"
#include "util/rational.h"
namespace dd {
class pdd;
class pdd_manager {
friend pdd;
typedef unsigned PDD;
const PDD null_pdd = UINT_MAX;
const PDD zero_pdd = 0;
const PDD one_pdd = 1;
enum pdd_op {
pdd_add_op = 2,
pdd_sub_op = 3,
pdd_mul_op = 4,
pdd_minus_op = 5,
pdd_reduce_op = 6,
pdd_no_op = 7
};
struct pdd_node {
pdd_node(unsigned level, PDD lo, PDD hi):
m_refcount(0),
m_level(level),
m_lo(lo),
m_hi(hi),
m_index(0)
{}
pdd_node(unsigned value):
m_refcount(0),
m_level(0),
m_lo(value),
m_hi(0),
m_index(0)
{}
pdd_node(): m_refcount(0), m_level(0), m_lo(0), m_hi(0), m_index(0) {}
unsigned m_refcount : 10;
unsigned m_level : 22;
PDD m_lo;
PDD m_hi;
unsigned m_index;
unsigned hash() const { return mk_mix(m_level, m_lo, m_hi); }
bool is_internal() const { return m_lo == 0 && m_hi == 0; }
void set_internal() { m_lo = 0; m_hi = 0; }
};
struct hash_node {
unsigned operator()(pdd_node const& n) const { return n.hash(); }
};
struct eq_node {
bool operator()(pdd_node const& a, pdd_node const& b) const {
return a.m_lo == b.m_lo && a.m_hi == b.m_hi && a.m_level == b.m_level;
}
};
typedef hashtable<pdd_node, hash_node, eq_node> node_table;
struct const_info {
unsigned m_value_index;
unsigned m_node_index;
};
typedef map<rational, const_info, rational::hash_proc, rational::eq_proc> mpq_table;
struct op_entry {
op_entry(PDD l, PDD r, PDD op):
m_pdd1(l),
m_pdd2(r),
m_op(op),
m_result(0)
{}
PDD m_pdd1;
PDD m_pdd2;
PDD m_op;
PDD m_result;
unsigned hash() const { return mk_mix(m_pdd1, m_pdd2, m_op); }
};
struct hash_entry {
unsigned operator()(op_entry* e) const { return e->hash(); }
};
struct eq_entry {
bool operator()(op_entry * a, op_entry * b) const {
return a->m_pdd1 == b->m_pdd2 && a->m_pdd2 == b->m_pdd2 && a->m_op == b->m_op;
}
};
typedef ptr_hashtable<op_entry, hash_entry, eq_entry> op_table;
svector<pdd_node> m_nodes;
vector<rational> m_values;
op_table m_op_cache;
node_table m_node_table;
mpq_table m_mpq_table;
svector<PDD> m_pdd_stack;
op_entry* m_spare_entry;
svector<PDD> m_var2pdd;
unsigned_vector m_var2level, m_level2var;
unsigned_vector m_free_nodes;
small_object_allocator m_alloc;
mutable svector<unsigned> m_mark;
mutable unsigned m_mark_level;
mutable svector<double> m_count;
mutable svector<PDD> m_todo;
bool m_disable_gc;
bool m_is_new_node;
unsigned m_max_num_pdd_nodes;
PDD make_node(unsigned level, PDD l, PDD r);
PDD insert_node(pdd_node const& n);
bool is_new_node() const { return m_is_new_node; }
PDD apply(PDD arg1, PDD arg2, pdd_op op);
PDD reduce_on_match(PDD a, PDD b);
bool lm_divides(PDD p, PDD q) const;
PDD lt_quotient(PDD p, PDD q);
PDD apply_rec(PDD arg1, PDD arg2, pdd_op op);
PDD imk_val(rational const& r);
PDD minus_rec(PDD a);
void push(PDD b);
void pop(unsigned num_scopes);
PDD read(unsigned index);
op_entry* pop_entry(PDD l, PDD r, PDD op);
void push_entry(op_entry* e);
bool check_result(op_entry*& e1, op_entry const* e2, PDD a, PDD b, PDD c);
void alloc_free_nodes(unsigned n);
void init_mark();
void set_mark(unsigned i) { m_mark[i] = m_mark_level; }
bool is_marked(unsigned i) { return m_mark[i] == m_mark_level; }
static const unsigned max_rc = (1 << 10) - 1;
inline bool is_zero(PDD b) const { return b == zero_pdd; }
inline bool is_one(PDD b) const { return b == one_pdd; }
inline bool is_val(PDD b) const { return hi(b) == 0; }
inline unsigned level(PDD b) const { return m_nodes[b].m_level; }
inline unsigned var(PDD b) const { return m_level2var[level(b)]; }
inline PDD lo(PDD b) const { return m_nodes[b].m_lo; }
inline PDD hi(PDD b) const { return m_nodes[b].m_hi; }
inline rational const& val(PDD b) const { SASSERT(is_val(b)); return m_values[lo(b)]; }
inline void inc_ref(PDD b) { if (m_nodes[b].m_refcount != max_rc) m_nodes[b].m_refcount++; SASSERT(!m_free_nodes.contains(b)); }
inline void dec_ref(PDD b) { if (m_nodes[b].m_refcount != max_rc) m_nodes[b].m_refcount--; SASSERT(!m_free_nodes.contains(b)); }
inline PDD level2pdd(unsigned l) const { return m_var2pdd[m_level2var[l]]; }
unsigned pdd_size(pdd const& b);
void try_gc();
void reserve_var(unsigned v);
bool well_formed();
unsigned_vector m_p, m_q;
rational m_pc, m_qc;
pdd spoly(pdd const& a, pdd const& b, unsigned_vector const& p, unsigned_vector const& q, rational const& pc, rational const& qc);
bool common_factors(pdd const& a, pdd const& b, unsigned_vector& p, unsigned_vector& q, rational& pc, rational& qc);
struct scoped_push {
pdd_manager& m;
unsigned m_size;
scoped_push(pdd_manager& m) :m(m), m_size(m.m_pdd_stack.size()) {}
~scoped_push() { m.m_pdd_stack.shrink(m_size); }
};
public:
struct mem_out {};
pdd_manager(unsigned nodes);
~pdd_manager();
void set_max_num_nodes(unsigned n) { m_max_num_pdd_nodes = n; }
void set_var_order(unsigned_vector const& levels); // TBD: set variable order (m_var2level, m_level2var) before doing anything else.
pdd mk_var(unsigned i);
pdd mk_val(rational const& r);
pdd minus(pdd const& a);
pdd add(pdd const& a, pdd const& b);
pdd add(rational const& a, pdd const& b);
pdd sub(pdd const& a, pdd const& b);
pdd mul(pdd const& a, pdd const& b);
pdd mul(rational const& c, pdd const& b);
pdd reduce(pdd const& a, pdd const& b);
bool try_spoly(pdd const& a, pdd const& b, pdd& r);
std::ostream& display(std::ostream& out);
std::ostream& display(std::ostream& out, pdd const& b);
void gc();
};
class pdd {
friend class pdd_manager;
unsigned root;
pdd_manager* m;
pdd(unsigned root, pdd_manager* m): root(root), m(m) { m->inc_ref(root); }
public:
pdd(pdd & other): root(other.root), m(other.m) { m->inc_ref(root); }
pdd(pdd && other): root(0), m(other.m) { std::swap(root, other.root); }
pdd& operator=(pdd const& other);
~pdd() { m->dec_ref(root); }
pdd lo() const { return pdd(m->lo(root), m); }
pdd hi() const { return pdd(m->hi(root), m); }
unsigned var() const { return m->var(root); }
rational const& val() const { SASSERT(is_val()); return m->val(root); }
bool is_val() const { return m->is_val(root); }
pdd operator+(pdd const& other) const { return m->add(*this, other); }
pdd operator-(pdd const& other) const { return m->sub(*this, other); }
pdd operator*(pdd const& other) const { return m->mul(*this, other); }
pdd operator*(rational const& other) { return m->mul(other, *this); }
pdd operator+(rational const& other) { return m->add(other, *this); }
pdd reduce(pdd const& other) { return m->reduce(*this, other); }
std::ostream& display(std::ostream& out) const { return m->display(out, *this); }
bool operator==(pdd const& other) const { return root == other.root; }
bool operator!=(pdd const& other) const { return root != other.root; }
unsigned size() const { return m->pdd_size(*this); }
};
inline pdd operator*(rational const& r, pdd& b) { return b * r; }
inline pdd operator+(rational const& r, pdd& b) { return b + r; }
std::ostream& operator<<(std::ostream& out, pdd const& b);
}
#endif