diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2017-09-21 10:18:41 +0200 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2017-09-23 15:32:07 +0200 |
commit | a3150ecab4c4032ea2c8de96e540ccbae277e233 (patch) | |
tree | 87cefd41aedde5b73d0350013e4960aaecd2525f /test-suite | |
parent | 7e4535d62c4f8abc6537206e7abc34f1bb0be69d (diff) |
Fixing #5749 (bug in fold_constr_with_binders introduced in 4e70791).
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/5749.v | 18 |
1 files changed, 18 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5749.v b/test-suite/bugs/closed/5749.v new file mode 100644 index 000000000..81bfe351c --- /dev/null +++ b/test-suite/bugs/closed/5749.v @@ -0,0 +1,18 @@ +(* Checking computation of free vars of a term for generalization *) + +Definition Decision := fun P : Prop => {P} + {~ P}. +Class SetUnfold (P Q : Prop) : Prop := Build_SetUnfold { set_unfold : P <-> Q +}. + +Section Filter_Help. + + Context {A: Type}. + Context (fold_right : forall A B : Type, (B -> A -> A) -> A -> list B -> A). + Definition lType2 := (sigT (fun (P : A -> Prop) => forall a, Decision (P +a))). + Definition test (X: lType2) := let (x, _) := X in x. + + Global Instance foo `{fhl1 : list lType2} m Q: + SetUnfold (Q) + (fold_right _ _ (fun (s : lType2) => let (P, _) := s in and (P +m)) (Q) (fhl1)). |