diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2017-04-19 09:18:31 +0200 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2017-04-19 09:18:31 +0200 |
commit | 59b0041147a9d2dddc1fe14f624a2cf5695f2ea2 (patch) | |
tree | d4967d23e54ea5162b0dfb8670857bba3f9360c2 /test-suite | |
parent | 727ef1bd345f9ad9e08d9e4f136e2db7d034a93d (diff) | |
parent | 031d0fbcea7c1390dc7e6cf89cfaee8609ecfed1 (diff) |
Merge PR#538: Correction of bug #4306
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/4306.v | 32 |
1 files changed, 32 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4306.v b/test-suite/bugs/closed/4306.v new file mode 100644 index 000000000..4aef5bb95 --- /dev/null +++ b/test-suite/bugs/closed/4306.v @@ -0,0 +1,32 @@ +Require Import List. +Require Import Arith. +Require Import Recdef. +Require Import Omega. + +Function foo (xys : (list nat * list nat)) {measure (fun xys => length (fst xys) + length (snd xys))} : list nat := + match xys with + | (nil, _) => snd xys + | (_, nil) => fst xys + | (x :: xs', y :: ys') => match Compare_dec.nat_compare x y with + | Lt => x :: foo (xs', y :: ys') + | Eq => x :: foo (xs', ys') + | Gt => y :: foo (x :: xs', ys') + end + end. +Proof. + intros; simpl; omega. + intros; simpl; omega. + intros; simpl; omega. +Qed. + +Function bar (xys : (list nat * list nat)) {measure (fun xys => length (fst xys) + length (snd xys))} : list nat := + let (xs, ys) := xys in + match (xs, ys) with + | (nil, _) => ys + | (_, nil) => xs + | (x :: xs', y :: ys') => match Compare_dec.nat_compare x y with + | Lt => x :: foo (xs', ys) + | Eq => x :: foo (xs', ys') + | Gt => y :: foo (xs, ys') + end + end.
\ No newline at end of file |