aboutsummaryrefslogtreecommitdiff
path: root/theories
diff options
context:
space:
mode:
authorPierre Roux2020-12-31 18:08:29 +0100
committerPierre Roux2021-01-18 12:09:11 +0100
commitf724ed1e270eb48060a510ff99219227c342ad6c (patch)
tree0552f45d72d5efa46ba19762ca4259899792af2c /theories
parent1b0f76026a553bcd76efb2bf99048235ad847ada (diff)
Fix #13579 (hnf on primitives raises an anomaly)
Also works for simpl.
Diffstat (limited to 'theories')
-rw-r--r--theories/Numbers/Cyclic/Int63/Int63.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Numbers/Cyclic/Int63/Int63.v b/theories/Numbers/Cyclic/Int63/Int63.v
index f324bbf52b..7bb725538b 100644
--- a/theories/Numbers/Cyclic/Int63/Int63.v
+++ b/theories/Numbers/Cyclic/Int63/Int63.v
@@ -954,6 +954,7 @@ Proof.
intros _ HH; generalize (HH H1); discriminate.
clear H.
generalize (ltb_spec j i); case Int63.ltb; intros H2; unfold bit; simpl.
+ change 62%int63 with (digits - 1)%int63.
assert (F2: (φ j < φ i)%Z) by (case H2; auto); clear H2.
replace (is_zero (((x << i) >> j) << (digits - 1))) with true; auto.
case (to_Z_bounded j); intros H1j H2j.