aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/complexity
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-12 18:25:06 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-12 18:25:06 +0000
commit15bbdcfa63dd7fee30b3d03f98cf0795e4baf087 (patch)
treed547b755963a3f6c59fb2da66d30ab81ae4fa4de /test-suite/complexity
parent651a23b4b21045733d44a4bc944b6b56d449fe2e (diff)
MAJ et bricoles diverses
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10923 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/complexity')
-rw-r--r--test-suite/complexity/ring.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/complexity/ring.v b/test-suite/complexity/ring.v
new file mode 100644
index 000000000..5a541bc24
--- /dev/null
+++ b/test-suite/complexity/ring.v
@@ -0,0 +1,7 @@
+(* This example, checks the efficiency of the abstract machine used by ring *)
+(* Expected time < 1.00s *)
+
+Require Import ZArith.
+Open Scope Z_scope.
+Goal forall a, a+a+a+a+a+a+a+a+a+a+a+a+a = a*13.
+Time intro; ring.