aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/ZSyntax.v8
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/output/ZSyntax.v8')
-rw-r--r--test-suite/output/ZSyntax.v817
1 files changed, 0 insertions, 17 deletions
diff --git a/test-suite/output/ZSyntax.v8 b/test-suite/output/ZSyntax.v8
deleted file mode 100644
index 0412f6d68..000000000
--- a/test-suite/output/ZSyntax.v8
+++ /dev/null
@@ -1,17 +0,0 @@
-Require Import ZArith.
-Check 32%Z.
-Check (fun f : nat -> Z => (f 0%nat + 0)%Z).
-Check (fun x : positive => Zpos (xO x)).
-Check (fun x : positive => (Zpos x + 1)%Z).
-Check (fun x : positive => Zpos x).
-Check (fun x : positive => Zneg (xO x)).
-Check (fun x : positive => (Zpos (xO x) + 0)%Z).
-Check (fun x : positive => (- Zpos (xO x))%Z).
-Check (fun x : positive => (- Zpos (xO x) + 0)%Z).
-Check (Z_of_nat 0 + 1)%Z.
-Check (0 + Z_of_nat (0 + 0))%Z.
-Check (Z_of_nat 0 = 0%Z).
-
-(* Submitted by Pierre Casteran *)
-Require Import Arith.
-Check (0 + Z_of_nat 11)%Z. \ No newline at end of file