index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
proofs
/
proof.ml
Commit message (
Expand
)
Author
Age
*
Adding a printer for Proof.proof reflecting the focusing layout.
Hugo Herbelin
2017-01-26
*
Merge branch 'v8.6'
Pierre-Marie Pédrot
2016-10-12
|
\
|
*
Merge branch 'v8.5' into v8.6
Pierre-Marie Pédrot
2016-10-12
|
|
\
|
|
*
Fix bug #5123: mark all shelved evars unresolvable
Matthieu Sozeau
2016-10-11
*
|
|
Make the user_err header an optional parameter.
Emilio Jesus Gallego Arias
2016-08-19
*
|
|
Remove errorlabstrm in favor of user_err
Emilio Jesus Gallego Arias
2016-08-19
|
/
/
*
|
errors.ml renamed into cErrors.ml (avoid clash with an OCaml compiler-lib mod...
Pierre Letouzey
2016-07-03
*
|
Moving Refine to its proper module.
Pierre-Marie Pédrot
2016-03-20
*
|
Extruding the code for the Existential command from Proofview.
Pierre-Marie Pédrot
2016-03-20
|
/
*
Update copyright headers.
Maxime Dénès
2016-01-20
*
Proof: suggest Admitted->Qed only if the proof is really complete (#4349)
Enrico Tassi
2015-09-20
*
STM/Univ: save initial univs (the ones in the statement) in Proof.proof
Enrico Tassi
2015-05-29
*
Update headers.
Maxime Dénès
2015-01-12
*
Make sure the goals on the shelve are identified as goal and unresolvable for...
Arnaud Spiwack
2014-12-12
*
Fix (somewhat obsolete) [Existential] command, which conflicted with the shelf.
Arnaud Spiwack
2014-11-28
*
new: Optimize Proof, Optimize Heap
Enrico Tassi
2014-11-09
*
Add [Info] command.
Arnaud Spiwack
2014-11-01
*
An API for info traces.
Arnaud Spiwack
2014-11-01
*
Evd.future_goals: forgot to revert the list in two places.
Arnaud Spiwack
2014-10-23
*
Proofview: move [list_goto] to the [CList] module.
Arnaud Spiwack
2014-10-22
*
Proofview: remove a redundant primitive.
Arnaud Spiwack
2014-10-22
*
Proofview: move more functions to the Unsafe module.
Arnaud Spiwack
2014-10-22
*
Remove unused functions for side effects.
Arnaud Spiwack
2014-10-22
*
Refactoring proofview: make the definition of the logic monad polymorphic.
Arnaud Spiwack
2014-10-16
*
Put evars remaining after a tactic on the shelf.
Arnaud Spiwack
2014-10-16
*
Goal: remove [advance] from the API.
Arnaud Spiwack
2014-10-16
*
Factored out IDE goal structure.
Carst Tankink
2014-10-01
*
Small reorganisation in proof.ml.
Arnaud Spiwack
2014-07-25
*
Fail gracefully when focusing on non-existing goals with user commands.
Arnaud Spiwack
2014-07-25
*
Proof_global.start_dependent_proof: properly threads the sigma through the te...
Arnaud Spiwack
2014-07-23
*
Transfering the initial goals from the proofview to the proof object.
Pierre-Marie Pédrot
2014-04-07
*
Fixing backtrace registering of various tactic-related try-with blocks.
Pierre-Marie Pédrot
2013-12-11
*
Allow proofs to start with dependent goals.
Arnaud Spiwack
2013-12-04
*
Allowing proofs starting with a non-empty evarmap.
ppedrot
2013-11-04
*
Update comments.
aspiwack
2013-11-02
*
Adds a tactic give_up.
aspiwack
2013-11-02
*
Adds a shelve tactic.
aspiwack
2013-11-02
*
The tactic [admit] exits with the "unsafe" status.
aspiwack
2013-11-02
*
Getting rid of Goal.here, and all the related exceptions and combinators.
aspiwack
2013-11-02
*
Moving side effects into evar_map. There was no reason to keep another
ppedrot
2013-10-05
*
Removing a bunch of generic equalities.
ppedrot
2013-09-27
*
get rid of closures in global/proof state
gareuselesinge
2013-08-08
*
State Transaction Machine
gareuselesinge
2013-08-08
*
Merging Context and Sign.
ppedrot
2013-04-29
*
another Errors.push in a exception reraise
letouzey
2013-03-16
*
Restrict (try...with...) to avoid catching critical exn (part 12)
letouzey
2013-03-13
*
Monomorphization (proof)
ppedrot
2012-11-25
*
Remove the unused "intel" field in Proof.proof_state
letouzey
2012-10-02
*
Remove some more "open" and dead code thanks to OCaml4 warnings
letouzey
2012-10-02
*
Updating headers.
herbelin
2012-08-08
[next]