package coq
Formal proof management system
Install
Dune Dependency
Authors
Maintainers
Sources
coq-8.14.1.tar.gz
sha256=3cbfc1e1a72b16d4744f5b64ede59586071e31d9c11c811a0372060727bfd9c3
doc/coq-core.tactics/Autorewrite/index.html
Module Autorewrite
Source
This files implements the autorewrite tactic.
Source
type raw_rew_rule =
(Constr.constr Univ.in_universe_context_set
* bool
* Genarg.raw_generic_argument option)
CAst.t
Rewriting rules before tactic interpretation
To add rewriting rules to a base
Source
val autorewrite :
?conds:Equality.conditions ->
unit Proofview.tactic ->
string list ->
unit Proofview.tactic
The AutoRewrite tactic. The optional conditions tell rewrite how to handle matching and side-condition solving. Default is Naive: first match in the clause, don't look at the side-conditions to tell if the rewrite succeeded.
Source
val autorewrite_in :
?conds:Equality.conditions ->
Names.Id.t ->
unit Proofview.tactic ->
string list ->
unit Proofview.tactic
Source
type rew_rule = {
rew_lemma : Constr.constr;
rew_type : Constr.types;
rew_pat : Constr.constr;
rew_ctx : Univ.ContextSet.t;
rew_l2r : bool;
rew_tac : Genarg.glob_generic_argument option;
}
Rewriting rules
Source
val auto_multi_rewrite :
?conds:Equality.conditions ->
string list ->
Locus.clause ->
unit Proofview.tactic
Source
val auto_multi_rewrite_with :
?conds:Equality.conditions ->
unit Proofview.tactic ->
string list ->
Locus.clause ->
unit Proofview.tactic
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>