3
0
Fork 0
mirror of https://github.com/Z3Prover/z3 synced 2026-01-19 00:38:57 +00:00

Convert internal class enums to enum class for type safety (#8158)

* Initial plan

* Convert plain enums to enum class in EUF module

- Convert eq_status in euf::ac_plugin to enum class
- Convert undo_kind in euf::ac_plugin to enum class
- Convert undo_t in euf::arith_plugin to enum class
- Convert to_merge_t in euf::egraph to enum class
- Update all usage sites to use scoped enum syntax

Co-authored-by: NikolajBjorner <3085284+NikolajBjorner@users.noreply.github.com>

* Convert more plain enums to enum class

- Convert state enum in substitution class
- Convert instruction enum in generic_model_converter class
- Convert eq_type enum in bit2int class
- Update all usage sites to use scoped enum syntax

Co-authored-by: NikolajBjorner <3085284+NikolajBjorner@users.noreply.github.com>

---------

Co-authored-by: copilot-swe-agent[bot] <198982749+Copilot@users.noreply.github.com>
Co-authored-by: NikolajBjorner <3085284+NikolajBjorner@users.noreply.github.com>
This commit is contained in:
Copilot 2026-01-11 17:44:59 -08:00 committed by GitHub
parent 31122b0c10
commit ee037dcafe
No known key found for this signature in database
GPG key ID: B5690EEEBB952194
11 changed files with 54 additions and 54 deletions

View file

@ -32,7 +32,7 @@ Notes:
void generic_model_converter::add(func_decl * d, expr* e) { void generic_model_converter::add(func_decl * d, expr* e) {
VERIFY(e); VERIFY(e);
VERIFY(d->get_range() == e->get_sort()); VERIFY(d->get_range() == e->get_sort());
m_entries.push_back(entry(d, e, m, ADD)); m_entries.push_back(entry(d, e, m, instruction::ADD));
} }
void generic_model_converter::operator()(model_ref & md) { void generic_model_converter::operator()(model_ref & md) {
@ -138,9 +138,9 @@ void generic_model_converter::convert_initialize_value(vector<std::pair<expr_ref
auto& [var, value] = var2value[i]; auto& [var, value] = var2value[i];
for (auto const& e : m_entries) { for (auto const& e : m_entries) {
switch (e.m_instruction) { switch (e.m_instruction) {
case HIDE: case instruction::HIDE:
break; break;
case ADD: case instruction::ADD:
if (is_uninterp_const(var) && e.m_f == to_app(var)->get_decl()) if (is_uninterp_const(var) && e.m_f == to_app(var)->get_decl())
convert_initialize_value(e.m_def, i, var2value); convert_initialize_value(e.m_def, i, var2value);
break; break;
@ -203,14 +203,14 @@ void generic_model_converter::get_units(obj_map<expr, bool>& units) {
for (unsigned i = m_entries.size(); i-- > 0;) { for (unsigned i = m_entries.size(); i-- > 0;) {
entry const& e = m_entries[i]; entry const& e = m_entries[i];
switch (e.m_instruction) { switch (e.m_instruction) {
case HIDE: case instruction::HIDE:
tmp = m.mk_const(e.m_f); tmp = m.mk_const(e.m_f);
if (units.contains(tmp)) { if (units.contains(tmp)) {
m.dec_ref(tmp); m.dec_ref(tmp);
units.remove(tmp); units.remove(tmp);
} }
break; break;
case ADD: case instruction::ADD:
if (e.m_f->get_arity() == 0 && m.is_bool(e.m_f->get_range())) { if (e.m_f->get_arity() == 0 && m.is_bool(e.m_f->get_range())) {
tmp = m.mk_const(e.m_f); tmp = m.mk_const(e.m_f);
if (units.contains(tmp)) { if (units.contains(tmp)) {

View file

@ -23,7 +23,7 @@ Notes:
class generic_model_converter : public model_converter { class generic_model_converter : public model_converter {
public: public:
enum instruction { HIDE, ADD }; enum class instruction { HIDE, ADD };
struct entry { struct entry {
func_decl_ref m_f; func_decl_ref m_f;
expr_ref m_def; expr_ref m_def;
@ -44,7 +44,7 @@ public:
void hide(expr* e) { SASSERT(is_app(e) && to_app(e)->get_num_args() == 0); hide(to_app(e)->get_decl()); } void hide(expr* e) { SASSERT(is_app(e) && to_app(e)->get_num_args() == 0); hide(to_app(e)->get_decl()); }
void hide(func_decl * f) { m_entries.push_back(entry(f, nullptr, m, HIDE)); } void hide(func_decl * f) { m_entries.push_back(entry(f, nullptr, m, instruction::HIDE)); }
void add(func_decl * d, expr* e); void add(func_decl * d, expr* e);

View file

@ -154,64 +154,64 @@ namespace euf {
for (auto arg : ns) { for (auto arg : ns) {
arg->shared.push_back(idx); arg->shared.push_back(idx);
m_node_trail.push_back(arg); m_node_trail.push_back(arg);
push_undo(is_add_shared_index); push_undo(undo_kind::is_add_shared_index);
} }
m_shared_nodes.setx(n->get_id(), true, false); m_shared_nodes.setx(n->get_id(), true, false);
sort(monomial(m)); sort(monomial(m));
m_shared_todo.insert(idx); m_shared_todo.insert(idx);
m_shared.push_back({ n, m, justification::axiom(get_id()) }); m_shared.push_back({ n, m, justification::axiom(get_id()) });
push_undo(is_register_shared); push_undo(undo_kind::is_register_shared);
} }
void ac_plugin::push_scope_eh() { void ac_plugin::push_scope_eh() {
push_undo(is_push_scope); push_undo(undo_kind::is_push_scope);
} }
void ac_plugin::undo() { void ac_plugin::undo() {
auto k = m_undo.back(); auto k = m_undo.back();
m_undo.pop_back(); m_undo.pop_back();
switch (k) { switch (k) {
case is_queue_eq: { case undo_kind::is_queue_eq: {
m_queued.pop_back(); m_queued.pop_back();
break; break;
} }
case is_add_node: { case undo_kind::is_add_node: {
auto* n = m_node_trail.back(); auto* n = m_node_trail.back();
m_node_trail.pop_back(); m_node_trail.pop_back();
m_nodes[n->n->get_id()] = nullptr; m_nodes[n->n->get_id()] = nullptr;
n->~node(); n->~node();
break; break;
} }
case is_push_scope: { case undo_kind::is_push_scope: {
m_active.reset(); m_active.reset();
m_passive.reset(); m_passive.reset();
m_units.reset(); m_units.reset();
m_queue_head = 0; m_queue_head = 0;
break; break;
} }
case is_add_monomial: { case undo_kind::is_add_monomial: {
m_monomials.pop_back(); m_monomials.pop_back();
break; break;
} }
case is_add_shared_index: { case undo_kind::is_add_shared_index: {
auto n = m_node_trail.back(); auto n = m_node_trail.back();
m_node_trail.pop_back(); m_node_trail.pop_back();
n->shared.pop_back(); n->shared.pop_back();
break; break;
} }
case is_add_eq_index: { case undo_kind::is_add_eq_index: {
auto n = m_node_trail.back(); auto n = m_node_trail.back();
m_node_trail.pop_back(); m_node_trail.pop_back();
n->eqs.pop_back(); n->eqs.pop_back();
break; break;
} }
case is_register_shared: { case undo_kind::is_register_shared: {
auto s = m_shared.back(); auto s = m_shared.back();
m_shared_nodes[s.n->get_id()] = false; m_shared_nodes[s.n->get_id()] = false;
m_shared.pop_back(); m_shared.pop_back();
break; break;
} }
case is_update_shared: { case undo_kind::is_update_shared: {
auto [id, s] = m_update_shared_trail.back(); auto [id, s] = m_update_shared_trail.back();
m_shared[id] = s; m_shared[id] = s;
m_update_shared_trail.pop_back(); m_update_shared_trail.pop_back();
@ -345,7 +345,7 @@ namespace euf {
if (l == r) if (l == r)
return; return;
m_queued.push_back({ l, r }); m_queued.push_back({ l, r });
push_undo(is_queue_eq); push_undo(undo_kind::is_queue_eq);
} }
bool ac_plugin::init_equation(eq eq, bool is_active) { bool ac_plugin::init_equation(eq eq, bool is_active) {
@ -376,7 +376,7 @@ namespace euf {
if (!n->n->is_marked2()) { if (!n->n->is_marked2()) {
n->eqs.push_back(eq_id); n->eqs.push_back(eq_id);
n->n->mark2(); n->n->mark2();
push_undo(is_add_eq_index); push_undo(undo_kind::is_add_eq_index);
m_node_trail.push_back(n); m_node_trail.push_back(n);
for (auto s : n->shared) for (auto s : n->shared)
m_shared_todo.insert(s); m_shared_todo.insert(s);
@ -387,7 +387,7 @@ namespace euf {
if (!n->n->is_marked2()) { if (!n->n->is_marked2()) {
n->eqs.push_back(eq_id); n->eqs.push_back(eq_id);
n->n->mark2(); n->n->mark2();
push_undo(is_add_eq_index); push_undo(undo_kind::is_add_eq_index);
m_node_trail.push_back(n); m_node_trail.push_back(n);
for (auto s : n->shared) for (auto s : n->shared)
m_shared_todo.insert(s); m_shared_todo.insert(s);
@ -541,7 +541,7 @@ namespace euf {
unsigned ac_plugin::to_monomial(enode* e, ptr_vector<node> const& ms) { unsigned ac_plugin::to_monomial(enode* e, ptr_vector<node> const& ms) {
unsigned id = m_monomials.size(); unsigned id = m_monomials.size();
m_monomials.push_back({ ms, bloom(), e }); m_monomials.push_back({ ms, bloom(), e });
push_undo(is_add_monomial); push_undo(undo_kind::is_add_monomial);
return id; return id;
} }
@ -581,7 +581,7 @@ namespace euf {
if (m_nodes.size() > id && m_nodes[id]) if (m_nodes.size() > id && m_nodes[id])
return m_nodes[id]; return m_nodes[id];
auto* r = node::mk(get_region(), n); auto* r = node::mk(get_region(), n);
push_undo(is_add_node); push_undo(undo_kind::is_add_node);
m_nodes.setx(id, r, nullptr); m_nodes.setx(id, r, nullptr);
m_node_trail.push_back(r); m_node_trail.push_back(r);
if (is_op(n)) { if (is_op(n)) {
@ -1137,7 +1137,7 @@ namespace euf {
n->eqs.push_back(eq); n->eqs.push_back(eq);
m_node_trail.push_back(n); m_node_trail.push_back(n);
n->n->mark2(); n->n->mark2();
push_undo(is_add_eq_index); push_undo(undo_kind::is_add_eq_index);
} }
} }
for (auto n : old_r) for (auto n : old_r)
@ -1435,13 +1435,13 @@ namespace euf {
n->shared.push_back(idx); n->shared.push_back(idx);
m_shared_todo.insert(idx); m_shared_todo.insert(idx);
m_node_trail.push_back(n); m_node_trail.push_back(n);
push_undo(is_add_shared_index); push_undo(undo_kind::is_add_shared_index);
} }
} }
for (auto n : monomial(old_m)) for (auto n : monomial(old_m))
n->n->unmark2(); n->n->unmark2();
m_update_shared_trail.push_back({ idx, s }); m_update_shared_trail.push_back({ idx, s });
push_undo(is_update_shared); push_undo(undo_kind::is_update_shared);
m_shared[idx].m = new_m; m_shared[idx].m = new_m;
m_shared[idx].j = j; m_shared[idx].j = j;
TRACE(plugin_verbose, tout << "shared simplified to " << m_pp_ll(*this, monomial(new_m)) << "\n"); TRACE(plugin_verbose, tout << "shared simplified to " << m_pp_ll(*this, monomial(new_m)) << "\n");

View file

@ -56,7 +56,7 @@ namespace euf {
uint64_t m_filter = 0; uint64_t m_filter = 0;
}; };
enum eq_status { enum class eq_status {
is_processed_eq, is_passive_eq, is_to_simplify_eq, is_reducing_eq, is_dead_eq is_processed_eq, is_passive_eq, is_to_simplify_eq, is_reducing_eq, is_dead_eq
}; };
@ -65,7 +65,7 @@ namespace euf {
eq(unsigned l, unsigned r, justification j): eq(unsigned l, unsigned r, justification j):
l(l), r(r), j(j) {} l(l), r(r), j(j) {}
unsigned l, r; // refer to monomials unsigned l, r; // refer to monomials
eq_status status = is_to_simplify_eq; eq_status status = eq_status::is_to_simplify_eq;
justification j; // justification for equality justification j; // justification for equality
}; };
@ -146,7 +146,7 @@ namespace euf {
// backtrackable state // backtrackable state
enum undo_kind { enum class undo_kind {
is_queue_eq, is_queue_eq,
is_add_monomial, is_add_monomial,
is_add_node, is_add_node,

View file

@ -25,7 +25,7 @@ namespace euf {
class egraph; class egraph;
class arith_plugin : public plugin { class arith_plugin : public plugin {
enum undo_t { undo_add, undo_mul }; enum class undo_t { undo_add, undo_mul };
arith_util a; arith_util a;
svector<undo_t> m_undo; svector<undo_t> m_undo;
ac_plugin m_add, m_mul; ac_plugin m_add, m_mul;

View file

@ -661,14 +661,14 @@ namespace euf {
for (; i < m_to_merge.size() && m.limit().inc() && !inconsistent(); ++i) { for (; i < m_to_merge.size() && m.limit().inc() && !inconsistent(); ++i) {
auto const& w = m_to_merge[i]; auto const& w = m_to_merge[i];
switch (w.t) { switch (w.t) {
case to_merge_plain: case to_merge_t::to_merge_plain:
case to_merge_comm: case to_merge_t::to_merge_comm:
merge(w.a, w.b, justification::congruence(w.commutativity(), m_congruence_timestamp++)); merge(w.a, w.b, justification::congruence(w.commutativity(), m_congruence_timestamp++));
break; break;
case to_justified: case to_merge_t::to_justified:
merge(w.a, w.b, w.j); merge(w.a, w.b, w.j);
break; break;
case to_add_literal: case to_merge_t::to_add_literal:
add_literal(w.a, w.b); add_literal(w.a, w.b);
break; break;
} }

View file

@ -88,15 +88,15 @@ namespace euf {
typedef ptr_vector<trail> trail_stack; typedef ptr_vector<trail> trail_stack;
enum to_merge_t { to_merge_plain, to_merge_comm, to_justified, to_add_literal }; enum class to_merge_t { to_merge_plain, to_merge_comm, to_justified, to_add_literal };
struct to_merge { struct to_merge {
enode* a, * b; enode* a, * b;
to_merge_t t; to_merge_t t;
justification j; justification j;
bool commutativity() const { return t == to_merge_comm; } bool commutativity() const { return t == to_merge_t::to_merge_comm; }
to_merge(enode* a, enode* b, bool c) : a(a), b(b), t(c ? to_merge_comm : to_merge_plain) {} to_merge(enode* a, enode* b, bool c) : a(a), b(b), t(c ? to_merge_t::to_merge_comm : to_merge_t::to_merge_plain) {}
to_merge(enode* a, enode* b, justification j): a(a), b(b), t(to_justified), j(j) {} to_merge(enode* a, enode* b, justification j): a(a), b(b), t(to_merge_t::to_justified), j(j) {}
to_merge(enode* p, enode* ante): a(p), b(ante), t(to_add_literal) {} to_merge(enode* p, enode* ante): a(p), b(ante), t(to_merge_t::to_add_literal) {}
}; };
struct stats { struct stats {

View file

@ -138,14 +138,14 @@ bool bit2int::mk_comp(eq_type ty, expr* e1, expr* e2, expr_ref& result) {
align_sizes(tmp1, tmp2); align_sizes(tmp1, tmp2);
SASSERT(m_bv_util.get_bv_size(tmp1) == m_bv_util.get_bv_size(tmp2)); SASSERT(m_bv_util.get_bv_size(tmp1) == m_bv_util.get_bv_size(tmp2));
switch(ty) { switch(ty) {
case lt: case eq_type::lt:
tmp3 = m_rewriter.mk_ule(tmp2, tmp1); tmp3 = m_rewriter.mk_ule(tmp2, tmp1);
result = m.mk_not(tmp3); result = m.mk_not(tmp3);
break; break;
case le: case eq_type::le:
result = m_rewriter.mk_ule(tmp1, tmp2); result = m_rewriter.mk_ule(tmp1, tmp2);
break; break;
case eq: case eq_type::eq:
result = m.mk_eq(tmp1, tmp2); result = m.mk_eq(tmp1, tmp2);
break; break;
} }
@ -313,7 +313,7 @@ void bit2int::visit(app* n) {
is_bv_poly(e2, pos2, neg2) && is_bv_poly(e2, pos2, neg2) &&
mk_add(pos1, neg2, tmp1) && mk_add(pos1, neg2, tmp1) &&
mk_add(neg1, pos2, tmp2) && mk_add(neg1, pos2, tmp2) &&
mk_comp(eq, tmp1, tmp2, result)) { mk_comp(eq_type::eq, tmp1, tmp2, result)) {
cache_result(n, result); cache_result(n, result);
} }
else if (m_arith_util.is_le(n) && else if (m_arith_util.is_le(n) &&
@ -321,7 +321,7 @@ void bit2int::visit(app* n) {
is_bv_poly(e2, pos2, neg2) && is_bv_poly(e2, pos2, neg2) &&
mk_add(pos1, neg2, tmp1) && mk_add(pos1, neg2, tmp1) &&
mk_add(neg1, pos2, tmp2) && mk_add(neg1, pos2, tmp2) &&
mk_comp(le, tmp1, tmp2, result)) { mk_comp(eq_type::le, tmp1, tmp2, result)) {
cache_result(n, result); cache_result(n, result);
} }
else if (m_arith_util.is_lt(n) && else if (m_arith_util.is_lt(n) &&
@ -329,7 +329,7 @@ void bit2int::visit(app* n) {
is_bv_poly(e2, pos2, neg2) && is_bv_poly(e2, pos2, neg2) &&
mk_add(pos1, neg2, tmp1) && mk_add(pos1, neg2, tmp1) &&
mk_add(neg1, pos2, tmp2) && mk_add(neg1, pos2, tmp2) &&
mk_comp(lt, tmp1, tmp2, result)) { mk_comp(eq_type::lt, tmp1, tmp2, result)) {
cache_result(n, result); cache_result(n, result);
} }
else if (m_arith_util.is_ge(n) && else if (m_arith_util.is_ge(n) &&
@ -337,7 +337,7 @@ void bit2int::visit(app* n) {
is_bv_poly(e2, pos2, neg2) && is_bv_poly(e2, pos2, neg2) &&
mk_add(pos1, neg2, tmp1) && mk_add(pos1, neg2, tmp1) &&
mk_add(neg1, pos2, tmp2) && mk_add(neg1, pos2, tmp2) &&
mk_comp(le, tmp2, tmp1, result)) { mk_comp(eq_type::le, tmp2, tmp1, result)) {
cache_result(n, result); cache_result(n, result);
} }
else if (m_arith_util.is_gt(n) && else if (m_arith_util.is_gt(n) &&
@ -345,7 +345,7 @@ void bit2int::visit(app* n) {
is_bv_poly(e2, pos2, neg2) && is_bv_poly(e2, pos2, neg2) &&
mk_add(pos1, neg2, tmp1) && mk_add(pos1, neg2, tmp1) &&
mk_add(neg1, pos2, tmp2) && mk_add(neg1, pos2, tmp2) &&
mk_comp(lt, tmp2, tmp1, result)) { mk_comp(eq_type::lt, tmp2, tmp1, result)) {
cache_result(n, result); cache_result(n, result);
} }
else if (m_arith_util.is_mod(n) && else if (m_arith_util.is_mod(n) &&

View file

@ -27,7 +27,7 @@ class bit2int {
protected: protected:
typedef rational numeral; typedef rational numeral;
enum eq_type { enum class eq_type {
lt, lt,
le, le,
eq eq

View file

@ -26,7 +26,7 @@ substitution::substitution(ast_manager & m):
m_manager(m), m_manager(m),
m_refs(m), m_refs(m),
m_new_exprs(m), m_new_exprs(m),
m_state(CLEAN) { m_state(state::CLEAN) {
} }
void substitution::reset() { void substitution::reset() {
@ -44,7 +44,7 @@ void substitution::reset_cache() {
m_apply_cache.reset(); m_apply_cache.reset();
m_new_exprs.reset(); m_new_exprs.reset();
m_state = CLEAN; m_state = state::CLEAN;
} }
void substitution::pop_scope(unsigned num_scopes) { void substitution::pop_scope(unsigned num_scopes) {
@ -79,10 +79,10 @@ void substitution::apply(unsigned num_actual_offsets, unsigned const * deltas, e
// It is incorrect to cache results between different calls if we are applying a substitution // It is incorrect to cache results between different calls if we are applying a substitution
// modulo a substitution s -> t. // modulo a substitution s -> t.
if (m_state == INSERT || s != expr_offset(nullptr,0)) if (m_state == state::INSERT || s != expr_offset(nullptr,0))
reset_cache(); reset_cache();
m_state = APPLY; m_state = state::APPLY;
unsigned j; unsigned j;
expr * e = nullptr; expr * e = nullptr;

View file

@ -60,7 +60,7 @@ class substitution {
// keep track of how substitution state was last updated. // keep track of how substitution state was last updated.
enum state { CLEAN, APPLY, INSERT }; enum class state { CLEAN, APPLY, INSERT };
state m_state; state m_state;
#ifdef Z3DEBUG #ifdef Z3DEBUG
@ -137,7 +137,7 @@ public:
m_vars.push_back(var_offset(v_idx, offset)); m_vars.push_back(var_offset(v_idx, offset));
m_refs.push_back(t.get_expr()); m_refs.push_back(t.get_expr());
m_subst.insert(v_idx, offset, t); m_subst.insert(v_idx, offset, t);
m_state = INSERT; m_state = state::INSERT;
} }
void insert(var * v, unsigned offset, expr_offset const & t) { insert(v->get_idx(), offset, t); } void insert(var * v, unsigned offset, expr_offset const & t) { insert(v->get_idx(), offset, t); }
void insert(expr_offset v, expr_offset const & t) { void insert(expr_offset v, expr_offset const & t) {