Micromega_plugin.Certificate
module Mc = Micromega_core_plugin.Micromega
type zres = (Mc.zArithProof, int * Mc.z list) res
val q_cert_of_pos : Micromega_core_plugin.Sos_types.positivstellensatz -> Mc.q Mc.psatz
q_cert_of_pos prf
converts a Sos proof into a rational Rocq proof
val z_cert_of_pos : Micromega_core_plugin.Sos_types.positivstellensatz -> Mc.z Mc.psatz
z_cert_of_pos prf
converts a Sos proof into an integer Rocq proof
lia depth sys
generates an unsat proof for the linear constraints in sys
.
nlia depth sys
generates an unsat proof for the non-linear constraints in sys
. The solver is incomplete -- the problem is undecidable
linear_prover_with_cert depth sys
generates an unsat proof for the linear constraints in sys
. Over the rationals, the solver is complete.