aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/coq-syntax.el
Commit message (Expand)AuthorAge
...
* Fixes #484. Added syntax.Gravatar Pierre Courtieu2015-05-07
* bold unicode biders + Fixing highlighting in goals and response buffers + cle...Gravatar Pierre Courtieu2015-04-14
* Debugging font-lock for ∀, ∃, and λ.Gravatar Pierre Courtieu2015-04-13
* Added unicode forall in font-lock regexps.Gravatar Pierre Courtieu2015-04-10
* Fixed coq-id definition to be correct wrt to coq grammar.Gravatar Pierre Courtieu2015-04-07
* Fixed highlighting of evars.Gravatar Pierre Courtieu2015-04-07
* Fix disable evar colorizing in coq file.Gravatar Pierre Courtieu2015-03-27
* Colorizing hyps names robustified. Still incomplete.Gravatar Pierre Courtieu2015-03-26
* Fixed a smal bug in colorizing response buffer.Gravatar Pierre Courtieu2015-03-26
* fixed gfail hilighting.Gravatar Pierre Courtieu2015-03-24
* added some keywordsGravatar Pierre Courtieu2015-03-24
* Highlighting evars.Gravatar Pierre Courtieu2015-03-23
* Fixed lazymatch and multimatch indentation/highlighting.Gravatar Pierre Courtieu2015-03-23
* Some comments for future work.Gravatar Pierre Courtieu2015-03-13
* Added a command to send Queries to coq, with completion (C-c C-a C-q).Gravatar Pierre Courtieu2015-03-13
* Fixed Proof end/start detection on Proof using ...Gravatar Pierre Courtieu2015-03-04
* Fixed a bug in syntax table making fontlock and indentation fail.Gravatar Pierre Courtieu2015-02-23
* Fix colorization of for coq multiple hypothesis on the same line.Gravatar Pierre Courtieu2015-02-05
* Fixed previous commit (wrong regexp).Gravatar Pierre Courtieu2015-02-04
* coloring names in resposne and goalsGravatar Pierre Courtieu2015-02-03
* beautified a bit error messages.Gravatar Pierre Courtieu2015-02-03
* * coq/coq-smie.el: Fix precedence of 'else'.Gravatar Stefan Monnier2014-06-06
* Fixing #477. Adding Proposition as a goal-starter keyword.Gravatar Pierre Courtieu2013-07-10
* Fixing compilation. Still need to verify some smie stuff on different version...Gravatar Pierre Courtieu2012-07-24
* Complete rework of the indentation mechanism using smie. The firstGravatar Pierre Courtieu2012-06-28
* Trying to minimize the slowness of indentation when no "Proof." isGravatar Pierre Courtieu2012-06-11
* 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
* Added indentation for BeginSubProof/EndSubProof.Gravatar Pierre Courtieu2011-05-31
* Fixed #394. There is a bug with kfont-lock-keywords. The workaround isGravatar Pierre Courtieu2011-05-17
* * fix overwriting setq coq-prog-name before loading Proof GeneralGravatar Hendrik Tews2011-04-15
* Add preliminary support for multiple files for coq.Gravatar Hendrik Tews2011-01-12
* coq-generic-expression: fix this to match symbols, not merely words.Gravatar David Aspinall2010-10-10
* 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
* 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