aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2011-07-08 13:08:04 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2011-07-08 13:08:04 +0000
commit7238c3d7555b01d814666e12ec24e87a1ed154c5 (patch)
treedf3b5854d8e069ee486ddc451fbb8d315150c3b6 /coq/ex
parent6d8943cef5aba5364adafd029b7d74a5a7f8391e (diff)
Fixing the scripting of new subproof script parenthesizing ({ and }).
Diffstat (limited to 'coq/ex')
-rw-r--r--coq/ex/indent.v27
1 files changed, 21 insertions, 6 deletions
diff --git a/coq/ex/indent.v b/coq/ex/indent.v
index f2ba0f9d..3e1b60ed 100644
--- a/coq/ex/indent.v
+++ b/coq/ex/indent.v
@@ -16,11 +16,12 @@ Proof.
}}
Qed.
-
-Lemma L : forall x:nat , nat_iter x (A:=nat) (plus 2) 0 >= x.
-Proof.
- induction x;simpl;intros;auto with arith.
-Qed.
+Module Y.
+ Lemma L : forall x:nat , nat_iter x (A:=nat) (plus 2) 0 >= x.
+ Proof with auto with arith.
+ induction x;simpl;intros...
+ Qed.
+End Y.
Function div2 (n : nat) {struct n}: nat :=
match n with
@@ -86,7 +87,7 @@ Module M1'.
].
}
auto.
- }
+ }
Qed.
{destruct n.
{
@@ -97,6 +98,20 @@ Module M1'.
End M2'.
End M1'.
+
+Module M1''.
+ Module M2''.
+ Lemma l7: forall n:nat, n = n.
+ destruct n.
+ { auto. }
+ { destruct n.
+ { idtac; [ auto ]. }
+ auto. }
+ Qed.
+ End M2''.
+End M1''.
+
+
Record rec:Set := {
fld1:nat;
fld2:nat;