aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/goal.ml
Commit message (Expand)AuthorAge
* Use evar name to print goal.Gravatar Hugo Herbelin2014-09-12
* Only using filtered hyps in Goal.enter.Gravatar Pierre-Marie Pédrot2014-09-04
* Ensuring the invariant that hypotheses and named context of the environment ofGravatar Pierre-Marie Pédrot2014-09-04
* Fix: shelve_unifiable did not work modulo evar instantiation.Gravatar Arnaud Spiwack2014-09-04
* Putting back normalized goals when entering them.Gravatar Pierre-Marie Pédrot2014-09-03
* Removing unused parts of the Goal.sensitive monad.Gravatar Pierre-Marie Pédrot2014-08-21
* Removing a use of Goal.refine.Gravatar Pierre-Marie Pédrot2014-08-19
* Goal: API to get the solution of a goalGravatar Enrico Tassi2014-08-05
* Tentative optimization not to nf_evar too often in the compatibilityGravatar Pierre-Marie Pédrot2014-06-17
* Better representation of evar filters: we represent the vacuous filters ofGravatar Pierre-Marie Pédrot2014-04-23
* Adding phantom types to discriminate normalized goals, and adding a way toGravatar Pierre-Marie Pédrot2014-03-19
* Potentially unused computation in Goal.Gravatar Pierre-Marie Pédrot2014-03-07
* Code refactoring thanks to the new Monad module.Gravatar Arnaud Spiwack2014-02-27
* TC: honor the use_typeclasses flag in pretypingGravatar Enrico Tassi2014-02-12
* Useless Array.of_listGravatar Pierre-Marie Pédrot2014-01-10
* Exporting the full pretyper options in Goal.constr_of_raw.Gravatar Pierre-Marie Pédrot2014-01-10
* Fixing ltac constr variable handling in refine.Gravatar Pierre-Marie Pédrot2013-11-30
* Useless computation in Goal handle augmentation.Gravatar ppedrot2013-11-12
* Partial applications in Goal.Gravatar ppedrot2013-11-09
* Less partial applications in Vars, as well as better memory allocation.Gravatar ppedrot2013-11-06
* Add primitives in Goal.V82 to access the goal in nf_evar'd form.Gravatar aspiwack2013-11-02
* A tactic shelve_unifiable.Gravatar aspiwack2013-11-02
* Normalise goals with respect to evars in the new tactics.Gravatar aspiwack2013-11-02
* Tachmach.New is now in Proofview.Goal.enter style.Gravatar aspiwack2013-11-02
* A better version of Goal.advance.Gravatar aspiwack2013-11-02
* More optimisations of partial applications.Gravatar aspiwack2013-11-02
* Try to remove intermediate allocations when dealing with goal-specific tactics.Gravatar aspiwack2013-11-02
* A whole new implemenation of the refine tactic.Gravatar aspiwack2013-11-02
* Getting rid of Goal.here, and all the related exceptions and combinators.Gravatar aspiwack2013-11-02
* Makes the new Proofview.tactic the basic type of Ltac.Gravatar aspiwack2013-11-02
* Abstracting evar filter away. The API is not perfect, but better than nothing.Gravatar ppedrot2013-10-27
* More monomorphic List.mem + List.assoc + ...Gravatar letouzey2013-10-24
* Removing dubious use of evarmap manipulating functions in printingGravatar ppedrot2013-10-05
* Moving side effects into evar_map. There was no reason to keep anotherGravatar ppedrot2013-10-05
* At least made the evar type opaque! There are still 5 remaining unsafeGravatar ppedrot2013-09-18
* Removing almost all new_untyped_evar, and a bunch of Evd.add.Gravatar ppedrot2013-09-18
* State Transaction MachineGravatar gareuselesinge2013-08-08
* A uniformization step around understand_* and interp_* functions.Gravatar herbelin2013-05-09
* Splitting Term into five unrelated interfaces:Gravatar ppedrot2013-04-29
* Restrict (try...with...) to avoid catching critical exn (part 12)Gravatar letouzey2013-03-13
* Allowing different types of, not to be mixed, generic Stores throughGravatar ppedrot2013-03-12
* No reason a priori for using unfiltered env for printingGravatar herbelin2013-01-29
* Fixing bug #2969 (admit failing after Grab Existential Variables dueGravatar herbelin2013-01-29
* Fixed synchronicity of filter with evar context in new_goal_with.Gravatar herbelin2013-01-29
* Renaming evar_env/evar_unfiltered_env into evar_filtered_env/evar_envGravatar herbelin2013-01-29
* Uniformization of the "anomaly" command.Gravatar ppedrot2013-01-28
* Modulification of identifierGravatar ppedrot2012-12-14
* Renamed Option.Misc.compare to the more uniform Option.equal.Gravatar ppedrot2012-12-13
* Monomorphization (proof)Gravatar ppedrot2012-11-25
* Updating headers.Gravatar herbelin2012-08-08