aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Prelude.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-03-14 11:29:50 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-03-14 11:29:50 +0000
commit4b7200cbbf4f2462d6f1398a191377b4d57f7655 (patch)
tree3366f1dc2aeb1ff51961e100af8682fd44441683 /theories/Init/Prelude.v
parentc7219aeff951fead91fef7f1bb7ffb91617779e4 (diff)
Better mechanism for loading initial plugins
Instead of dirty hacks in toplevel/coqtop.ml, we simply add some Declare ML Module in Prelude.v. Gain: now that coqdep is clever enough, dependencies are automatic, and we can simplify the Makefile quite a lot: no more references to INITPLUGINSBEST and the like. Besides, mltop.ml4 can also be simplified a lot: by giving $(CONTRIBSTATIC) to coqmktop instead of contrib.cma, now coqtop is aware that it already contain the static plugins (or not), and subsequent ML Module are ignored correctly without us having to do anything :-) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11979 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Prelude.v')
-rw-r--r--theories/Init/Prelude.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/theories/Init/Prelude.v b/theories/Init/Prelude.v
index f0c67df3a..84de55e24 100644
--- a/theories/Init/Prelude.v
+++ b/theories/Init/Prelude.v
@@ -15,3 +15,11 @@ Require Export Specif.
Require Export Peano.
Require Export Coq.Init.Wf.
Require Export Coq.Init.Tactics.
+(* Initially available plugins *)
+Declare ML Module "extraction_plugin".
+Declare ML Module "cc_plugin".
+Declare ML Module "ground_plugin".
+Declare ML Module "dp_plugin".
+Declare ML Module "recdef_plugin".
+Declare ML Module "subtac_plugin".
+Declare ML Module "xml_plugin".