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.14.0.tar.gz
    
    
        
    
  
  
  
    
  
        sha256=b1501d686c21836302191ae30f610cca57fb309214c126518ca009363ad2cd3c
    
    
  doc/ltac_plugin/Ltac_plugin/Rewrite/index.html
Module Ltac_plugin.RewriteSource
TODO: document and clean me!
Source
type ('constr, 'redexpr) strategy_ast = - | StratId
- | StratFail
- | StratRefl
- | StratUnary of unary_strategy * ('constr, 'redexpr) strategy_ast
- | StratBinary of binary_strategy * ('constr, 'redexpr) strategy_ast * ('constr, 'redexpr) strategy_ast
- | StratConstr of 'constr * bool
- | StratTerms of 'constr list
- | StratHints of bool * string
- | StratEval of 'redexpr
- | StratFold of 'constr
Source
type rewrite_result_info = {- rew_car : EConstr.constr;
- rew_from : EConstr.constr;
- rew_to : EConstr.constr;
- rew_prf : rewrite_proof;
- rew_evars : evars;
}Source
val strategy_of_ast : 
  Tacinterp.interp_sign ->
  (Genintern.glob_constr_and_expr, Tacexpr.glob_red_expr) strategy_ast ->
  strategyEntry point for user-level "rewrite_strat"
Source
val cl_rewrite_clause : 
  (Tacinterp.interp_sign
   * (Genintern.glob_constr_and_expr
      * Genintern.glob_constr_and_expr Tactypes.bindings)) ->
  bool ->
  Locus.occurrences ->
  Names.Id.t option ->
  unit Proofview.tacticEntry point for user-level "setoid_rewrite"
Source
val is_applied_rewrite_relation : 
  Environ.env ->
  Evd.evar_map ->
  EConstr.rel_context ->
  EConstr.constr ->
  EConstr.types optionSource
val declare_relation : 
  rewrite_attributes ->
  ?binders:Constrexpr.local_binder_expr list ->
  Constrexpr.constr_expr ->
  Constrexpr.constr_expr ->
  Names.Id.t ->
  Constrexpr.constr_expr option ->
  Constrexpr.constr_expr option ->
  Constrexpr.constr_expr option ->
  unitSource
val add_setoid : 
  rewrite_attributes ->
  Constrexpr.local_binder_expr list ->
  Constrexpr.constr_expr ->
  Constrexpr.constr_expr ->
  Constrexpr.constr_expr ->
  Names.Id.t ->
  unitSource
val add_morphism_interactive : 
  rewrite_attributes ->
  Constrexpr.constr_expr ->
  Names.Id.t ->
  Declare.Proof.tSource
val add_morphism_as_parameter : 
  rewrite_attributes ->
  Constrexpr.constr_expr ->
  Names.Id.t ->
  unitSource
val add_morphism : 
  rewrite_attributes ->
  Constrexpr.local_binder_expr list ->
  Constrexpr.constr_expr ->
  Constrexpr.constr_expr ->
  Names.Id.t ->
  Declare.Proof.tSource
val get_reflexive_proof : 
  Environ.env ->
  Evd.evar_map ->
  EConstr.constr ->
  EConstr.constr ->
  Evd.evar_map * EConstr.constrSource
val get_symmetric_proof : 
  Environ.env ->
  Evd.evar_map ->
  EConstr.constr ->
  EConstr.constr ->
  Evd.evar_map * EConstr.constrSource
val get_transitive_proof : 
  Environ.env ->
  Evd.evar_map ->
  EConstr.constr ->
  EConstr.constr ->
  Evd.evar_map * EConstr.constrSource
val default_morphism : 
  ((EConstr.types * EConstr.constr option) option list
   * (EConstr.types * EConstr.types option) option) ->
  EConstr.constr ->
  EConstr.constr * EConstr.constrSource
val apply_strategy : 
  strategy ->
  Environ.env ->
  Names.Id.Set.t ->
  EConstr.constr ->
  (bool * EConstr.constr) ->
  evars ->
  rewrite_result sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >