aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4372.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-10-19 17:23:48 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-10-19 17:26:57 +0200
commitb3b04d0a5c7c39140e2125321a17957ddcaf2b33 (patch)
tree0e95edfa3516eda6483de378bcf14c397e32b8a1 /test-suite/bugs/closed/4372.v
parentc3967bd7a71df53a004478d23b072309f13f2ff5 (diff)
Test for #4372 (anomaly in inversion in the presence of fake dependency).
Diffstat (limited to 'test-suite/bugs/closed/4372.v')
-rw-r--r--test-suite/bugs/closed/4372.v20
1 files changed, 20 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4372.v b/test-suite/bugs/closed/4372.v
new file mode 100644
index 000000000..428192a34
--- /dev/null
+++ b/test-suite/bugs/closed/4372.v
@@ -0,0 +1,20 @@
+(* Tactic inversion was raising an anomaly because of a fake
+ dependency of TypeDenote into its argument *)
+
+Inductive expr :=
+| ETrue.
+
+Inductive IntermediateType : Set := ITbool.
+
+Definition TypeDenote (IT : IntermediateType) : Type :=
+ match IT with
+ | _ => bool
+ end.
+
+Inductive ValueDenote : forall (e:expr) it, TypeDenote it -> Prop :=
+| VT : ValueDenote ETrue ITbool true.
+
+Goal forall it v, @ValueDenote ETrue it v -> True.
+ intros it v H.
+ inversion H.
+Abort.