aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/coq-syntax.el
Commit message (Collapse)AuthorAge
* Complete rework of the indentation mechanism using smie. The firstGravatar Pierre Courtieu2012-06-28
| | | | | | version of smie indentation code was a good first try but this one is much faster and cleaner. All desambiguations are done in the lexers, it is still a bit slow on large proofs. Some bugs remain to be fixed.
* Trying to minimize the slowness of indentation when no "Proof." isGravatar Pierre Courtieu2012-06-11
| | | | given. Seems to work.
* Trying to fix some minor indentation bugs with infox operators.Gravatar Pierre Courtieu2012-06-06
|
* Fix of a bug. coq id can start with underscore.Gravatar Pierre Courtieu2012-05-31
|
* Move coq-prog-name back to coq.elGravatar David Aspinall2011-08-23
|
* Fixing track 414 by adding Preterm as a state preserving command.Gravatar Pierre Courtieu2011-07-29
|
* Updated the old code for indentation, in case Stefan cannot finish theGravatar Pierre Courtieu2011-06-04
| | | | | | | new one for the release. Added also support for an experimental syntax modification: { .. } is a new syntax for Beginsubproof. ... EndSubproof. There a also few minor behavior changes. The code has changed a lot though.
* Added indentation for BeginSubProof/EndSubProof.Gravatar Pierre Courtieu2011-05-31
| | | | + added some tactics syntax.
* Fixed #394. There is a bug with kfont-lock-keywords. The workaround isGravatar Pierre Courtieu2011-05-17
| | | | to change the order in which keywords appear. TO FIX.
* * fix overwriting setq coq-prog-name before loading Proof GeneralGravatar Hendrik Tews2011-04-15
| | | | * more complete callback listing in proof-action list doc
* Add preliminary support for multiple files for coq.Gravatar Hendrik Tews2011-01-12
| | | | | | | | | | | | | | | The following points are implemented already: - recompile either via an external command (make) or let ProofGeneral handle everything internally - complete dependency tracking and recompilation for coq files in internal mode - support for extending the LoadPath: does almost work, even if specified file-locally - move back to clean state if recompilation fails There are the following known problems: - coq-load-path extensions are not retracted - fails on partially qualified library names
* coq-generic-expression: fix this to match symbols, not merely words.Gravatar David Aspinall2010-10-10
| | | | Otherwise we only see first word of symbols using underscores!
* ReFixed bug trac 356.Gravatar Pierre Courtieu2010-10-01
|
* Fixed colorization bug #356, introduced by a previous fix of bug 140.Gravatar Pierre Courtieu2010-09-28
|
* Fix bug trac 140 by writing a cleaner regexp than (proof-ids ... " ").Gravatar Pierre Courtieu2010-09-22
|
* Fix some bugs in coq regexp generationGravatar David Aspinall2010-09-22
|
* Remove support for Emacs <21 in syntax tableGravatar David Aspinall2010-09-22
|
* Cleaning indentation code.Gravatar Pierre Courtieu2010-09-09
|
* Fixed indentation which was broken by a previous commit.Gravatar Pierre Courtieu2010-09-03
|
* Adding some keywords.Gravatar Pierre Courtieu2010-09-03
|
* First fix of bug introduced by the last font-lock fix. Not finished.Gravatar Pierre Courtieu2010-09-03
|
* Fixed bug #346. Coq code was using proof-ids-to-regexp on regexpGravatar Pierre Courtieu2010-09-01
| | | | instead of pure strings.
* Fix commentGravatar David Aspinall2010-08-30
|
* Fix syntax for Local prefix (see Trac #348)Gravatar David Aspinall2010-08-30
|
* Added a "remember this" window. Experimental.Gravatar Pierre Courtieu2010-05-17
|
* Added some more syntax keywords. Made admit tactic with its own redGravatar Pierre Courtieu2009-09-17
| | | | culpabilizing face.
* Added some syntax keywords thanks to Mathieu Sozeau.Gravatar Pierre Courtieu2009-09-17
|
* Clean compileGravatar David Aspinall2009-09-10
|
* Fix compilation for Coq, including requires and some old/renamed settings.Gravatar David Aspinall2009-09-10
|
* Remove Coq 8.0 codeGravatar David Aspinall2009-09-08
|
* Remove more of 80 codeGravatar David Aspinall2009-09-08
|
* Fix compile warnings and ensure compiled code behaves as expected.Gravatar David Aspinall2009-09-07
|
* Clean whitespaceGravatar David Aspinall2009-09-05
|
* Made customizable holes mode completion in abbreviations.Gravatar Pierre Courtieu2009-08-31
|
* Minor changes from Stefan Monnier's patchGravatar David Aspinall2009-08-17
|
* Merge changes from Version4Branch.Gravatar David Aspinall2008-07-24
|
* todo added fo coq.Gravatar Pierre Courtieu2008-07-21
|
* Fixed a bug with coq-prog-name.Gravatar Pierre Courtieu2008-05-20
|
* Small fix with response buffer scrolling.Gravatar Pierre Courtieu2008-04-11
| | | | + starting the "insert as" feature.
* fixed syntax table + thing-at-point.Gravatar Pierre Courtieu2008-03-05
|
* coq:cutomizable bound variable highlight (finally working)Gravatar Assia Mahboubi2008-02-01
|
* Updated.Gravatar David Aspinall2008-01-31
|
* Use proof-locate-executable so works out-of-the-box on Windows.Gravatar David Aspinall2008-01-31
|
* Remove CVS merge junk!Gravatar David Aspinall2008-01-31
|
* updated CHANGESGravatar Assia Mahboubi2008-01-31
| | | | added an example file in coq/
* coq : sorry, reverting previous buggy customizationGravatar Assia Mahboubi2008-01-30
|
* Added a boolean defcustom test to make optional the highlight of variablesGravatar Assia Mahboubi2008-01-30
|
* coq : changing highlight of solve, adding ExportGravatar Assia Mahboubi2008-01-30
|
* Fixed indentation and goal display.Gravatar Pierre Courtieu2008-01-28
|
* Fixed a problem with a wrong side effect on syntax databases (whenGravatar Pierre Courtieu2008-01-28
| | | | sorting for menus).