aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorThéo Zimmermann2019-05-07 14:18:51 +0200
committerThéo Zimmermann2019-05-07 14:18:51 +0200
commit403f8784706d54e5e91bf20e56b0bf8ea40f4df3 (patch)
treeb265ee33a8ec49cc86d9d28686c72a9722bae787
parentc828bca2c11d83a329facd56051abd4d27e16850 (diff)
parent590ee35546f3528ac7ccb32306fb86e78fdce93b (diff)
Merge PR #10053: Document change_no_check variants
Ack-by: JasonGross Reviewed-by: Zimmi48
-rw-r--r--doc/sphinx/proof-engine/tactics.rst20
1 files changed, 20 insertions, 0 deletions
diff --git a/doc/sphinx/proof-engine/tactics.rst b/doc/sphinx/proof-engine/tactics.rst
index 1f339e7761..658ac857fb 100644
--- a/doc/sphinx/proof-engine/tactics.rst
+++ b/doc/sphinx/proof-engine/tactics.rst
@@ -4841,6 +4841,26 @@ Performance-oriented tactic variants
exact I.
Fail Qed.
+ :tacn:`change_no_check` supports all of `change`'s variants.
+
+ .. tacv:: change_no_check @term with @term’
+ :undocumented:
+
+ .. tacv:: change_no_check @term at {+ @num} with @term’
+ :undocumented:
+
+ .. tacv:: change_no_check @term {? {? at {+ @num}} with @term} in @ident
+
+ .. example::
+
+ .. coqtop:: all abort
+
+ Goal True -> False.
+ intro H.
+ change_no_check False in H.
+ exact H.
+ Fail Qed.
+
.. tacv:: convert_concl_no_check @term
:name: convert_concl_no_check