aboutsummaryrefslogtreecommitdiff
path: root/plugins
diff options
context:
space:
mode:
authoraspiwack2013-11-02 15:35:08 +0000
committeraspiwack2013-11-02 15:35:08 +0000
commitd45d2232e9dae87162a841a21cc708769259a184 (patch)
treeea4ddfc4c74f8b3fa60144bd7c80d9ec72ff5558 /plugins
parent75a1dffa93afa21a686883ba20dc8d2988a97b14 (diff)
Cleanup of comments.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16976 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins')
-rw-r--r--plugins/decl_mode/g_decl_mode.ml44
1 files changed, 1 insertions, 3 deletions
diff --git a/plugins/decl_mode/g_decl_mode.ml4 b/plugins/decl_mode/g_decl_mode.ml4
index a4f8641ddb..a3a2b25e44 100644
--- a/plugins/decl_mode/g_decl_mode.ml4
+++ b/plugins/decl_mode/g_decl_mode.ml4
@@ -8,8 +8,6 @@
(*i camlp4deps: "grammar/grammar.cma" i*)
-(* arnaud: veiller à l'aspect tutorial des commentaires *)
-
open Compat
open Pp
open Tok
@@ -36,7 +34,7 @@ let pr_goal gs =
str "============================" ++ fnl () ++
thesis ++ str " " ++ pc) ++ fnl ()
-(* arnaud: rebrancher ça
+(* arnaud: rebrancher ça ?
let pr_open_subgoals () =
let p = Proof_global.give_me_the_proof () in
let { Evd.it = goals ; sigma = sigma } = Proof.V82.subgoals p in