aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-11 15:14:10 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-11 15:14:10 +0000
commita252a5d44a7793ae8ed9accf582a27dcdbd1721d (patch)
tree798c013cd6661fa4102ee78bc066d48575ff7b75 /test-suite
parent279896398b21a92291295bf04854eeed2d704079 (diff)
Correction d'un bug de clear
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10552 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/success/clear.v13
1 files changed, 11 insertions, 2 deletions
diff --git a/test-suite/success/clear.v b/test-suite/success/clear.v
index 444146f7f..8169361c4 100644
--- a/test-suite/success/clear.v
+++ b/test-suite/success/clear.v
@@ -1,6 +1,15 @@
Goal forall x:nat, (forall x, x=0 -> True)->True.
intros; eapply H.
instantiate (1:=(fun y => _) (S x)).
- simpl.
- clear x || trivial.
+ simpl.
+ clear x. trivial.
Qed.
+
+Goal forall y z, (forall x:nat, x=y -> True) -> y=z -> True.
+ intros; eapply H.
+ rename z into z'.
+ clear H0.
+ clear z'.
+ reflexivity.
+Qed.
+