summaryrefslogtreecommitdiff
path: root/test-suite/complexity/ring.v
blob: 5a541bc24a832fe9674e72e34f5d66cff2fbd96e (plain)
1
2
3
4
5
6
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.