@@ -38,6 +38,8 @@ OTHERBINARIES:=$(COQMKTOPBYTE) $(COQCBYTE)
38
38
39
39
MINICOQ:=bin/minicoq$(EXE)
40
40
41
+ CSDPCERT:=bin/csdpcert
42
+
41
43
###########################################################################
42
44
# tools
43
45
###########################################################################
@@ -212,13 +214,8 @@ TOPLEVEL:=\
212
214
213
215
HIGHTACTICS:=\
214
216
tactics/refine.cmo tactics/extraargs.cmo \
215
- tactics/extratactics.cmo tactics/eauto.cmo tactics/class_tactics.cmo
216
-
217
- SPECTAC:= tactics/tauto.ml4 tactics/eqdecide.ml4
218
- USERTAC:= $(SPECTAC)
219
-
220
- USERTACCMO:=$(USERTAC:.ml4=.cmo)
221
- USERTACCMX:=$(USERTAC:.ml4=.cmx)
217
+ tactics/extratactics.cmo tactics/eauto.cmo tactics/class_tactics.cmo \
218
+ tactics/tauto.cmo tactics/eqdecide.cmo
222
219
223
220
OMEGACMO:=\
224
221
contrib/omega/omega.cmo contrib/omega/coq_omega.cmo \
@@ -228,6 +225,12 @@ ROMEGACMO:=\
228
225
contrib/romega/const_omega.cmo \
229
226
contrib/romega/refl_omega.cmo contrib/romega/g_romega.cmo
230
227
228
+ MICROMEGACMO:=\
229
+ contrib/micromega/mutils.cmo contrib/micromega/vector.cmo \
230
+ contrib/micromega/micromega.cmo contrib/micromega/mfourier.cmo \
231
+ contrib/micromega/certificate.cmo \
232
+ contrib/micromega/coq_micromega.cmo contrib/micromega/g_micromega.cmo
233
+
231
234
RINGCMO:=\
232
235
contrib/ring/quote.cmo contrib/ring/g_quote.cmo \
233
236
contrib/ring/ring.cmo contrib/ring/g_ring.cmo
@@ -302,7 +305,8 @@ SUBTACCMO:=contrib/subtac/subtac_utils.cmo contrib/subtac/eterm.cmo \
302
305
RTAUTOCMO:=contrib/rtauto/proof_search.cmo contrib/rtauto/refl_tauto.cmo \
303
306
contrib/rtauto/g_rtauto.cmo
304
307
305
- CONTRIB:=$(OMEGACMO) $(ROMEGACMO) $(RINGCMO) $(NEWRINGCMO) $(DPCMO) $(FIELDCMO) \
308
+ CONTRIB:=$(OMEGACMO) $(ROMEGACMO) $(MICROMEGACMO) \
309
+ $(RINGCMO) $(NEWRINGCMO) $(DPCMO) $(FIELDCMO) \
306
310
$(FOURIERCMO) $(EXTRACTIONCMO) $(JPROVERCMO) $(XMLCMO) \
307
311
$(CCCMO) $(FOCMO) $(SUBTACCMO) $(RTAUTOCMO) \
308
312
$(FUNINDCMO)
@@ -325,7 +329,7 @@ LINKCMX:=$(LINKCMOCMXA:.cmo=.cmx)
325
329
# objects known by the toplevel of Coq
326
330
OBJSCMO:=$(CONFIG) $(LIBREP) $(KERNEL) $(LIBRARY) $(PRETYPING) $(INTERP) \
327
331
$(PROOFS) $(PARSING) $(TACTICS) $(TOPLEVEL) $(HIGHPARSING) \
328
- $(HIGHTACTICS) $(USERTACMO) $( CONTRIB)
332
+ $(HIGHTACTICS) $(CONTRIB)
329
333
330
334
COQIDECMO:=ide/utils/okey.cmo ide/utils/config_file.cmo \
331
335
ide/utils/configwin_keys.cmo ide/utils/configwin_types.cmo \
@@ -375,6 +379,12 @@ PARSERCMX:= $(PARSERREQUIRESCMX) $(PARSERCODE:.cmo=.cmx)
375
379
376
380
INTERFACERC:= contrib/interface/vernacrc
377
381
382
+ CSDPCERTCMO:= contrib/micromega/mutils.cmo contrib/micromega/micromega.cmo \
383
+ contrib/micromega/vector.cmo contrib/micromega/mfourier.cmo \
384
+ contrib/micromega/certificate.cmo \
385
+ contrib/micromega/sos.cmo contrib/micromega/csdpcert.cmo
386
+ CSDPCERTCMX:= $(CSDPCERTCMO:.cmo=.cmx)
387
+
378
388
DEBUGPRINTERS:=dev/top_printers.cmo dev/vm_printers.cmo dev/printers.cma
379
389
380
390
COQDEPCMO:=config/coq_config.cmo tools/coqdep_lexer.cmo tools/coqdep.cmo
@@ -704,6 +714,15 @@ OMEGAVO:=$(addprefix contrib/omega/, \
704
714
ROMEGAVO:=$(addprefix contrib/romega/, \
705
715
ReflOmegaCore.vo ROmega.vo )
706
716
717
+ MICROMEGAVO:=$(addprefix contrib/micromega/, \
718
+ CheckerMaker.vo Refl.vo \
719
+ Env.vo RingMicromega.vo \
720
+ EnvRing.vo VarMap.vo \
721
+ OrderedRing.vo ZCoeff.vo \
722
+ Micromegatac.vo ZMicromega.vo \
723
+ QMicromega.vo RMicromega.vo \
724
+ Tauto.vo )
725
+
707
726
RINGVO:=$(addprefix contrib/ring/, \
708
727
LegacyArithRing.vo Ring_normalize.vo \
709
728
LegacyRing_theory.vo LegacyRing.vo \
@@ -751,9 +770,9 @@ SUBTACVO:=$(addprefix theories/Program/, \
751
770
RTAUTOVO:=$(addprefix contrib/rtauto/, \
752
771
Bintree.vo Rtauto.vo )
753
772
754
- CONTRIBVO:= $(OMEGAVO) $(ROMEGAVO) $(RINGVO ) $(FIELDVO ) $(XMLVO ) \
755
- $(FOURIERVO ) $(JPROVERVO ) $(CCVO ) $(FUNINDVO ) $(SUBTACVO ) \
756
- $(RTAUTOVO) $(RECDEFVO) $(NEWRINGVO) $(DPVO)
773
+ CONTRIBVO:= $(OMEGAVO) $(ROMEGAVO) $(MICROMEGAVO ) $(RINGVO ) $(FIELDVO ) \
774
+ $(XMLVO ) $(FOURIERVO ) $(JPROVERVO ) $(CCVO ) $(FUNINDVO ) \
775
+ $(SUBTACVO) $( RTAUTOVO) $(RECDEFVO) $(NEWRINGVO) $(DPVO)
757
776
758
777
ALLVO:= $(INITVO) $(THEORIESVO) $(CONTRIBVO)
759
778
@@ -808,12 +827,12 @@ STAGE1_TARGETS:= $(STAGE1) \
808
827
STAGE2_TARGETS:=$(COQBINARIES) lib kernel byterun library proofs tactics \
809
828
interp parsing pretyping highparsing toplevel hightactics \
810
829
coqide-binaries coqide-byte coqide-opt $(COQIDEOPT) $(COQIDEBYTE) $(COQIDE) \
811
- pcoq-binaries $(COQINTERFACE) coqbinaries pcoq $(TOOLS) tools \
830
+ pcoq-binaries $(COQINTERFACE) $(CSDPCERT) coqbinaries pcoq $(TOOLS) tools \
812
831
printers $(MINICOQ) debug
813
832
VO_TARGETS:=logic arith bool narith zarith qarith lists strings sets \
814
833
fsets allfsets relations wellfounded ints reals allreals \
815
834
setoids sorting natural integer rational numbers noreal \
816
- omega ring setoid_ring dp xml extraction field fourier jprover \
835
+ omega micromega ring setoid_ring dp xml extraction field fourier jprover \
817
836
funind cc programs subtac rtauto
818
837
DOC_TARGETS:=doc doc-html doc-ps doc-pdf stdlib refman tutorial faq rectutorial
819
838
STAGE3_TARGETS:=world install coqide coqide-files coq coqlib \
0 commit comments