aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3284.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-06-13 11:45:51 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-06-13 12:08:34 +0200
commit8cb6251702b09186ca41c5ce67464b83ccfb3d16 (patch)
treef767419e2ce8cad27fa7fe55d4427c782dff6538 /test-suite/bugs/closed/3284.v
parent176f40f976741c8fb6e020c0eaeac4df59a474bc (diff)
Fixing "clear" in internal_cut_replace: forbid dependencies in the
name of replaced hypothesis.
Diffstat (limited to 'test-suite/bugs/closed/3284.v')
-rw-r--r--test-suite/bugs/closed/3284.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3284.v b/test-suite/bugs/closed/3284.v
index a942887ee..34cd09c6f 100644
--- a/test-suite/bugs/closed/3284.v
+++ b/test-suite/bugs/closed/3284.v
@@ -13,5 +13,11 @@ Proof.
intros A B C f g x H.
Fail apply @functional_extensionality_dep in H.
Fail apply functional_extensionality_dep in H.
+ eapply functional_extensionality_dep in H.
+Abort.
+
+Goal forall A B C (f g : forall (x : A) (y : B x), C x y), forall x:A, (forall x y, f x y = g x y) -> True.
+Proof.
+ intros A B C f g x H.
specialize (H x).
apply functional_extensionality_dep in H.