aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/indent.v
diff options
context:
space:
mode:
authorGravatar Pierre Courtieu <courtieu@lri.fr>2011-06-17 17:03:16 +0000
committerGravatar Pierre Courtieu <courtieu@lri.fr>2011-06-17 17:03:16 +0000
commit2c80f2c38e3d9bb7e9bf6b7e0b304a87e42a60a0 (patch)
tree07587f08662852627e8b186366f2c9637c704468 /coq/ex/indent.v
parent6529a8dfa67fa4e1751f2ae8d8ee7398efd4d8d6 (diff)
oops, undo last commit.
Diffstat (limited to 'coq/ex/indent.v')
-rw-r--r--coq/ex/indent.v13
1 files changed, 11 insertions, 2 deletions
diff --git a/coq/ex/indent.v b/coq/ex/indent.v
index 38240988..8ca17cae 100644
--- a/coq/ex/indent.v
+++ b/coq/ex/indent.v
@@ -7,8 +7,7 @@ Require Import Arith.
Lemma L : forall x:nat , nat_iter x (A:=nat) (plus 2) 0 >= x.
Proof.
- intros x;
- toto.
+ induction x;simpl;intros;auto with arith.
Qed.
Function div2 (n : nat) {struct n}: nat :=
@@ -167,5 +166,15 @@ Module foo.
| 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 * .
+ intro.
+ intros y H.
+ intuition ; specialize (H x0) ; intuition.
+ Qed.
+
End foo.