Micromega_plugin.Polynomial
module Mc = Micromega
module Monomial : sig ... end
module MonMap : sig ... end
module Poly : sig ... end
Representation of polonomial with rational coefficient. a1.m1 + ... + c where
val eval_op : op -> NumCompat.Q.t -> NumCompat.Q.t -> bool
val is_strict : cstr -> bool
is_strict c
module LinPoly : sig ... end
Linear(ised) polynomials represented as a Vect.t
i.e a sorted association list. The constant is the coefficient of the variable 0
module ProofFormat : sig ... end
Proof format used by the proof-generating procedures. It is fairly close to Coq format but a bit more liberal.
val output_cstr : Stdlib.out_channel -> cstr -> unit
module WithProof : sig ... end
module WithProof
constructs polynomials packed with the proof that their sign is correct.
module BoundWithProof : sig ... end