aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/coq.el
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2004-03-19 12:58:29 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2004-03-19 12:58:29 +0000
commit4791a7e43e5bb3dba154265abf3caa684663db83 (patch)
tree4ee84e05b24d63dffa42c004071c2b53f5a46969 /coq/coq.el
parent0ce0b8071577f7edd546b1e12135021bdbfeac10 (diff)
coq < 8.0 menu and abbrevs.
Diffstat (limited to 'coq/coq.el')
-rw-r--r--coq/coq.el174
1 files changed, 6 insertions, 168 deletions
diff --git a/coq/coq.el b/coq/coq.el
index d4c779f2..f8f3beff 100644
--- a/coq/coq.el
+++ b/coq/coq.el
@@ -84,174 +84,12 @@
:group 'coq)
-;; ----- coq specific menu
-
-;TODO: build the command submenu automatically from abbrev table
-(defpgdefault menu-entries
- '(
- ("Insert Command"
- "COMMAND ABBREVIATION"
- ["Definition def<C-BS>" (insert-and-expand "def") t]
- ["Fixpoint fix<C-BS>" (insert-and-expand "fix") t]
- ["Lemma l<C-BS>" (insert-and-expand "l") t]
- ""
- ["Inductive indv<C-BS>" (insert-and-expand "indv") t]
- ["Inductive1 indv1<C-BS>" (insert-and-expand "indv1") t]
- ["Inductive2 indv2<C-BS>" (insert-and-expand "indv2") t]
- ["Inductive3 indv3<C-BS>" (insert-and-expand "indv3") t]
- ["Inductive4 indv4<C-BS>" (insert-and-expand "indv4") t]
- ""
- ["Section..." coq-insert-section t]
- ""
- ("Modules"
- "COMMAND ABBREVIATION"
- ["Module (interactive)... " coq-insert-module t]
- ["Module mo<C-BS>" (insert-and-expand "mo") t]
- ["Module (<:) mo2<C-BS>" (insert-and-expand "mo") t]
-; ["Module (interactive) moi<C-BS>" (insert-and-expand "moi") t]
-; ["Module (interactive <:) moi2<C-BS>" (insert-and-expand "moi2") t]
- ["Module Type mt<C-BS>" (insert-and-expand "mt") t]
-; ["Module Type (interactive) mti<C-BS>" (insert-and-expand "mti") t]
-; ""
- ["Declare Module dm<C-BS>" (insert-and-expand "dm") t]
- ["Declare Module (<:) dm2<C-BS>" (insert-and-expand "dm") t]
-; ["Declare Module (inter.) dmi<C-BS>" (insert-and-expand "dmi") t]
-; ["Declare Module (inter. <:) dmi2<C-BS>" (insert-and-expand "dmi2") t]
- )
- ("Hints"
- "COMMAND ABBREVIATION"
- ["Hint Constructors hc<C-BS>" (insert-and-expand "hc") t]
- ["Hint Immediate hi<C-BS>" (insert-and-expand "hi") t]
- ["Hint Resolve hr<C-BS>" (insert-and-expand "hr") t]
- ["Hint Rewrite hrw<C-BS>" (insert-and-expand "hrw") t]
- ["Hint Extern he<C-BS>" (insert-and-expand "he") t]
- )
- ("Schemes"
- "COMMAND ABBREVIATION"
- ["Scheme sc<C-BS>" (insert-and-expand "sc") t]
- ["Functional Scheme fs<C-BS>" (insert-and-expand "fs") t]
- ["Functional Scheme with fsw<C-BS>" (insert-and-expand "fsw") t]
- )
- ("Notations"
- "COMMAND ABBREVIATION"
- ["infix inf<C-BS>" (insert-and-expand "inf") t]
- ["Notation (no assoc) nota<C-BS>" (insert-and-expand "nota") t]
- ["Notation (assoc) notas<C-BS>" (insert-and-expand "notas") t]
- ["Notation (no assoc, scope) notasc<C-BS>" (insert-and-expand "notasc") t]
- ["Notation (assoc, scope) notassc<C-BS>" (insert-and-expand "notassc") t]
- )
- )
-
- ("Insert term"
- "FORM ABBREVIATION"
- ["forall fo<C-BS>" (insert-and-expand "fo") t]
- ["forall1 fo1<C-BS>" (insert-and-expand "fo1") t]
- ["forall2 fo2<C-BS>" (insert-and-expand "fo2") t]
- ["forall3 fo3<C-BS>" (insert-and-expand "fo3") t]
- ["forall4 fo4<C-BS>" (insert-and-expand "fo4") t]
- ""
- ["fun f<ctrl-bacspace>" (insert-and-expand "f") t]
- ["fun1 f1<ctrl-bacspace>" (insert-and-expand "f1") t]
- ["fun2 f2<C-BS>" (insert-and-expand "f2") t]
- ["fun3 f3<C-BS>" (insert-and-expand "f3") t]
- ["fun4 f4<C-BS>" (insert-and-expand "f4") t]
- ""
- ["if then else if<C-BS>" (insert-and-expand "li") t]
- ["let in li<C-BS>" (insert-and-expand "li") t]
- ""
- ["match m<C-BS>" (insert-and-expand "m") t]
- ["match2 m2<C-BS>" (insert-and-expand "m2") t]
- ["match3 m3<C-BS>" (insert-and-expand "m3") t]
- ["match4 m4<C-BS>" (insert-and-expand "m4") t]
- )
-
- ("Insert tactic (a-f)"
- "TACTIC ABBREVIATION"
- ["absurd abs<C-BS>" (insert-and-expand "abs") t]
- ["assumption as<C-BS>" (insert-and-expand "as") t]
- ["assert ass<C-BS>" (insert-and-expand "ass") t]
- ["auto a<C-BS>" (insert-and-expand "a") t]
- ["auto with aw<C-BS>" (insert-and-expand "aw") t]
- ["auto with arith awa<C-BS>" (insert-and-expand "awa") t]
- ["autorewrite ar<C-BS>" (insert-and-expand "ar") t]
- ["cases c<C-BS>" (insert-and-expand "c") t]
- ["change ch<C-BS>" (insert-and-expand "ch") t]
- ["change in chi<C-BS>" (insert-and-expand "chi") t]
- ["change with in chwi<C-BS>" (insert-and-expand "chwi") t]
- ["constructor con<C-BS>" (insert-and-expand "con") t]
- ["congruence cong<C-BS>" (insert-and-expand "cong") t]
- ["decompose dec<C-BS>" (insert-and-expand "dec") t]
- ["decide equality deg<C-BS>" (insert-and-expand "deg") t]
- ["destruct des<C-BS>" (insert-and-expand "des") t]
- ["destruct using desu<C-BS>" (insert-and-expand "desu") t]
- ["destruct as desa<C-BS>" (insert-and-expand "desa") t]
- ["discriminate dis<C-BS>" (insert-and-expand "dis") t]
- ["eauto ea<C-BS>" (insert-and-expand "ea") t]
- ["eauto with eaw<C-BS>" (insert-and-expand "dec") t]
- ["elim e<C-BS>" (insert-and-expand "e") t]
- ["elim using elu<C-BS>" (insert-and-expand "elu") t]
- ["exists ex<C-BS>" (insert-and-expand "ex") t]
- ["field fld<C-BS>" (insert-and-expand "fld") t]
- ["firstorder fsto<C-BS>" (insert-and-expand "fsto") t]
- ["fourier fou<C-BS>" (insert-and-expand "fou") t]
- ["functional induction fi<C-BS>" (insert-and-expand "fi") t]
- )
-
- ("Insert tactic (g-z)"
- "TACTIC ABBREVIATION"
- ["generalize g<C-BS>" (insert-and-expand "g") t]
- ["induction ind<C-BS>" (insert-and-expand "ind") t]
- ["injection inj<C-BS>" (insert-and-expand "inj") t]
- ["intro i<C-BS>" (insert-and-expand "i") t]
- ["intros is<C-BS>" (insert-and-expand "is") t]
- ["intuition intu<C-BS>" (insert-and-expand "intu") t]
- ["inversion inv<C-BS>" (insert-and-expand "inv") t]
- ["omega om<C-BS>" (insert-and-expand "om") t]
- ["pose po<C-BS>" (insert-and-expand "om") t]
- ["reflexivity refl<C-BS>" (insert-and-expand "refl") t]
- ["replace rep<C-BS>" (insert-and-expand "rep") t]
- ["rewrite r<C-BS>" (insert-and-expand "r") t]
- ["rewrite in ri<C-BS>" (insert-and-expand "ri") t]
- ["rewrite <- r<<C-BS>" (insert-and-expand "rl") t]
- ["rewrite <- in ri<<C-BS>" (insert-and-expand "ril") t]
- ["set set<C-BS>" (insert-and-expand "set") t]
- ["set in hyp seth<C-BS>" (insert-and-expand "seth") t]
- ["set in goal setg<C-BS>" (insert-and-expand "setg") t]
- ["set in seti<C-BS>" (insert-and-expand "seti") t]
- ["simpl s<C-BS>" (insert-and-expand "s") t]
- ["simpl si<C-BS>" (insert-and-expand "si") t]
- ["split sp<C-BS>" (insert-and-expand "sp") t]
- ["subst su<C-BS>" (insert-and-expand "su") t]
- ["symmetry sym<C-BS>" (insert-and-expand "sym") t]
- ["transitivity trans<C-BS>" (insert-and-expand "trans") t]
- ["trivial t<C-BS>" (insert-and-expand "t") t]
- ["tauto ta<C-BS>" (insert-and-expand "ta") t]
- ["unfold u<C-BS>" (insert-and-expand "u") t]
- )
-
- ["What are those highlighted chars??" (holes-short-doc) t]
- ("holes"
- "make a hole active click on it"
- "disable a hole click on it (button 2)"
- "destroy a hole click on it (button 3)"
- "make a hole with mouse C-M-select"
- ["make a hole at point C-M-h" (set-make-active-hole) t]
- ["make selection a hole C-M-h" (set-make-active-hole) t]
- ["replace active hole by selection C-M-y" (replace-update-active-hole) t]
- "replace active hole with mouse C-M-Shift select"
- ["jump to active hole M-return" (set-point-next-hole-destroy) t]
- ["forget all holes in this buffer" (clear-all-buffer-holes) t]
- ["What are those holes?" (holes-short-doc) t]
- )
- ["expand abbrev at point" expand-abbrev t]
- ["list abbrevs" list-abbrevs t]
- ["Print..." coq-Print t]
- ["Check..." coq-Check t]
- ["Hints" coq-PrintHint t]
- ["Show ith goal..." coq-Show t]
- ["Search isos/pattern..." coq-SearchIsos t]
- ["3 buffers view" coq-three-b t]
- ["Compile" coq-Compile t] ))
+;; ----- coq specific menu is defined in coq-abbrev.el
+
+(cond
+ (coq-version-is-V8 (require 'coq-abbrev))
+ (t (require 'coq-abbrev-V7))
+ )