package coq-core
 sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >
  
  
On This Page
  
  
  The Coq Proof Assistant -- Core Binaries and Tools
Install
    
    dune-project
 Dependency
Authors
Maintainers
Sources
  
    
      coq-8.18.0.tar.gz
    
    
        
    
  
  
  
    
  
  
    
  
        md5=8d852367b54f095d9fbabd000304d450
    
    
  sha512=46922d5f2eb6802a148a52fd3e7f0be8370c93e7bc33cee05cf4a2044290845b10ccddbaa306f29c808e7c5019700763e37e45ff6deb507b874a4348010fed50
    
    
  doc/coq-core.vernac/ComFixpoint/index.html
Module ComFixpointSource
Fixpoints and cofixpoints
Entry points for the vernacular commands Fixpoint and CoFixpoint
Source
val do_fixpoint_interactive : 
  scope:Locality.definition_scope ->
  ?clearbody:bool ->
  poly:bool ->
  ?typing_flags:Declarations.typing_flags ->
  ?deprecation:Deprecation.t ->
  Vernacexpr.fixpoint_expr list ->
  Declare.Proof.tSource
val do_fixpoint : 
  ?scope:Locality.definition_scope ->
  ?clearbody:bool ->
  poly:bool ->
  ?typing_flags:Declarations.typing_flags ->
  ?deprecation:Deprecation.t ->
  ?using:Vernacexpr.section_subset_expr ->
  Vernacexpr.fixpoint_expr list ->
  unitSource
val do_cofixpoint_interactive : 
  scope:Locality.definition_scope ->
  poly:bool ->
  ?deprecation:Deprecation.t ->
  Vernacexpr.cofixpoint_expr list ->
  Declare.Proof.tSource
val do_cofixpoint : 
  scope:Locality.definition_scope ->
  poly:bool ->
  ?deprecation:Deprecation.t ->
  ?using:Vernacexpr.section_subset_expr ->
  Vernacexpr.cofixpoint_expr list ->
  unitInternal API
Typing global fixpoints and cofixpoint_expr
Source
val adjust_rec_order : 
  structonly:bool ->
  Constrexpr.local_binder_expr list ->
  Constrexpr.recursion_order_expr option ->
  Names.lident optionSource
type ('constr, 'types) recursive_preentry =
  Names.Id.t list * Sorts.relevance list * 'constr option list * 'types listnames / relevance / defs / types
Source
val interp_recursive : 
  Environ.env ->
  program_mode:bool ->
  cofix:bool ->
  Names.lident option Vernacexpr.fix_expr_gen list ->
  (Environ.env * EConstr.named_context * UState.universe_decl * Evd.evar_map)
  * (EConstr.t, EConstr.types) recursive_preentry
  * (EConstr.rel_context * Impargs.manual_implicits * int option) listExported for Program
Exported for Funind
Source
val interp_fixpoint : 
  ?check_recursivity:bool ->
  ?typing_flags:Declarations.typing_flags ->
  cofix:bool ->
  Names.lident option Vernacexpr.fix_expr_gen list ->
  (Constr.t, Constr.types) recursive_preentry
  * UState.universe_decl
  * UState.t
  * (EConstr.rel_context * Impargs.manual_implicits * int option) listSource
val compute_possible_guardness_evidences : 
  (('a, 'b) Context.Rel.pt * 'c * int option) ->
  int listVery private function, do not use
 sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >
  
  
  On This Page