summaryrefslogtreecommitdiff
path: root/test-suite/success/Abstract.v8
diff options
context:
space:
mode:
authorGravatar Samuel Mimram <smimram@debian.org>2006-04-28 14:59:16 +0000
committerGravatar Samuel Mimram <smimram@debian.org>2006-04-28 14:59:16 +0000
commit3ef7797ef6fc605dfafb32523261fe1b023aeecb (patch)
treead89c6bb57ceee608fcba2bb3435b74e0f57919e /test-suite/success/Abstract.v8
parent018ee3b0c2be79eb81b1f65c3f3fa142d24129c8 (diff)
Imported Upstream version 8.0pl3+8.1alphaupstream/8.0pl3+8.1alpha
Diffstat (limited to 'test-suite/success/Abstract.v8')
-rw-r--r--test-suite/success/Abstract.v826
1 files changed, 0 insertions, 26 deletions
diff --git a/test-suite/success/Abstract.v8 b/test-suite/success/Abstract.v8
deleted file mode 100644
index 21a985bc..00000000
--- a/test-suite/success/Abstract.v8
+++ /dev/null
@@ -1,26 +0,0 @@
-
-(* 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.