index
:
coq
master
The formal proof system
about
summary
refs
log
tree
commit
diff
log msg
author
committer
range
path:
root
/
proofs
Age
Commit message (
Expand
)
Author
2020-05-12
Remove a unused legacy tactic from Clenv.
Pierre-Marie Pédrot
2020-05-12
Write the outermost part of the legacy refiner directly in the monad.
Pierre-Marie Pédrot
2020-05-12
Clean up the legacy refiner implementation.
Pierre-Marie Pédrot
2020-05-12
Remove legacy Refiner error constructors.
Pierre-Marie Pédrot
2020-05-12
Wrap the legacy refiner type into the Logic API.
Pierre-Marie Pédrot
2020-05-12
Do not use Unsafe.to_constr for old refiner conclusion.
Pierre-Marie Pédrot
2020-05-07
Deprecate the legacy tacticals from module Refiner.
Pierre-Marie Pédrot
2020-05-05
Fix GeoCoq slowdown.
Pierre-Marie Pédrot
2020-05-03
Remove a very specific low-level tactical from Refiner.
Pierre-Marie Pédrot
2020-05-03
Wrap Refiner.refiner in the tactic monad.
Pierre-Marie Pédrot
2020-05-03
Remove a critical call to V82.tactic in Clenvtac.
Pierre-Marie Pédrot
2020-04-21
Merge PR #11896: Use lists instead of arrays in evar instances.
Maxime Dénès
2020-04-15
[proof] Move functions related to `Proof.t` to `Proof`
Emilio Jesus Gallego Arias
2020-04-15
[proof] Merge `Pfedit` into proofs.
Emilio Jesus Gallego Arias
2020-04-15
[proofs] Move pfedit to `proofs`
Emilio Jesus Gallego Arias
2020-04-06
Clean and fix definitions of options.
Théo Zimmermann
2020-04-06
Use lists instead of arrays in evar instances.
Pierre-Marie Pédrot
2020-03-31
Try only using TC for conversion in cominductive (not great but let's see)
Gaëtan Gilbert
2020-03-30
Merge PR #11921: Remove some cruft from Reductionops API.
Gaëtan Gilbert
2020-03-30
Merge PR #11817: [cleanup] Remove unnecessary Map/Set module creation
Gaëtan Gilbert
2020-03-28
Remove some cruft from Reductionops API.
Pierre-Marie Pédrot
2020-03-22
[proof] Deprecate unused tacmach functions.
Emilio Jesus Gallego Arias
2020-03-19
Merge PR #11735: Deprecating catchable_exception
Pierre-Marie Pédrot
2020-03-18
Update headers in the whole code base.
Théo Zimmermann
2020-03-13
[cleanup] Remove unnecessary Map/Set module creation
Emilio Jesus Gallego Arias
2020-03-13
Deprecation of catchable_exception, to be replaced by noncritical in try-with.
Hugo Herbelin
2020-03-13
Removing catchable_exception test in tclOR/tclORELSE.
Hugo Herbelin
2020-03-03
[exninfo] Deprecate aliases for exception re-raising.
Emilio Jesus Gallego Arias
2020-02-24
[exn] Forbid raising in exn printers, make them return Pp.t option
Emilio Jesus Gallego Arias
2020-02-18
Deprecate unsafe_type_of
Gaëtan Gilbert
2020-02-12
Remove Goptions.opt_name field
Gaëtan Gilbert
2020-02-06
unsafe_type_of -> type_of in Logic.check_typability
Gaëtan Gilbert
2020-02-06
Remove Clenv.mk_clenv_type_of (hidden unsafe_type_of)
Gaëtan Gilbert
2020-02-06
unsafe_type_of -> type_of in Celenv.mk_clenv_type_of
Gaëtan Gilbert
2020-01-30
[exn] Don't reraise in exception printers
Emilio Jesus Gallego Arias
2020-01-06
Fix #11140: Bidirectionality hints perform (surprising?) simplification
Maxime Dénès
2019-12-26
Remove uses of Global in Evd API.
Pierre-Marie Pédrot
2019-12-14
Fix refine and eapply to mark shelved goals as non-resolvable, always
Matthieu Sozeau
2019-11-21
[coq] Untabify the whole ML codebase.
Emilio Jesus Gallego Arias
2019-08-30
Merge PR #10714: Solve universe error with SSR 'rewrite !term'
Pierre-Marie Pédrot
2019-08-29
Solve universe error with SSR 'rewrite !term'
Andreas Lynge
2019-08-27
[declare] Move proof_entry type to declare, put interactive proof data on top...
Emilio Jesus Gallego Arias
2019-08-17
Delay the computation of frozen evars in legacy unification.
Pierre-Marie Pédrot
2019-07-11
[proof] Minor cleanup in proof.ml
Emilio Jesus Gallego Arias
2019-06-24
[proof] Remove last case of optional `?poly` arguments.
Emilio Jesus Gallego Arias
2019-06-24
[proof] Move initial_euctx to proof_global
Emilio Jesus Gallego Arias
2019-06-24
[proof] API Documentation fixes.
Emilio Jesus Gallego Arias
2019-06-24
[api] Remove `polymorphic` type alias, use labels instead.
Emilio Jesus Gallego Arias
2019-06-24
[lemmas] [proof] Split proof kinds into per-layer components.
Emilio Jesus Gallego Arias
2019-06-24
[proof] More uniformity in proof start labels.
Emilio Jesus Gallego Arias
[next]