diff options
author | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2004-03-24 18:27:49 +0000 |
---|---|---|
committer | barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2004-03-24 18:27:49 +0000 |
commit | 070d631038dbf7ccbc8e0907c542588548ebe566 (patch) | |
tree | 19ec54e994ce9b3185eb2902b9185203f4074210 /test-suite/success | |
parent | 51a914f29174fe3cb455b668e83e98e08f88edc1 (diff) |
*** empty log message ***
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5555 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/Abstract.v8 | 26 |
1 files changed, 26 insertions, 0 deletions
diff --git a/test-suite/success/Abstract.v8 b/test-suite/success/Abstract.v8 new file mode 100644 index 000000000..21a985bcd --- /dev/null +++ b/test-suite/success/Abstract.v8 @@ -0,0 +1,26 @@ + +(* 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. |