aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/evars.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-26 22:34:57 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2017-05-28 18:41:12 +0200
commit1a169b01458829f9420aea9c855b1ef28e5c847d (patch)
treeb9bf1316921444c8210e6a20c66689569772a74e /test-suite/success/evars.v
parent1c74df16e7a539f21418ddb09419ff0106960789 (diff)
Fixing a subtle bug in tclWITHHOLES.
This fixes Théo's bug on eset.
Diffstat (limited to 'test-suite/success/evars.v')
-rw-r--r--test-suite/success/evars.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/success/evars.v b/test-suite/success/evars.v
index 4e2bf4511..4b2f7b53e 100644
--- a/test-suite/success/evars.v
+++ b/test-suite/success/evars.v
@@ -414,4 +414,10 @@ Axiom test : forall P1 P2, P1 = P2 -> P1 -> P2.
Import EqNotations.
Definition test2 {A B:Type} {H:A=B} (a:A) : B := rew H in a.
+(* Check that pre-existing evars are not counted as newly undefined in "set" *)
+(* Reported by Théo *)
+Goal exists n : nat, n = n -> True.
+eexists.
+set (H := _ = _).
+Abort.