index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
proofs
/
proof.mli
Commit message (
Expand
)
Author
Age
*
[proof] [api] Rename proof types in preparation for functionalization.
Emilio Jesus Gallego Arias
2017-11-29
*
[api] Remove aliases of `Evar.t`
Emilio Jesus Gallego Arias
2017-11-26
*
[proof] Attempt to deprecate some V82 parts of the proof API.
Emilio Jesus Gallego Arias
2017-11-19
*
[api] Insert miscellaneous API deprecation back to core.
Emilio Jesus Gallego Arias
2017-11-13
*
deprecate Pp.std_ppcmds type alias
Matej Košík
2017-07-27
*
Bump year in headers.
Pierre-Marie Pédrot
2017-07-04
*
Merge branch 'master'.
Pierre-Marie Pédrot
2017-02-14
|
\
*
|
Evar-normalizing functions now act on EConstrs.
Pierre-Marie Pédrot
2017-02-14
|
*
Adding a printer for Proof.proof reflecting the focusing layout.
Hugo Herbelin
2017-01-26
|
/
*
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
*
Fix some typos in comments.
Guillaume Melquiond
2015-02-23
*
Update headers.
Maxime Dénès
2015-01-12
*
new: Optimize Proof, Optimize Heap
Enrico Tassi
2014-11-09
*
Add [Info] command.
Arnaud Spiwack
2014-11-01
*
Remove unused functions for side effects.
Arnaud Spiwack
2014-10-22
*
Factored out IDE goal structure.
Carst Tankink
2014-10-01
*
Making the error message about bullets more precise.
Pierre Courtieu
2014-07-31
*
Proof_global.start_dependent_proof: properly threads the sigma through the te...
Arnaud Spiwack
2014-07-23
*
Proofs now take and return an evar_universe_context, simplifying interfaces
Matthieu Sozeau
2014-06-18
*
Correct rebase on STM code. Thanks to E. Tassi for help on dealing with
Matthieu Sozeau
2014-05-06
*
This commit adds full universe polymorphism and fast projections to Coq.
Matthieu Sozeau
2014-05-06
*
Remove many superfluous 'open' indicated by ocamlc -w +33
Pierre Letouzey
2014-03-05
*
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
*
Moving side effects into evar_map. There was no reason to keep another
ppedrot
2013-10-05
*
State Transaction Machine
gareuselesinge
2013-08-08
*
Merging Context and Sign.
ppedrot
2013-04-29
*
Remove the unused "intel" field in Proof.proof_state
letouzey
2012-10-02
*
Updating headers.
herbelin
2012-08-08
*
Small change in the printing of proofs for use by coqide.
aspiwack
2012-07-10
*
Change how the number of open goals is printed.
aspiwack
2012-07-04
*
New files intf/constrexpr.mli and intf/notation_term.mli out of Topconstr
letouzey
2012-05-29
*
Added a command "Unfocused" which returns an error when the proof is
aspiwack
2012-03-30
*
Arranged for the desirable behaviour that bullets do not see beyond braces.
aspiwack
2012-03-20
*
Removed a superfluous function in proof.mli. Preparing for incoming
aspiwack
2012-03-01
*
A "Grab Existential Variables" to transform the unresolved evars at the end o...
aspiwack
2012-02-07
*
Typo in comments.
aspiwack
2012-02-07
*
Proof using ...
gareuselesinge
2011-12-12
*
In emacs mode, prints a list of the dependent existential variables introduced
aspiwack
2011-11-23
*
Adds a new command Show Goal (e.g. Show Goal "42") printing a goal using the...
aspiwack
2011-09-12
*
Fixed bullets so that they would play well with { }.
aspiwack
2011-07-06
*
Fixed a bug causing inconsistent states during proof editting.
aspiwack
2011-04-29
*
Some comments.
aspiwack
2011-04-29
*
Started to fix the declarative proof mode (C-zar).
aspiwack
2011-02-10
[next]