aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2012-06-08 11:40:43 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2012-06-08 11:40:43 +0000
commit7ecdbfb869b5e9d6cd75c610ef125823b3727071 (patch)
tree39fca488052f051211f00ca7e3c0f15a809c6a9c /coq/ex
parent3d730bd7c3b25afdcc4a14ddc7c79b9c8ec37fd3 (diff)
Indentation is a bit more accurate.
Diffstat (limited to 'coq/ex')
-rw-r--r--coq/ex/indent.v49
1 files changed, 28 insertions, 21 deletions
diff --git a/coq/ex/indent.v b/coq/ex/indent.v
index 80b7313b..72f1d4f6 100644
--- a/coq/ex/indent.v
+++ b/coq/ex/indent.v
@@ -9,6 +9,13 @@ 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.
+
+
Lemma toto:nat.
Proof.
{{
@@ -96,8 +103,8 @@ Module M1'.
destruct n.
{
idtac;[
- auto
- ].
+ auto
+ ].
}
auto.
}
@@ -150,16 +157,16 @@ End M1''.
Record rec:Set := {
- fld1:nat;
- fld2:nat;
- fld3:bool
- }.
+ fld1:nat;
+ fld2:nat;
+ fld3:bool
+ }.
Class cla {X:Set}:Set := {
- cfld1:nat;
- cld2:nat;
- cld3:bool
- }.
+ cfld1:nat;
+ cld2:nat;
+ cld3:bool
+ }.
@@ -194,12 +201,12 @@ Module X.
intros r.
{{
idtac;
- exists
- {|
- fld1:=r.(fld2);
- fld2:=r.(fld1);
- fld3:=false
- |}.
+ exists
+ {|
+ fld1:=r.(fld2);
+ fld2:=r.(fld1);
+ fld3:=false
+ |}.
(* ltac *)
match goal with
| _:rec |- ?a /\ ?b => split
@@ -226,17 +233,17 @@ Module foo.
Proof.
firstorder.
Qed.
-
-
+
+
Program Fixpoint f (x:nat) {struct x} : nat :=
match x with
| 0 => 0
| S y => S (f y)
end.
-
+
Program Instance all_iff_morphism {A : Type} :
Proper (pointwise_relation A iff ==> iff) (@all A).
-
+
Next Obligation.
Proof.
unfold pointwise_relation, all in * .
@@ -255,7 +262,7 @@ Section SET.
Require Import Program.
-
+
Definition eq_n : forall A n (v:Vector.t A n) n', n=n' -> Vector.t A n'.
Proof.
intros A n v n' H.