aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/TODO
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2011-11-10 12:12:32 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2011-11-10 12:12:32 +0000
commita2007818ad381dad0f489cbea8817df401e57c9f (patch)
tree2ce5ca251c025c5418d0c465a0f6d01a3486fec4 /coq/TODO
parentfc7465f44f3c02c187502de42b4111837b4e960a (diff)
fixed some small bugs in coq indentation smie code.
Diffstat (limited to 'coq/TODO')
-rw-r--r--coq/TODO51
1 files changed, 51 insertions, 0 deletions
diff --git a/coq/TODO b/coq/TODO
new file mode 100644
index 00000000..09140d77
--- /dev/null
+++ b/coq/TODO
@@ -0,0 +1,51 @@
+-*- outline -*-
+
+** important: deal with different levels of the "in" keyword
+
+let x := y in : expression
+eval x in y : commande
+unfold x in y : tactique
+
+
+** important: Have an option for indenting style:
+
+Current behavior:
+
+Lemma foo: forall x,
+ f x = 0.
+
+and:
+
+functionfoo bar1 bar2
+ bar3
+
+
+Commonly used behavior:
+
+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.
+
+
+Workaroud for the moment, write the script like this:
+
+Proof with
+ auto.
+ intro.
+
+