Vernacstate.LemmaStack
val pop : t -> Declare.Proof.t * t option
val push : t option -> Declare.Proof.t -> t
val map : f:( Declare.Proof.t -> Declare.Proof.t ) -> t -> t
val map_top : f:( Declare.Proof.t -> Declare.Proof.t ) -> t -> t
val with_top : t -> f:( Declare.Proof.t -> 'a ) -> 'a
val get_top : t -> Declare.Proof.t
val get_all_proof_names : t -> Names.Id.t list