aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/micromega
Commit message (Expand)AuthorAge
* Oups, repair the compilation (micromega + Morphism_prop)Gravatar letouzey2013-10-24
* Turn many List.assoc into List.assoc_fGravatar letouzey2013-10-24
* Reintroduce "or" instead of "||" as the latter is redifined in "sos_lib.ml" w...Gravatar xclerc2013-10-16
* Remove some uses of local modules (some were unused, some were costly).Gravatar xclerc2013-10-14
* Getting rid of the use of deprecated elements (from the OCaml standard library).Gravatar xclerc2013-10-14
* Get rid of the uses of deprecated OCaml elements (still remaining compatible ...Gravatar xclerc2013-09-19
* Misc changes around coqtop.ml :Gravatar letouzey2013-08-22
* micromega: remove empty file CheckerMakerGravatar letouzey2013-08-22
* Restrict (try...with...) to avoid catching critical exn (part 15)Gravatar letouzey2013-03-13
* Restrict (try...with...) to avoid catching critical exn (part 11)Gravatar letouzey2013-03-13
* invalid_arg instead of raise (Invalid_argement ...)Gravatar letouzey2013-03-12
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* Unset Asymmetric PatternsGravatar pboutill2013-01-18
* Modulification of identifierGravatar ppedrot2012-12-14
* Ensure that a function declared with a label is used with itGravatar letouzey2012-12-08
* Monomorphized a lot of equalities over OCaml integers, thanks toGravatar ppedrot2012-11-08
* still some more dead code removalGravatar letouzey2012-10-06
* Remove some more "open" and dead code thanks to OCaml4 warningsGravatar letouzey2012-10-02
* The new ocaml compiler (4.00) has a lot of very cool warnings,Gravatar regisgia2012-09-14
* Updating headers.Gravatar herbelin2012-08-08
* Try to make the use of Unix.lockf in micromega compatible with Win32Gravatar letouzey2012-08-06
* Ring_polynom : a restricted simpl instead of a unfold;foldGravatar letouzey2012-07-07
* Legacy Ring and Legacy Field migrated to contribsGravatar letouzey2012-07-05
* rewrite_db : a first attempt at using rewrite_strat for a quicker autorewriteGravatar letouzey2012-07-05
* More cleanup in Ring_polynom and EnvRingGravatar letouzey2012-07-05
* ZArith + other : favor the use of modern names instead of compat notationsGravatar letouzey2012-07-05
* Cleaning opening of the standard List module.Gravatar ppedrot2012-06-28
* More cleaningGravatar ppedrot2012-06-01
* place all files specific to camlp4 syntax extensions in grammar/Gravatar letouzey2012-05-29
* locus.mli for occurrences+clauses, misctypes.mli for various little thingsGravatar letouzey2012-05-29
* lib directory is cut in 2 cma.Gravatar pboutill2012-04-12
* Noise for nothingGravatar pboutill2012-03-02
* coq_micromega.ml: fix order of recursive calls to rconstantGravatar glondu2012-01-14
* More newlines in debugging output of psatzlGravatar glondu2012-01-14
* theories/, plugins/ and test-suite/ ported to the Arguments vernacularGravatar gareuselesinge2011-11-21
* Coq_micromega: generic = on constr replaced by eq_constrGravatar puech2011-07-29
* update of Micromega docGravatar fbesson2011-06-29
* improved tactic namesGravatar fbesson2011-06-28
* Numbers: a particular case of div_uniqueGravatar letouzey2011-06-24
* Q2R -> IQRGravatar fbesson2011-05-25
* git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14152 85f007b7-540e-0...Gravatar fbesson2011-05-23
* added support to handle division by a constant over RGravatar fbesson2011-05-20
* cbv delta - [...] before calling liaGravatar fbesson2011-05-18
* apply zeta reduction before syntaxificationGravatar fbesson2011-05-18
* Improved lia + experimental nliaGravatar fbesson2011-05-09
* Modularization of BinInt, related fixes in the stdlibGravatar letouzey2011-05-05
* Modularization of BinNat + fixes of stdlibGravatar letouzey2011-05-05
* Modularization of BinPos + fixes in StdlibGravatar letouzey2011-05-05
* Definitions of positive, N, Z moved in Numbers/BinNums.vGravatar letouzey2011-05-05
* bug fix: concurrent access of persistent_cacheGravatar fbesson2011-04-21