aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/refine.v
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-08 12:39:34 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-11-08 12:39:34 +0100
commit7e42041f5c4711a9fece32ce601ef99ca8ab272f (patch)
treef2330be6cbe2a8d0be1a7de17875c7ed62770e1f /test-suite/success/refine.v
parent0d81e80a09db7d352408be4dfc5ba263f6ed98ef (diff)
parentdd56ef10395a2ced84612aa799690b034306806e (diff)
Merge PR #922: New beta-iota compatibility refinements
Diffstat (limited to 'test-suite/success/refine.v')
-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 b8a8ff756..22fb4d757 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.