Skip to content

Commit a283ca5

Browse files
committed
Review #2
1 parent 7257bf2 commit a283ca5

File tree

2 files changed

+4
-4
lines changed

2 files changed

+4
-4
lines changed

doc/sphinx/language/core/basic.rst

+2-2
Original file line numberDiff line numberDiff line change
@@ -160,15 +160,15 @@ Numbers
160160

161161
.. coqtop:: all reset
162162

163-
Fail Compute 100000 + 100000. (* gives a stack overflow (not shown) *)
163+
Fail Eval compute in 100000 + 100000. (* gives a stack overflow (not shown) *)
164164
165165
.. coqtop:: in
166166

167167
Require Import ZArith. (* for definition of Z *)
168168
169169
.. coqtop:: all
170170

171-
Compute (1000000000000000000000000000000000 + 1)%Z.
171+
Eval compute in (1000000000000000000000000000000000 + 1)%Z.
172172

173173
Strings
174174
Strings begin and end with ``"`` (double quote). Use ``""`` to represent

doc/sphinx/user-extensions/syntax-extensions.rst

+2-2
Original file line numberDiff line numberDiff line change
@@ -2041,8 +2041,8 @@ Number notations
20412041

20422042
:n:`abstract after @bignat`
20432043
returns :n:`(@qualid__parse m)` when parsing a literal
2044-
:n:`m` that's greater than :n:`@bignat` rather than reducing it to a normal form.
2045-
Here :g:`m` will be a
2044+
:n:`m` that's greater than or equal to :n:`@bignat` rather than reducing
2045+
it to a normal form. Here :g:`m` will be a
20462046
:g:`Number.int`, :g:`Number.uint`, :g:`Z` or :g:`Number.number`, depending on the
20472047
type of the parsing function :n:`@qualid__parse`. This allows for a
20482048
more compact representation of literals in types such as :g:`nat`,

0 commit comments

Comments
 (0)