aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/seq.v
diff options
context:
space:
mode:
authorGeorges Gonthier2019-05-08 09:38:02 +0200
committerGitHub2019-05-08 09:38:02 +0200
commit51b9988f608625c60184dbe90133d64cdaa2a1f9 (patch)
tree5315fbaebdbeca10f6a9ffba448ea424d16252b3 /mathcomp/ssreflect/seq.v
parent02830d7cf24f9198d5e7cb81843d6ca5cb69f68a (diff)
parent6c4382c69e72b81fb7e81b0b753e5d3c83b1064a (diff)
Merge pull request #344 from soraros/ssrnat-remove-arith-lemmas
remove dependence on Arith lemmas
Diffstat (limited to 'mathcomp/ssreflect/seq.v')
-rw-r--r--mathcomp/ssreflect/seq.v5
1 files changed, 2 insertions, 3 deletions
diff --git a/mathcomp/ssreflect/seq.v b/mathcomp/ssreflect/seq.v
index 3685c23..76acaca 100644
--- a/mathcomp/ssreflect/seq.v
+++ b/mathcomp/ssreflect/seq.v
@@ -497,7 +497,7 @@ Lemma all_nseqb (b : bool) x : all (nseq b x) = b ==> a x.
Proof. by rewrite all_nseq eqb0 implybE. Qed.
Lemma find_nseq n x : find (nseq n x) = ~~ a x * n.
-Proof. by elim: n => //= n ->; case: (a x). Qed.
+Proof. by elim: n => /= [|n ->]; case: (a x). Qed.
Lemma nth_find s : has s -> a (nth s (find s)).
Proof. by elim: s => //= x s IHs; case Hx: (a x). Qed.
@@ -928,7 +928,7 @@ Proof. by rewrite -size_eq0 size_filter has_count lt0n. Qed.
Fixpoint mem_seq (s : seq T) :=
if s is y :: s' then xpredU1 y (mem_seq s') else xpred0.
-Definition seq_eqclass := seq T.
+Definition seq_eqclass := seq T.
Identity Coercion seq_of_eqclass : seq_eqclass >-> seq.
Coercion pred_of_seq (s : seq_eqclass) : {pred T} := mem_seq s.
@@ -3068,4 +3068,3 @@ Notation perm_uniq :=
deprecate perm_uniq eq_uniq T s1 s2 eq_sz12 eq_s12)
_ _ _)
(only parsing).
-