package coq
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>
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 Classes
Source
Instance declaration
Source
val 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.
Source
val existing_instance :
Hints.hint_locality ->
Libnames.qualid ->
Vernacexpr.hint_info_expr option ->
unit
globality, reference, optional priority and pattern information
Source
val 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
Source
val new_instance :
locality:Hints.hint_locality ->
poly:bool ->
Constrexpr.name_decl ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
(bool * Constrexpr.constr_expr) ->
?hook:(Names.GlobRef.t -> unit) ->
Vernacexpr.hint_info_expr ->
Names.Id.t
Source
val new_instance_program :
locality:Hints.hint_locality ->
pm:Declare.OblState.t ->
poly:bool ->
Constrexpr.name_decl ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
(bool * Constrexpr.constr_expr) option ->
?hook:(Names.GlobRef.t -> unit) ->
Vernacexpr.hint_info_expr ->
Declare.OblState.t * Names.Id.t
Source
val 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
Source
val set_typeclass_transparency :
locality:Hints.hint_locality ->
Tacred.evaluable_global_reference list ->
bool ->
unit
Source
val set_typeclass_transparency_com :
locality:Hints.hint_locality ->
Libnames.qualid list ->
bool ->
unit
For generation on names based on classes only
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>