package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type _ t =
  1. | Ignore : unit t
  2. | Reject : unit t
  3. | Use : Declare.Proof.t t
  4. | UseOpt : Declare.Proof.t option t
val cast : Declare.Proof.t option -> 'a t -> 'a