aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/interactive
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-01-13 18:38:41 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2014-01-13 18:49:35 +0100
commite6b3b63eab1ca2a9586ef2c49a8df6c2e2a29adf (patch)
tree2f950ca259372a8baddf73565dec3764b42fde8c /test-suite/interactive
parent23e44c7a421d47c71318d12b1a7c5d27fb5f393a (diff)
rename Paral-ITP demo file
Diffstat (limited to 'test-suite/interactive')
-rw-r--r--test-suite/interactive/ParalITP.v (renamed from test-suite/interactive/Paral-ITP.v)14
1 files changed, 10 insertions, 4 deletions
diff --git a/test-suite/interactive/Paral-ITP.v b/test-suite/interactive/ParalITP.v
index 69d3b8b88..a96d4a5c7 100644
--- a/test-suite/interactive/Paral-ITP.v
+++ b/test-suite/interactive/ParalITP.v
@@ -14,17 +14,21 @@ Let time := 18.
(* Beginning of demo *)
+Section Demo.
+
+Variable i : True.
+
Lemma a : True.
-Proof.
+Proof using i.
sleep time.
idtac.
sleep time.
(* Error, jump back to fix it, then Qed again *)
- exact (I I).
+ exact (i i).
Qed.
Lemma b : True.
-Proof.
+Proof using i.
sleep time.
idtac.
sleep time.
@@ -33,9 +37,11 @@ Proof.
Qed.
Lemma work_here : True /\ True.
-Proof.
+Proof using i.
(* Jump directly here, Coq reacts immediately *)
split.
exact b. (* We can use the lemmas above *)
exact a.
+Qed.
+End Demo. \ No newline at end of file