module VC_Lemma: sig .. end
sig
end
type t = {
lemma : Wp.Definitions.dlemma;
Wp.Definitions.dlemma
depends : Wp.LogicUsage.logic_lemma list;
Wp.LogicUsage.logic_lemma list
mutable sequent : Wp.Conditions.sequent option;
Wp.Conditions.sequent option
}
val is_trivial : t -> bool
t -> bool
val cache_descr : t -> (Wp.VCS.prover * Wp.VCS.result) list -> string
t -> (Wp.VCS.prover * Wp.VCS.result) list -> string