Module Vernactypes.InProof
type _ t
=
|
Ignore : unit t
|
Reject : unit t
|
Use : Declare.Proof.t t
|
UseOpt : Declare.Proof.t option t
val cast : Declare.Proof.t option -> 'a t -> 'a
Vernactypes.InProof
type _ t
=
| Ignore : unit t |
| Reject : unit t |
| Use : Declare.Proof.t t |
| UseOpt : Declare.Proof.t option t |
val cast : Declare.Proof.t option -> 'a t -> 'a