aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_10031.v
blob: b76ea7d3372ca0dbbe991af48db74c103ee454fc (plain)
1
2
3
4
5
6
7
8
9
Require Import Int63 ZArith.

Open Scope int63_scope.

Goal False.
cut (let (q, r) := (0, 0) in (φ q, φ r) = (9223372036854775808%Z, 0%Z));
  [discriminate| ].
Fail (change (0, 0) with (diveucl_21 1 0 1); apply diveucl_21_spec).
Abort.