diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2017-11-30 15:54:12 +0100 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2017-11-30 15:54:12 +0100 |
commit | 0bb126dae41b410fdf4f6531024c64cac20dac06 (patch) | |
tree | cc3a9c0d8133eae3902b3a441246d50c48f02436 /test-suite/bugs | |
parent | ee45637ac2431fe2df1994f2337d8801e2aeff9a (diff) | |
parent | 08da05299d32886bb516124fa497347b40249006 (diff) |
Merge PR #6274: Attempt to fix inversion disregarding singleton types (fixes #3125)
Diffstat (limited to 'test-suite/bugs')
-rw-r--r-- | test-suite/bugs/closed/3125.v | 27 |
1 files changed, 27 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3125.v b/test-suite/bugs/closed/3125.v new file mode 100644 index 000000000..797146174 --- /dev/null +++ b/test-suite/bugs/closed/3125.v @@ -0,0 +1,27 @@ +(* Not considering singleton template-polymorphic inductive types as + propositions for injection/inversion *) + +(* This is also #4560 and #6273 *) + +Inductive foo := foo_1. + +Goal forall (a b : foo), Some a = Some b -> a = b. +Proof. + intros a b H. + inversion H. + reflexivity. +Qed. + +(* Check that Prop is not concerned *) + +Inductive bar : Prop := bar_1. + +Goal + forall (a b : bar), + Some a = Some b -> + a = b. +Proof. + intros a b H. + inversion H. + Fail reflexivity. +Abort. |