diff options
author | Maxime Dénès <mail@maximedenes.fr> | 2017-04-28 11:25:29 +0200 |
---|---|---|
committer | Maxime Dénès <mail@maximedenes.fr> | 2017-04-28 11:25:29 +0200 |
commit | 66a68a4329ce199f25184ba8b2d98b4679e7ddae (patch) | |
tree | ce90c93341c58e82813da8b1a567ce6a3f3ed424 /test-suite/success | |
parent | 0a255f51809e8d29a7239bfbd9fe57a8b2b41705 (diff) | |
parent | 2ddc9d12bd4616f10245c40bc0c87ae548911809 (diff) |
Merge PR#531: Fixing bug #5420 and many similar bugs due to the presence of let-ins
Diffstat (limited to 'test-suite/success')
-rw-r--r-- | test-suite/success/ImplicitArguments.v | 6 |
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/success/ImplicitArguments.v b/test-suite/success/ImplicitArguments.v index f702aa62f..f07773f8b 100644 --- a/test-suite/success/ImplicitArguments.v +++ b/test-suite/success/ImplicitArguments.v @@ -21,3 +21,9 @@ Fixpoint app {A : Type} {n m : nat} (v : vector A n) (w : vector A m) : vector A (* Test sharing information between different hypotheses *) Parameters (a:_) (b:a=0). + +(* These examples were failing due to a lifting wrongly taking let-in into account *) + +Definition foo6 (x:=1) : forall {n:nat}, n=n := fun n => eq_refl. + +Fixpoint foo7 (x:=1) (n:nat) {p:nat} {struct n} : nat. |