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/ltac_plugin/Ltac_plugin/G_obligations/index.html

Module Ltac_plugin.G_obligationsSource

Sourceval set_default_tactic : Vernacexpr.locality_flag -> Tacexpr.glob_tactic_expr -> unit
Sourceval get_default_tactic : unit -> Vernacexpr.locality_flag * unit Proofview.tactic
Sourceval print_default_tactic : unit -> Pp.t
Sourceval with_tac : (Genarg.glob_generic_argument option -> 'a) -> Tacexpr.raw_tactic_expr option -> 'a
Sourcemodule Tactic = Pltac
Sourcetype 'a withtac_argtype = (Tacexpr.raw_tactic_expr option, 'a) Genarg.abstract_argument_type
Sourceval obligation : pm:Declare.OblState.t -> (int * Names.Id.t option * Constrexpr.constr_expr option) -> Tacexpr.raw_tactic_expr option -> Declare.Proof.t
Sourceval next_obligation : pm:Declare.OblState.t -> Names.Id.t option -> Tacexpr.raw_tactic_expr option -> Declare.Proof.t
OCaml

Innovation. Community. Security.