aboutsummaryrefslogtreecommitdiff
path: root/coq/coq-indent.el
AgeCommit message (Expand)Author
2020-10-16Fix #514 + support for named goal selector.Pierre Courtieu
2019-12-04Uncommented coq-find-comment-start, coq-find-comment-end as quick fix for #444Vadim Zaliva
2019-02-12Simpler fix for #411.Pierre Courtieu
2019-02-12Fixes #411.Pierre Courtieu
2018-12-26Make coq-mode work without generic/proof-*Stefan Monnier
2018-12-15Cosmetic cleanup of coq-smie, coq-syntax, and coq-abbrev.Stefan Monnier
2018-12-12Cleanup patch; Moving defvar to toplevelStefan Monnier
2018-08-23Fix most doc issues raised by (checkdoc)Erik Martin-Dorel
2018-02-21Update copyright messages and improve the header of elisp files.Erik Martin-Dorel
2018-01-26look for vernac controls before focus bracket, fix for #223Paul Steckler
2018-01-15Experimental fix for #220.Pierre Courtieu
2017-03-08Fix incorrect uses of defvarClément Pit--Claudel
2016-05-27Fixing a smal glitch in indentation.Pierre Courtieu
2016-01-14Fix #29 + indentation glitch + regexp refactoring.Pierre Courtieu
2015-12-07Speeding up indentation (regexp optim).Pierre Courtieu
2015-12-07Speeding up indentation.Pierre Courtieu
2015-12-05Fixed #15 + more speedup of indentation.Pierre Courtieu
2015-01-27Fixed a bug in script navigation. Updated CHANGEPierre Courtieu
2014-12-30removed debug message.Pierre Courtieu
2014-12-30fixed indentation (lexing of 'with') + made local coq-load-path.Pierre Courtieu
2014-12-24fixed a bug in command parsing for coq, due to recent changes.Pierre Courtieu
2014-12-23Supporting more bullets (coq 8.5), like ++ or ++++.Pierre Courtieu
2012-08-30Summary: Don't quote lambda expressionsStefan Monnier
2012-07-05Fixed a syntactic recognition function. Should Fix #2819.Pierre Courtieu
2012-06-14Fix a bug in coq indet code when at the beginning of a buffer.Pierre Courtieu
2012-06-11Trying to minimize the slowness of indentation when no "Proof." isPierre Courtieu
2012-02-10Fixed an ineficiency in comment detection.Pierre Courtieu
2012-02-01Cleaning some code.Pierre Courtieu
2012-02-01Quick fix of a regression introduced by my last commit. Looking for aPierre Courtieu
2012-02-01Fixed command end recognition in presence of operators of the form .+Pierre Courtieu
2011-12-16Adapting coq syntax recognition to the future v8.4 behavior of bulletsPierre Courtieu
2011-09-04Fix trac #420 indentation freezing.Pierre Courtieu
2011-08-23Crude patch for Trac #416. I haven't tried to understand indent code fully, ...David Aspinall
2011-07-08Fixing the scripting of new subproof script parenthesizing ({ and }).Pierre Courtieu
2011-06-19Removed { and } as command terminators for now.Pierre Courtieu
2011-06-10Fix trac #410.Pierre Courtieu
2011-06-09Fix compile errors (seems to be code duplication between coq.el and coq-indent)David Aspinall
2011-06-072011-06-07 Stefan Monnier <monnier@iro.umontreal.ca>Stefan Monnier
2011-06-04Updated the old code for indentation, in case Stefan cannot finish thePierre Courtieu
2011-05-31Some small fixes in indentation for coq.Pierre Courtieu
2011-05-31Added indentation for BeginSubProof/EndSubProof.Pierre Courtieu
2010-09-09Fixed the cleaning of goals buffer when proof completedPierre Courtieu
2010-09-09Cleaning indentation code.Pierre Courtieu
2010-09-09Fixed indentation at end of file.Pierre Courtieu
2010-09-09Fixed small bugs in indentation.Pierre Courtieu
2010-09-07Finished fixing the small indentation bug at buffer top.Pierre Courtieu
2010-09-07Fix of previous commit.Pierre Courtieu
2010-09-07half fixed the indentation bug at buffer start.Pierre Courtieu
2010-09-03First fix of bug introduced by the last font-lock fix. Not finished.Pierre Courtieu
2010-09-01Fixed bug #346. Coq code was using proof-ids-to-regexp on regexpPierre Courtieu