package coq

  1. Overview
  2. Docs
Formal proof management system

Install

Dune Dependency

Authors

Maintainers

Sources

coq-8.14.1.tar.gz
sha256=3cbfc1e1a72b16d4744f5b64ede59586071e31d9c11c811a0372060727bfd9c3

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 -> Goptions.option_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 : Goptions.option_locality -> Libnames.qualid -> Vernacexpr.hint_info_expr option -> unit

globality, reference, optional priority and pattern information

Sourceval new_instance_interactive : ?locality:Goptions.option_locality -> poly:bool -> Constrexpr.name_decl -> Constrexpr.local_binder_expr list -> Constrexpr.constr_expr -> ?generalize:bool -> ?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 new_instance : ?locality:Goptions.option_locality -> poly:bool -> Constrexpr.name_decl -> Constrexpr.local_binder_expr list -> Constrexpr.constr_expr -> (bool * Constrexpr.constr_expr) -> ?generalize:bool -> ?hook:(Names.GlobRef.t -> unit) -> Vernacexpr.hint_info_expr -> Names.Id.t
Sourceval new_instance_program : ?locality:Goptions.option_locality -> pm:Declare.OblState.t -> poly:bool -> Constrexpr.name_decl -> Constrexpr.local_binder_expr list -> Constrexpr.constr_expr -> (bool * Constrexpr.constr_expr) option -> ?generalize:bool -> ?hook:(Names.GlobRef.t -> unit) -> Vernacexpr.hint_info_expr -> Declare.OblState.t * Names.Id.t
Sourceval declare_new_instance : ?locality:Goptions.option_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 : Tacred.evaluable_global_reference -> bool -> bool -> unit

For generation on names based on classes only

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

Innovation. Community. Security.