aboutsummaryrefslogtreecommitdiffhomepage
path: root/ide/coq_commands.ml
diff options
context:
space:
mode:
authorGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-04 15:30:44 +0000
committerGravatar coq <coq@85f007b7-540e-0410-9357-904b9bb8a0f7>2004-02-04 15:30:44 +0000
commit836276d44d2bad23c2dbc8ee66a74c7f71856a5f (patch)
tree1d3325b539b6635979e813019be9f6da53a8dbc5 /ide/coq_commands.ml
parentcf45343a65cc1c84dc5c521a34c6c112fb7b5fe7 (diff)
search window
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@5288 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'ide/coq_commands.ml')
-rw-r--r--ide/coq_commands.ml1
1 files changed, 1 insertions, 0 deletions
diff --git a/ide/coq_commands.ml b/ide/coq_commands.ml
index 86b7744c9..640d1c383 100644
--- a/ide/coq_commands.ml
+++ b/ide/coq_commands.ml
@@ -120,6 +120,7 @@ let commands = [
"Remove Printing Let";
"Require";
"Require Export";
+ "Require Import";
(* "Reset"; *)
"Reset Extraction Inline";
(* "Reset Initial"; *)