summaryrefslogtreecommitdiff
path: root/test-suite/success/destruct.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/destruct.v')
-rw-r--r--test-suite/success/destruct.v32
1 files changed, 32 insertions, 0 deletions
diff --git a/test-suite/success/destruct.v b/test-suite/success/destruct.v
index 9f938e10..5aa78816 100644
--- a/test-suite/success/destruct.v
+++ b/test-suite/success/destruct.v
@@ -23,3 +23,35 @@ set (b := true) in *.
try destruct b.
Abort.
+(* Used to fail with error "n is used in conclusion" before revision 9447 *)
+
+Goal forall n, n = S n.
+induction S.
+Abort.
+
+(* Check that elimination with remaining evars do not raise an bad
+ error message *)
+
+Theorem Refl : forall P, P <-> P. tauto. Qed.
+Goal True.
+case Refl || ecase Refl.
+Abort.
+
+
+(* Submitted by B. Baydemir (bug #1882) *)
+
+Require Import List.
+
+Definition alist R := list (nat * R)%type.
+
+Section Properties.
+ Variables A : Type.
+ Variables a : A.
+ Variables E : alist A.
+
+ Lemma silly : E = E.
+ Proof.
+ clear. induction E. (* this fails. *)
+ Abort.
+
+End Properties.