aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/complexity
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-09 15:47:52 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-09 15:47:52 +0000
commit66d792dd1ffc706394fd31627e9da4a1e424f2ee (patch)
tree75261574608673754181f0af183aeea6be4901dd /test-suite/complexity
parent33c70d36141ef619825ca8746b6d4ae170db7c41 (diff)
test-suite/complexity/ring2.v: Zeqb_ok -> Zbool.Zeq_bool_eq
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11216 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/complexity')
-rw-r--r--test-suite/complexity/ring2.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/complexity/ring2.v b/test-suite/complexity/ring2.v
index 9f9685dde..e1a799f07 100644
--- a/test-suite/complexity/ring2.v
+++ b/test-suite/complexity/ring2.v
@@ -1,7 +1,7 @@
(* This example, checks the efficiency of the abstract machine used by ring *)
(* Expected time < 1.00s *)
-Require Import BinInt.
+Require Import BinInt Zbool.
Definition Zplus x y :=
match x with
@@ -42,7 +42,7 @@ Ltac Zcst t :=
end.
Add Ring Zr : Zth
- (decidable Zeqb_ok, constants [Zcst]).
+ (decidable Zeq_bool_eq, constants [Zcst]).
Open Scope Z_scope.
Infix "+" := Zplus : Z_scope.