aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-12-18 16:35:46 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-12-18 17:08:07 +0100
commitb49d803286ba9ed711313702bb4269c5e9c516fa (patch)
tree1f0c6407edb61f112c0872377ba2cef34386d554 /test-suite/success
parentfc3b70a11aff48eedd7b235f5732cd170a6ab8be (diff)
Proof using: New vernacular to name sets of section variables
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/proof_using.v31
1 files changed, 31 insertions, 0 deletions
diff --git a/test-suite/success/proof_using.v b/test-suite/success/proof_using.v
index bf302df44..d2691e763 100644
--- a/test-suite/success/proof_using.v
+++ b/test-suite/success/proof_using.v
@@ -65,3 +65,34 @@ End S1.
Check (deep 3 4 : 3 = 4).
Check (deep2 3 4 : 3 = 4).
+
+Section P1.
+
+Variable x : nat.
+Variable y : nat.
+Variable z : nat.
+
+
+Package TOTO := x y.
+
+Package TITI := TOTO - x.
+
+Lemma t1 : True. Proof using TOTO. trivial. Qed.
+Lemma t2 : True. Proof using TITI. trivial. Qed.
+
+ Section P2.
+ Package TOTO := x.
+ Lemma t3 : True. Proof using TOTO. trivial. Qed.
+ End P2.
+
+Lemma t4 : True. Proof using TOTO. trivial. Qed.
+
+End P1.
+
+Lemma t5 : True. Fail Proof using TOTO. trivial. Qed.
+
+Check (t1 1 2 : True).
+Check (t2 1 : True).
+Check (t3 1 : True).
+Check (t4 1 2 : True).
+