aboutsummaryrefslogtreecommitdiff
path: root/plugins/syntax
diff options
context:
space:
mode:
authorPierre Roux2020-01-28 12:43:51 +0100
committerPierre Roux2020-01-28 22:19:27 +0100
commit85b3be5f6998287d90acf89de96129571b244cd7 (patch)
tree97d8f65bb143e2d69d449857fe2cc1ed5422f8e6 /plugins/syntax
parent614643e6fb1b5029d1c2bf50cd51f95d621010cf (diff)
Fix #11467
'e' was not displayed when printing decimal notations in R : Require Import Reals. Check (1.23e1, 32e+1, 0.1)%R. was giving < (123-1%R, 321%R, 1-1%R) instead of < (123e-1%R, 32e1%R, 1e-1%R) This was introduced in #8764 (in Coq 8.10).
Diffstat (limited to 'plugins/syntax')
-rw-r--r--plugins/syntax/r_syntax.ml2
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/syntax/r_syntax.ml b/plugins/syntax/r_syntax.ml
index 70c1077106..f6fbdaa958 100644
--- a/plugins/syntax/r_syntax.ml
+++ b/plugins/syntax/r_syntax.ml
@@ -164,7 +164,7 @@ let rawnum_of_r c = match DAst.get c with
let s, i = if is_pos_or_zero i then SPlus, i else SMinus, neg i in
let i = Bigint.to_string i in
let se = if is_gr md glob_Rdiv then "-" else "" in
- let e = se ^ Bigint.to_string e in
+ let e = "e" ^ se ^ Bigint.to_string e in
s, { NumTok.int = i; frac = ""; exp = e }
| _ -> raise Non_closed_number
end