aboutsummaryrefslogtreecommitdiff
path: root/stm/proofBlockDelimiter.ml
AgeCommit message (Expand)Author
2020-09-01Unify the shelvesMaxime Dénès
2020-08-26Move given_up goals to evar_mapMaxime Dénès
2020-06-26[declare] Move proof information to declare.Emilio Jesus Gallego Arias
2020-04-15[declare] Rename `Declare.t` to `Declare.Proof.t`Emilio Jesus Gallego Arias
2020-04-15[proof] Merge `Proof_global` into `Declare`Emilio Jesus Gallego Arias
2020-03-18Update headers in the whole code base.Théo Zimmermann
2019-11-21[coq] Untabify the whole ML codebase.Emilio Jesus Gallego Arias
2019-08-14[vernac] Refactor Vernacular Control Attributes into a listEmilio Jesus Gallego Arias
2019-06-25[lemmas] Move `Stack` out of Lemmas.Emilio Jesus Gallego Arias
2019-06-17Update ml-style headers to new year.Théo Zimmermann
2019-06-09[proof] Move proofs that have an associated constant to `Lemmas`Emilio Jesus Gallego Arias
2019-06-04Proof_global: pass only 1 pstate when we don't want the proof stackGaëtan Gilbert
2019-05-13Passing evar_map to evars_of_term rather than expecting the term to be evar-nf.Hugo Herbelin
2019-05-13Moving Evd.evars_of_term from constr to econstr + consequences.Hugo Herbelin
2019-04-25[vernac] [ast] Make location info an attribute of vernaculars.Emilio Jesus Gallego Arias
2019-03-27[vernac] Adapt to removal of imperative proof state.Emilio Jesus Gallego Arias
2018-12-14[proof] Rework proof interface.Emilio Jesus Gallego Arias
2018-05-01[api] Move bullets and goals selectors to `proofs/`Emilio Jesus Gallego Arias
2018-04-13Evar maps contain econstrs.Gaëtan Gilbert
2018-02-27Update headers following #6543.Théo Zimmermann
2018-01-08[vernac] vernac_expr no longer recursiveVincent Laporte
2017-12-20Separate vernac controls and regular commands.Maxime Dénès
2017-11-19[plugins] Prepare plugin API for functional handling of state.Emilio Jesus Gallego Arias
2017-10-17[stm] Move interpretation state to VernacentriesEmilio Jesus Gallego Arias
2017-10-06[stm] Switch to a functional APIEmilio Jesus Gallego Arias
2017-07-04Bump year in headers.Pierre-Marie Pédrot
2016-10-18[stm] Fix record field name clash.Emilio Jesus Gallego Arias
2016-06-07DocumentationEnrico Tassi
2016-06-06Error box detection run only on errorEnrico Tassi
2016-06-06STM: proof block detection for indentationEnrico Tassi
2016-06-06STM: proof block detection for par:Enrico Tassi
2016-06-06STM: proof block detection for bullets and { block }Enrico Tassi