aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-07-26 22:34:43 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-08-21 13:14:43 +0200
commitdd56ef10395a2ced84612aa799690b034306806e (patch)
treee6fe2bc49b5154c5f6ee8f951a900905f4260af0 /test-suite/success
parent9490c6099e1da94fcf315aba48125993cd180327 (diff)
Fixing another regression with 8.4 wrt to βι-normalization of created hyps.
This one is a continuation of e2a8edaf59 which was βι-normalizing the hypotheses created by a "match". We forgot to do it for "let" and "if". This is what this commit is doing.
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/refine.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/success/refine.v b/test-suite/success/refine.v
index 352abb2af..4f6505f58 100644
--- a/test-suite/success/refine.v
+++ b/test-suite/success/refine.v
@@ -122,3 +122,13 @@ Abort.
Goal (forall A : Prop, A -> ~~A).
Proof. refine(fun A a f => _).
+
+(* Checking beta-iota normalization of hypotheses in created evars *)
+
+Goal {x|x=0} -> True.
+refine (fun y => let (x,a) := y in _).
+match goal with a:_=0 |- _ => idtac end.
+
+Goal (forall P, {P 0}+{P 1}) -> True.
+refine (fun H => if H (fun x => x=x) then _ else _).
+match goal with _:0=0 |- _ => idtac end.