package coq

  1. Overview
  2. Docs
Formal proof management system

Install

dune-project
 Dependency

Authors

Maintainers

Sources

coq-8.15.1.tar.gz
sha256=513e953b7183d478acb75fd6e80e4dc32ac1a918cf4343ac31a859cfb4e9aad2

doc/coq-core.vernac/Classes/index.html

Module ClassesSource

Instance declaration

Sourceval declare_instance : ?warn:bool -> Environ.env -> Evd.evar_map -> Typeclasses.hint_info option -> Hints.hint_locality -> Names.GlobRef.t -> unit

Declares the given global reference as an instance of its type. Does nothing — or emit a “not-a-class” warning if the warn argument is set — when said type is not a registered type class.

Sourceval existing_instance : Hints.hint_locality -> Libnames.qualid -> Vernacexpr.hint_info_expr option -> unit

globality, reference, optional priority and pattern information

Sourceval new_instance_interactive : locality:Hints.hint_locality -> poly:bool -> Constrexpr.name_decl -> Constrexpr.local_binder_expr list -> Constrexpr.constr_expr -> ?tac:unit Proofview.tactic -> ?hook:(Names.GlobRef.t -> unit) -> Vernacexpr.hint_info_expr -> (bool * Constrexpr.constr_expr) option -> Names.Id.t * Declare.Proof.t
Sourceval declare_new_instance : locality:Hints.hint_locality -> program_mode:bool -> poly:bool -> Constrexpr.ident_decl -> Constrexpr.local_binder_expr list -> Constrexpr.constr_expr -> Vernacexpr.hint_info_expr -> unit

Setting opacity

Sourceval set_typeclass_transparency : locality:Hints.hint_locality -> Tacred.evaluable_global_reference list -> bool -> unit
Sourceval tc_transparency_locality : Hints.hint_locality Attributes.attribute
Sourceval set_typeclass_transparency_com : locality:Hints.hint_locality -> Libnames.qualid list -> bool -> unit

For generation on names based on classes only

Sourceval refine_att : bool Attributes.attribute
Sourcemodule Internal : sig ... end