diff options
author | glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-08-06 14:21:26 +0000 |
---|---|---|
committer | glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-08-06 14:21:26 +0000 |
commit | 99ceb8c7df67a37330820e3e6fbb4a3ccab2a9a5 (patch) | |
tree | f9418c2845f990ff3afd1d82d4b6df234a9bf69e /theories | |
parent | 1fc6c06dc34462f3df80f4c38aafd3408ef37578 (diff) |
Add lemmas on lists: nth_default_eq, map_nth_error
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11310 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r-- | theories/Lists/List.v | 14 |
1 files changed, 13 insertions, 1 deletions
diff --git a/theories/Lists/List.v b/theories/Lists/List.v index aabf9e379..c873338ac 100644 --- a/theories/Lists/List.v +++ b/theories/Lists/List.v @@ -402,6 +402,12 @@ Section Elts. | None => default end. + Lemma nth_default_eq : + forall n l (d:A), nth_default d l n = nth n l d. + Proof. + unfold nth_default; induction n; intros [ | ] ?; simpl; auto. + Qed. + Lemma nth_In : forall (n:nat) (l:list A) (d:A), n < length l -> In (nth n l d) l. @@ -1056,7 +1062,13 @@ Section Map. Proof. induction l; simpl map; destruct n; firstorder. Qed. - + + Lemma map_nth_error : forall n l d, + nth_error l n = Some d -> nth_error (map l) n = Some (f d). + Proof. + induction n; intros [ | ] ? Heq; simpl in *; inversion Heq; auto. + Qed. + Lemma map_app : forall l l', map (l++l') = (map l)++(map l'). Proof. |