aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/coq/indent.v
diff options
context:
space:
mode:
Diffstat (limited to 'etc/coq/indent.v')
-rw-r--r--etc/coq/indent.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/etc/coq/indent.v b/etc/coq/indent.v
index 46839715..be27f9ef 100644
--- a/etc/coq/indent.v
+++ b/etc/coq/indent.v
@@ -64,5 +64,5 @@ Theorem p : forall (P : Prop), P -> P.
Proof.
try (simpl
in *).
- intros P H. apply H.
+ intros P H. apply H. (* da: shouldn't we outdent again here? *)
Qed.