aboutsummaryrefslogtreecommitdiff
path: root/doc/sphinx/proof-engine
diff options
context:
space:
mode:
authorHugo Herbelin2020-04-19 13:00:09 +0200
committerHugo Herbelin2020-05-01 23:17:27 +0200
commitdf8df4637dfb4106854554cc2ac94b4fdd565e80 (patch)
tree8bedbb603f032642d8bf1c553121ae091077f692 /doc/sphinx/proof-engine
parenta6b2029042ae2e5f51fcae6d922fc8437ae1ff13 (diff)
Fixing #11903: Fixpoints not truly recursive in standard library.
There was also a non truly recursive in the doc.
Diffstat (limited to 'doc/sphinx/proof-engine')
-rw-r--r--doc/sphinx/proof-engine/ssreflect-proof-language.rst2
1 files changed, 1 insertions, 1 deletions
diff --git a/doc/sphinx/proof-engine/ssreflect-proof-language.rst b/doc/sphinx/proof-engine/ssreflect-proof-language.rst
index 28c5359a04..4be18ccda9 100644
--- a/doc/sphinx/proof-engine/ssreflect-proof-language.rst
+++ b/doc/sphinx/proof-engine/ssreflect-proof-language.rst
@@ -286,7 +286,7 @@ example, the null and all list function(al)s can be defined as follows:
.. coqtop:: all
Variable d: Set.
- Fixpoint null (s : list d) :=
+ Definition null (s : list d) :=
if s is nil then true else false.
Variable a : d -> bool.
Fixpoint all (s : list d) : bool :=