aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coq.ml
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-16 19:28:14 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-16 19:28:14 +0000
commit842fc3a4314265a012f6903fc8e3c0093ee78920 (patch)
tree7e9090d56b22c02035dad787af21936a96b81837 /ide/coq.ml
parent5a6032ff8e8aec41bd78f3939142e0b6e0527b5d (diff)
add visibility of extraction messages in coqide
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10230 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'ide/coq.ml')
-rw-r--r--ide/coq.ml3
1 files changed, 3 insertions, 0 deletions
diff --git a/ide/coq.ml b/ide/coq.ml
index c764cd5e3..50536491c 100644
--- a/ide/coq.ml
+++ b/ide/coq.ml
@@ -153,6 +153,9 @@ let interp verbosely s =
| VernacCoFixpoint _
| VernacEndProof _
| VernacScheme _
+ | VernacExtend("Extraction", _)
+ | VernacExtend("ExtractionLibrary",_)
+ | VernacExtend("RecursiveExtractionLibrary",_)
-> Options.make_silent (not verbosely)
| _ -> ()
end;