aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2015-01-05 13:15:49 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2015-01-05 13:15:49 +0000
commit3a63958bc6466e283e0aec083229df20c8c2dd69 (patch)
treeebae559231e40bbec13e4513c0517595b4c88c53 /coq/ex
parentd2c699c9690ab2479647024c5326985bdac2a142 (diff)
Fixing indentation of pending curly braces.
Diffstat (limited to 'coq/ex')
-rw-r--r--coq/ex/indent.v54
1 files changed, 53 insertions, 1 deletions
diff --git a/coq/ex/indent.v b/coq/ex/indent.v
index c146f61d..edf1a536 100644
--- a/coq/ex/indent.v
+++ b/coq/ex/indent.v
@@ -267,7 +267,7 @@ End X.
Require Import Morphisms.
Generalizable All Variables.
-Open Local Scope signature_scope.
+Local Open Scope signature_scope.
Require Import RelationClasses.
Module TC.
@@ -344,3 +344,55 @@ Section SET.
end.
End SET.
+
+Module curlybracesatend.
+
+ Lemma foo: forall n: nat,
+ exists m:nat,
+ m = n + 1.
+ Proof.
+ intros n.
+ destruct n. {
+ exists 1.
+ reflexivity. }
+ exists (S (S n)).
+ simpl.
+ rewrite NPeano.Nat.add_1_r.
+ reflexivity.
+ Qed.
+
+ Lemma foo2: forall n: nat,
+ exists m:nat, (* This is strange compared to the same line in the previous lemma *)
+ m = n + 1.
+ Proof.
+ intros n.
+ destruct n. {
+ exists 1.
+ reflexivity. }
+
+ exists (S (S n)).
+ simpl.
+ rewrite NPeano.Nat.add_1_r.
+ reflexivity.
+ Qed.
+
+ Lemma foo3: forall n: nat,
+ exists m:nat, (* This is strange compared to the same line in the previous lemma *)
+ m = n + 1.
+ Proof.
+ intros n. cut (n = n). {
+ destruct n. {
+ exists 1.
+ reflexivity. } {
+ exists (S (S n)).
+ simpl.
+ rewrite NPeano.Nat.add_1_r.
+ reflexivity. }
+ }
+ idtac.
+ reflexivity.
+ Qed.
+
+
+End curlybracesatend.
+