Ltac_plugin.RewriteSourceTODO: document and clean me!
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 'constrtype rewrite_result_info = {rew_car : EConstr.constr;rew_from : EConstr.constr;rew_to : EConstr.constr;rew_prf : rewrite_proof;rew_evars : evars;}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"
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"
val is_applied_rewrite_relation :
Environ.env ->
Evd.evar_map ->
EConstr.rel_context ->
EConstr.constr ->
EConstr.types optionval 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 ->
unitval add_setoid :
rewrite_attributes ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr ->
Names.Id.t ->
unitval add_morphism_interactive :
rewrite_attributes ->
Constrexpr.constr_expr ->
Names.Id.t ->
Declare.Proof.tval add_morphism_as_parameter :
rewrite_attributes ->
Constrexpr.constr_expr ->
Names.Id.t ->
unitval add_morphism :
rewrite_attributes ->
Constrexpr.local_binder_expr list ->
Constrexpr.constr_expr ->
Constrexpr.constr_expr ->
Names.Id.t ->
Declare.Proof.tval get_reflexive_proof :
Environ.env ->
Evd.evar_map ->
EConstr.constr ->
EConstr.constr ->
Evd.evar_map * EConstr.constrval get_symmetric_proof :
Environ.env ->
Evd.evar_map ->
EConstr.constr ->
EConstr.constr ->
Evd.evar_map * EConstr.constrval get_transitive_proof :
Environ.env ->
Evd.evar_map ->
EConstr.constr ->
EConstr.constr ->
Evd.evar_map * EConstr.constrval default_morphism :
((EConstr.types * EConstr.constr option) option list
* (EConstr.types * EConstr.types option) option) ->
EConstr.constr ->
EConstr.constr * EConstr.constrval apply_strategy :
strategy ->
Environ.env ->
Names.Id.Set.t ->
EConstr.constr ->
(bool * EConstr.constr) ->
evars ->
rewrite_result