aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/indent.v
diff options
context:
space:
mode:
authorGravatar Stefan Monnier <monnier@iro.umontreal.ca>2014-06-03 02:51:24 +0000
committerGravatar Stefan Monnier <monnier@iro.umontreal.ca>2014-06-03 02:51:24 +0000
commit67f4332c9e802a0d272ac0670515d98d16cfebb4 (patch)
tree5194cf6085f03a400b521a8806039099b304a166 /coq/ex/indent.v
parent2ddd31c9984044e16a5bf5e1745fe9d33f8255a4 (diff)
Rename coq-smie-lexer.el to coq-smie.el.
Diffstat (limited to 'coq/ex/indent.v')
-rw-r--r--coq/ex/indent.v17
1 files changed, 12 insertions, 5 deletions
diff --git a/coq/ex/indent.v b/coq/ex/indent.v
index c574f715..b524d956 100644
--- a/coq/ex/indent.v
+++ b/coq/ex/indent.v
@@ -9,12 +9,19 @@ Record a : Type := make_a {
aa : nat
}.
-Inductive test : nat -> Prop :=
-| C1 : forall n, test n
-| C2 : forall n, test n
-| C3 : forall n, test n
-| C4 : forall n, test n.
+{
+ Inductive test : nat -> Prop :=
+ | C1 : forall n, test n
+ | C2 : forall n, test n
+ | C3 : forall n, test n
+ | C4 : forall n, test n.
+ Inductive test2 : nat -> Prop
+ := C1 : forall n, test n
+ | C2 : forall n, test n
+ | C3 : forall n, test n
+ | C4 : forall n, test n.
+}
Lemma toto:nat.
Proof.