aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coq_commands.ml
diff options
context:
space:
mode:
authorGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-30 09:56:20 +0000
committerGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-12-30 09:56:20 +0000
commitb2c056c881dcb3035158ab177f2363c1527df397 (patch)
tree7e13f45a340cc82721a7ca4962ea4852d287157b /ide/coq_commands.ml
parenta08c4181d9580aeaf4d52a382a5c84a4040d5995 (diff)
ameliorations coqide
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5161 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'ide/coq_commands.ml')
-rw-r--r--ide/coq_commands.ml197
1 files changed, 193 insertions, 4 deletions
diff --git a/ide/coq_commands.ml b/ide/coq_commands.ml
index 7173bfc2f..86b7744c9 100644
--- a/ide/coq_commands.ml
+++ b/ide/coq_commands.ml
@@ -38,9 +38,9 @@ let commands = [
"Defined.";
"Definition";
"Derive Dependent Inversion";
- "Derive Dependent Inversion_clear";
+ "Derive Dependent Inversion__clear";
"Derive Inversion";
- "Derive Inversion_clear";
+ "Derive Inversion__clear";
(* "Drop"; *)];
["End";
"End Silent.";
@@ -141,7 +141,7 @@ let commands = [
"Section";
"Set Extraction AutoInline";
"Set Extraction Optimize";
- "Set Hyps_limit";
+ "Set Hyps__limit";
"Set Implicit Arguments";
"Set Printing Coercion";
"Set Printing Coercions";
@@ -174,7 +174,7 @@ let commands = [
"Unfocus";
"Unset Extraction AutoInline";
"Unset Extraction Optimize";
- "Unset Hyps_limit";
+ "Unset Hyps__limit";
"Unset Implicit Arguments";
"Unset Printing Coercion";
"Unset Printing Coercions";
@@ -240,3 +240,192 @@ let state_preserving = [
"Test Printing Synth";
"Test Printing Wildcard";
]
+
+
+let tactics =
+ [
+ [
+ "abstract";
+ "absurd";
+ "apply";
+ "apply __ with";
+ "assert";
+ "assumption.";
+ "auto.";
+ "auto with";
+ "autorewrite";
+ ];
+
+ [
+ "case";
+ "case __ with";
+ "cbv";
+ "change";
+ "change __ in";
+ "clear";
+ "clearbody";
+ "compare";
+ "compute";
+ "congruence";
+ "constructor";
+ "constructor __ with";
+ "contradiction.";
+ "cut";
+ "cutrewrite";
+ ];
+
+ [
+ "decide equality.";
+ "decompose";
+ "decompose record";
+ "decompose sum";
+ "dependent inversion";
+ "dependent inversion __ with";
+ "dependent inversion__clear";
+ "dependent inversion__clear __ with";
+ "dependent rewrite ->";
+ "dependent rewrite <-";
+ "destruct";
+ "discriminate.";
+ "discriminate";
+ "discrR.";
+ "do";
+ "double induction";
+ ];
+
+ [
+ "eapply";
+ "eauto.";
+ "eauto with";
+ "elim";
+ "elim __ using";
+ "elim __ with";
+ "elimtype";
+ "exact";
+ "exists";
+ ];
+
+ [
+ "fail.";
+ "field.";
+ "first";
+ "firstorder.";
+ "firstorder";
+ "firstorder using";
+ "firstorder with";
+ "fold";
+ "fourier.";
+ "functional induction";
+ ];
+
+ [
+ "generalize";
+ "generalize dependent";
+ ];
+
+ [
+ "hnf";
+ ];
+
+ [
+ "idtac.";
+ "induction";
+ "info";
+ "injection";
+ "intro";
+ "intro after";
+ "intro __ after";
+ "intros";
+ "intros.";
+ "intros";
+ "intros <pattern> ";
+ "intros until";
+ "intuition.";
+ "intuition";
+ "inversion";
+ "inversion __ in";
+ "inversion __ using";
+ "inversion __ using __ in";
+ "inversion__clear";
+ "inversion__clear __ in";
+ ];
+
+ [
+ "jp <n>";
+ "jp.";
+ ];
+
+ [
+ "lapply";
+ "lazy";
+ "left";
+ ];
+
+ [
+ "move __ after";
+ ];
+
+ [
+ "omega";
+ ];
+
+ [
+ "pattern";
+ "pose";
+ "progress";
+ ];
+
+ [
+ "quote";
+ ];
+
+ [
+ "red.";
+ "red in";
+ "refine";
+ "reflexivity.";
+ "rename __ into";
+ "repeat";
+ "replace __ with";
+ "rewrite";
+ "rewrite __ in";
+ "rewrite ->";
+ "rewrite -> __ in";
+ "rewrite <-";
+ "rewrite <- __ in";
+ "right.";
+ "ring.";
+ ];
+
+ [
+ "set";
+ "setoid__replace";
+ "setoid__rewrite";
+ "simpl.";
+ "simpl __ in";
+ "simple destruct";
+ "simple induction";
+ "simple inversion";
+ "simplify__eq";
+ "solve";
+ "split.";
+ "split__Rabs.";
+ "split__Rmult.";
+ "subst";
+ "symmetry.";
+ ];
+
+ [
+ "tauto.";
+ "transitivity";
+ "trivial.";
+ "try";
+ ];
+
+ [
+ "unfold";
+ "unfold __ in";
+ ];
+]
+
+