diff options
| author | Pierre Roux | 2020-01-28 12:43:51 +0100 |
|---|---|---|
| committer | Pierre Roux | 2020-01-28 22:19:27 +0100 |
| commit | 85b3be5f6998287d90acf89de96129571b244cd7 (patch) | |
| tree | 97d8f65bb143e2d69d449857fe2cc1ed5422f8e6 /test-suite/output/QArithSyntax.v | |
| parent | 614643e6fb1b5029d1c2bf50cd51f95d621010cf (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 'test-suite/output/QArithSyntax.v')
| -rw-r--r-- | test-suite/output/QArithSyntax.v | 9 |
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/output/QArithSyntax.v b/test-suite/output/QArithSyntax.v new file mode 100644 index 0000000000..2f2ee0134a --- /dev/null +++ b/test-suite/output/QArithSyntax.v @@ -0,0 +1,9 @@ +Require Import QArith. +Open Scope Q_scope. +Check (eq_refl : 1.02 = 102 # 100). +Check (eq_refl : 1.02e1 = 102 # 10). +Check (eq_refl : 1.02e+03 = 1020). +Check (eq_refl : 1.02e+02 = 102 # 1). +Check (eq_refl : 10.2e-1 = 1.02). +Check (eq_refl : -0.0001 = -1 # 10000). +Check (eq_refl : -0.50 = - 50 # 100). |
