aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/fast_integer.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/ZArith/fast_integer.v')
-rw-r--r--theories/ZArith/fast_integer.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/fast_integer.v b/theories/ZArith/fast_integer.v
index f64093034..678e8b472 100644
--- a/theories/ZArith/fast_integer.v
+++ b/theories/ZArith/fast_integer.v
@@ -1147,7 +1147,7 @@ Save.
Theorem Zmult_Zopp_Zopp:
(x,y:Z) (Zmult (Zopp x) (Zopp y)) = (Zmult x y).
Proof.
-Destruct x; Destruct y; Reflexivity.
+NewDestruct x; NewDestruct y; Reflexivity.
Save.
Theorem weak_Zmult_plus_distr_r: