package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
val mismatched_params : Environ.env -> Constrexpr.constr_expr list -> Constr.rel_context -> 'a
val mismatched_props : Environ.env -> Constrexpr.constr_expr list -> Constr.rel_context -> 'a
val existing_instance : bool -> Libnames.qualid -> Hints.hint_info_expr option -> unit
val declare_instance_constant : Typeclasses.typeclass -> Hints.hint_info_expr -> bool -> Impargs.manual_explicitation list -> ?hook:(Names.GlobRef.t -> unit) -> Names.Id.t -> UState.universe_decl -> bool -> Evd.evar_map -> Constr.t -> Constr.types -> Names.Id.t
val new_instance : ?abstract:bool -> ?global:bool -> ?refine:bool -> program_mode:bool -> Decl_kinds.polymorphic -> Constrexpr.local_binder_expr list -> Vernacexpr.typeclass_constraint -> (bool * Constrexpr.constr_expr) option -> ?generalize:bool -> ?tac:unit Proofview.tactic -> ?hook:(Names.GlobRef.t -> unit) -> Hints.hint_info_expr -> Names.Id.t
val set_typeclass_transparency : Names.evaluable_global_reference -> bool -> bool -> unit
val id_of_class : Typeclasses.typeclass -> Names.Id.t