aboutsummaryrefslogtreecommitdiff
path: root/doc
diff options
context:
space:
mode:
Diffstat (limited to 'doc')
-rw-r--r--doc/changelog/05-tactic-language/13236-ltac2-printf.rst7
-rw-r--r--doc/stdlib/index-list.html.template1
2 files changed, 8 insertions, 0 deletions
diff --git a/doc/changelog/05-tactic-language/13236-ltac2-printf.rst b/doc/changelog/05-tactic-language/13236-ltac2-printf.rst
new file mode 100644
index 0000000000..02213f22e5
--- /dev/null
+++ b/doc/changelog/05-tactic-language/13236-ltac2-printf.rst
@@ -0,0 +1,7 @@
+- **Added:**
+ Added a ``printf`` macro to Ltac2. It can be made accessible by
+ importing the ``Ltac2.Printf`` module. See the documentation
+ there for more information
+ (`#13236 <https://github.com/coq/coq/pull/13236>`_,
+ fixes `#10108 <https://github.com/coq/coq/issues/10108>`_,
+ by Pierre-Marie Pédrot).
diff --git a/doc/stdlib/index-list.html.template b/doc/stdlib/index-list.html.template
index 27eb64a83b..b0f4e883be 100644
--- a/doc/stdlib/index-list.html.template
+++ b/doc/stdlib/index-list.html.template
@@ -692,6 +692,7 @@ through the <tt>Require Import</tt> command.</p>
user-contrib/Ltac2/Notations.v
user-contrib/Ltac2/Option.v
user-contrib/Ltac2/Pattern.v
+ user-contrib/Ltac2/Printf.v
user-contrib/Ltac2/Std.v
user-contrib/Ltac2/String.v
</dd>