diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2016-04-25 14:31:11 +0200 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2016-04-27 21:55:45 +0200 |
commit | 5d9cb7ad4b3e4ccc77f77456bbb9969c418fcce2 (patch) | |
tree | 2f941e85d5cef3eba857291ed5ccf47d1385ed28 /test-suite | |
parent | 0fc6d2dcdb7d12e37d43cbf44fecaf2c0fddadcc (diff) |
Fixing a "This clause is redundant" error when interpreting the "in"
clause of a "match" over an irrefutable pattern.
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/success/CaseInClause.v | 4 |
1 files changed, 4 insertions, 0 deletions
diff --git a/test-suite/success/CaseInClause.v b/test-suite/success/CaseInClause.v index 3679eead7..599b9566c 100644 --- a/test-suite/success/CaseInClause.v +++ b/test-suite/success/CaseInClause.v @@ -20,3 +20,7 @@ Theorem foo : forall (n m : nat) (pf : n = m), match pf in _ = N with | eq_refl => unit end. + +(* Check redundant clause is removed *) +Inductive I : nat * nat -> Type := C : I (0,0). +Check fun x : I (1,1) => match x in I (y,z) return y = z with C => eq_refl end. |