aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/ZArith/fast_integer.v9
1 files changed, 7 insertions, 2 deletions
diff --git a/theories/ZArith/fast_integer.v b/theories/ZArith/fast_integer.v
index 210e0846b..fe16e8dff 100644
--- a/theories/ZArith/fast_integer.v
+++ b/theories/ZArith/fast_integer.v
@@ -1481,5 +1481,10 @@ Intros x y;Case x;Case y; [
Qed.
End fast_integers.
-Syntactic Definition times1 := times.
-Syntactic Definition times1_convert := times_convert.
+V7only [
+ Comments "Compatibility with the old version of times and times_convert".
+ Syntactic Definition times1 :=
+ [x:positive;_:positive->positive;y:positive](times x y).
+ Syntactic Definition times1_convert :=
+ [x,y:positive;_:positive->positive](times_convert x y).
+].