aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/interactive
diff options
context:
space:
mode:
authorGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-20 12:43:42 +0000
committerGravatar gareuselesinge <gareuselesinge@85f007b7-540e-0410-9357-904b9bb8a0f7>2013-08-20 12:43:42 +0000
commit16a2717d25096fcbd07b252e775b66b6fbb6d2bd (patch)
treeaa27bd74810dbda95b19097ea486842eb8f7e33a /test-suite/interactive
parentc5b699f8feb54b7ada2cb6c6754a1909ebedcd3f (diff)
Universe counters on slaves are in sync with master
Simple framework for remote counters. The slaves ask the master for a fresh value. On the master the thread manager answers with a bunch of fresh values (so that further requests can be immediately satisfied). Remote counters are guarded with a mutex on the master, because all slave managers as well as the master thread can access the counter at the same time. I know the name sucks. These counters are remote for the slaves, and local for the master. I'm open to suggestions... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16713 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/interactive')
-rw-r--r--test-suite/interactive/Paral-ITP.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/interactive/Paral-ITP.v b/test-suite/interactive/Paral-ITP.v
index 09ec9de17..d8961c98d 100644
--- a/test-suite/interactive/Paral-ITP.v
+++ b/test-suite/interactive/Paral-ITP.v
@@ -22,6 +22,7 @@ Qed.
Lemma b : True.
Proof.
+ do 11 (cut Type; [ intro foo; clear foo | exact Type]).
sleep time.
idtac.
(* change in semantics: Print a. *)