package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type vernac_toplevel =
  1. | VernacBacktrack of int * int * int
  2. | VernacDrop
  3. | VernacQuit
  4. | VernacControl of Vernacexpr.vernac_control
module Toplevel_ : sig ... end
val vernac_toplevel : Pvernac.proof_mode option -> vernac_toplevel CAst.t option Pcoq.Entry.t
OCaml

Innovation. Community. Security.