diff options
author | notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-09-01 11:04:44 +0000 |
---|---|---|
committer | notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2006-09-01 11:04:44 +0000 |
commit | e81d7ccf99ac02476fb289042b7c653251160abf (patch) | |
tree | 1a29bb9b90fdd6cdf15bf9b82aed0291f772d979 /theories | |
parent | 81ed88d7722052181aa4106ebbeda8952068ffbc (diff) |
Indentation + typo
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9104 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r-- | theories/Lists/List.v | 4 |
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Lists/List.v b/theories/Lists/List.v index 67b8e4398..cd6ce35cf 100644 --- a/theories/Lists/List.v +++ b/theories/Lists/List.v @@ -1336,14 +1336,14 @@ End Fold_Right_Recursor. rewrite IHl; simpl; auto. Qed. - Lemma split_lenght_l : forall (l:list (A*B)), + Lemma split_length_l : forall (l:list (A*B)), length (fst (split l)) = length l. Proof. induction l; simpl; auto. destruct a; destruct (split l); simpl; auto. Qed. - Lemma split_lenght_r : forall (l:list (A*B)), + Lemma split_length_r : forall (l:list (A*B)), length (snd (split l)) = length l. Proof. induction l; simpl; auto. |