aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/TODO
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <Pierre.Courtieu@cnam.fr>2015-09-29 10:41:48 +0200
committerGravatar Pierre Courtieu <Pierre.Courtieu@cnam.fr>2015-09-29 13:22:21 +0200
commit8f984a7272de74d8a88cffcef2ca6160d710b335 (patch)
treeb229a2ef91bf3dede68941dac526c67a10324b2a /coq/TODO
parentbb5ea22b62d337eebb04aa17ca9bd0e6893b90e4 (diff)
Cleaned TODO file in coq/.
Diffstat (limited to 'coq/TODO')
-rw-r--r--coq/TODO47
1 files changed, 18 insertions, 29 deletions
diff --git a/coq/TODO b/coq/TODO
index ba8b310e..c503dc24 100644
--- a/coq/TODO
+++ b/coq/TODO
@@ -7,47 +7,36 @@ eval x in y : commande
unfold x in y : tactique
-** important: Have an option for indenting style:
+** important: fix indention of definitions:
Current behavior:
-Lemma foo: forall x,
- f x = 0.
+function foo bar1 bar2
+ bar3
-and:
+Should be
-functionfoo bar1 bar2
- bar3
+function foo bar1 bar2
+ <>bar3
+(<> length parameterized by coq-smie-after-bolp-indentation)
+or
+function foo bar1 bar2
+ bar3
-Commonly used behavior:
+depending on an option (coq-indent-box-style).
-Lemma foo: forall x,
- f x = 0.
-
-and
-
-functionfoo bar1 bar2
- bar3
-
-
-** (less important) Indent correctly this:
-
-Proof with auto.
- intro.
-
-instead of:
-
-Proof with auto.
- intro.
+** Fix indentation of ;
+Current behavior:
-Workaroud for the moment, write the script like this:
+idtac ;
+ idtac.
-Proof with
- auto.
- intro.
+but:
+idtac; idtac;
+idtac.
** dealing with several project files.