Module Vernacextend.OutProof
type _ t
=
|
No : unit t
|
Close : unit t
|
Yes : Declare.Proof.t t
type result
=
|
Ignored
|
Closed
|
Open of Declare.Proof.t
Vernacextend.OutProof
type _ t
=
| No : unit t |
| Close : unit t |
| Yes : Declare.Proof.t t |
type result
=
| Ignored |
| Closed |
| Open of Declare.Proof.t |