package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
  • deprecated Use [Declare.Proof.t]
val map_proof : (Proof.t -> Proof.t) -> Declare.Proof.t -> Declare.Proof.t
val get_proof : Declare.Proof.t -> Proof.t
type opacity_flag = Declare.opacity_flag =
  1. | Opaque
    (*
    • deprecated Use [Declare.Opaque]
    *)
  2. | Transparent
    (*
    • deprecated Use [Declare.Transparent]
    *)
OCaml

Innovation. Community. Security.