package coq

  1. Overview
  2. Docs
Formal proof management system

Install

Dune Dependency

Authors

Maintainers

Sources

coq-8.15.1.tar.gz
sha256=513e953b7183d478acb75fd6e80e4dc32ac1a918cf4343ac31a859cfb4e9aad2

doc/coq-core.toplevel/G_toplevel/index.html

Module G_toplevelSource

Sourcetype vernac_toplevel =
  1. | VernacBackTo of int
  2. | VernacDrop
  3. | VernacQuit
  4. | VernacControl of Vernacexpr.vernac_control
  5. | VernacShowGoal of {
    1. gid : int;
    2. sid : int;
    }
  6. | VernacShowProofDiffs of Proof_diffs.diffOpt
Sourcemodule Toplevel_ : sig ... end
Sourceval err : unit -> 'a
Sourceval test_show_goal : unit Pcoq.Entry.t
Sourceval vernac_toplevel : Pvernac.proof_mode option -> vernac_toplevel option Pcoq.Entry.t
OCaml

Innovation. Community. Security.