aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide
diff options
context:
space:
mode:
Diffstat (limited to 'ide')
-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;