aboutsummaryrefslogtreecommitdiff
path: root/test-suite/vio
diff options
context:
space:
mode:
authorPierre-Marie Pédrot2019-05-29 16:35:51 +0200
committerPierre-Marie Pédrot2019-05-31 13:46:11 +0200
commit30ed0b3385d80e2abe3d2d8c67ce09643a8bf74c (patch)
tree4fd6729fb0fc53c489a81b18efcb3a8981ff6322 /test-suite/vio
parent7032085c809993d6a173e51aec447c02828ae070 (diff)
Fix #10268: vio2vo produces incorrect term when discharging.
We do not partially abstract the section info. Instead, we reuse the same code in cook_constr and cook_constant and pass the same section info.
Diffstat (limited to 'test-suite/vio')
-rw-r--r--test-suite/vio/section.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/test-suite/vio/section.v b/test-suite/vio/section.v
new file mode 100644
index 0000000000..0e7722516a
--- /dev/null
+++ b/test-suite/vio/section.v
@@ -0,0 +1,12 @@
+Section Foo.
+ Variable A : Type.
+
+ Definition bla := A.
+
+ Variable B : bla.
+
+ Lemma blu : {X:Type & X}.
+ Proof using A B.
+ exists bla;exact B.
+ Qed.
+End Foo.