package coq

  1. Overview
  2. Docs
Formal proof management system

Install

Dune Dependency

Authors

Maintainers

Sources

coq-8.15.2.tar.gz
sha256=13a67c0a4559ae22e9765c8fdb88957b16c2b335a2d5f47e4d6d9b4b8b299926

doc/coq-core.proofs/Tacmach/Old/index.html

Module Tacmach.OldSource

Sourcetype tactic = Evar.t Evd.sigma -> Evar.t list Evd.sigma
Sourceval sig_it : 'a Evd.sigma -> 'a
Sourceval re_sig : 'a -> Evd.evar_map -> 'a Evd.sigma
Sourceval pf_nth_hyp_id : Goal.goal Evd.sigma -> int -> Names.Id.t
Sourceval pf_ids_of_hyps : Goal.goal Evd.sigma -> Names.Id.t list
  • deprecated This is a no-op now
Sourceval pf_apply : (Environ.env -> Evd.evar_map -> 'a) -> Goal.goal Evd.sigma -> 'a
Sourceval pf_eapply : (Environ.env -> Evd.evar_map -> 'a -> Evd.evar_map * 'b) -> Goal.goal Evd.sigma -> 'a -> Goal.goal Evd.sigma * 'b
  • deprecated Use the version in Tacmach.New
  • deprecated Use the version in Tacmach.New
  • deprecated Use the version in Tacmach.New
  • deprecated Use the version in Tacmach.New
  • deprecated Use the version in Tacmach.New
  • deprecated Use Tacred.pf_reduce_to_atomic_ind
  • deprecated Use the version in Tacmach.New
  • deprecated Use Tacred.unfoldn
  • deprecated Use Environ.constant_value_in
  • deprecated Use the version in Tacmach.New

Pretty-printing functions (debug only).

OCaml

Innovation. Community. Security.