aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorEnrico Tassi2021-02-09 16:20:08 +0100
committerEnrico Tassi2021-03-04 16:55:14 +0100
commit8ae0762db0616e1ff177335c9fc73c816634fc89 (patch)
tree3a6c2b0aead19858a41fecabf084544567dcfaba /test-suite
parenta5bea627d1fe742229497b466ca24b470c20d269 (diff)
[notation] option to fine tune printing of literals
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/output/primitive_tokens.out29
-rw-r--r--test-suite/output/primitive_tokens.v15
2 files changed, 44 insertions, 0 deletions
diff --git a/test-suite/output/primitive_tokens.out b/test-suite/output/primitive_tokens.out
new file mode 100644
index 0000000000..cbed08c0ca
--- /dev/null
+++ b/test-suite/output/primitive_tokens.out
@@ -0,0 +1,29 @@
+"foo"
+ : string
+1234
+ : nat
+String (Ascii.Ascii false true true false false true true false)
+ (String (Ascii.Ascii true true true true false true true false)
+ (String (Ascii.Ascii true true true true false true true false)
+ EmptyString))
+ : string
+S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S
+ (S (S (S (S (S (S ...)))))))))))))))))))))))
+ : nat
diff --git a/test-suite/output/primitive_tokens.v b/test-suite/output/primitive_tokens.v
new file mode 100644
index 0000000000..fe31107744
--- /dev/null
+++ b/test-suite/output/primitive_tokens.v
@@ -0,0 +1,15 @@
+Require Import String.
+
+Open Scope string_scope.
+
+Unset Printing Notations.
+
+Check "foo".
+Check 1234.
+Check 1 + 2.
+
+Unset Printing Primitive Tokens.
+
+Check "foo".
+Check 1234.
+Check 1 + 2.