summaryrefslogtreecommitdiff
path: root/test-suite/success/Abstract.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/Abstract.v')
-rw-r--r--test-suite/success/Abstract.v27
1 files changed, 27 insertions, 0 deletions
diff --git a/test-suite/success/Abstract.v b/test-suite/success/Abstract.v
new file mode 100644
index 00000000..fc8800a5
--- /dev/null
+++ b/test-suite/success/Abstract.v
@@ -0,0 +1,27 @@
+
+(* Cf coqbugs #546 *)
+
+Require Import Omega.
+
+Section S.
+
+Variables n m : nat.
+Variable H : n<m.
+
+Inductive Dummy : nat -> Set :=
+| Dummy0 : Dummy 0
+| Dummy2 : Dummy 2
+| DummyApp : forall i j, Dummy i -> Dummy j -> Dummy (i+j).
+
+Definition Bug : Dummy (2*n).
+Proof.
+induction n.
+ simpl ; apply Dummy0.
+ replace (2 * S n0) with (2*n0 + 2) ; auto with arith.
+ apply DummyApp.
+ 2:exact Dummy2.
+ apply IHn0 ; abstract omega.
+Defined.
+
+End S.
+