Skip to content
Snippets Groups Projects
Commit c5676b11 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Shorten proof.

parent b55715d3
No related branches found
No related tags found
No related merge requests found
......@@ -80,11 +80,7 @@ Section seq.
Lemma Forall_seq (P : nat Prop) i n :
Forall P (seq i n) j, i j < i + n P j.
Proof.
rewrite Forall_lookup. split.
- intros H j [??]. apply (H (j - i)), lookup_seq. lia.
- intros H j x [-> ?]%lookup_seq. auto with lia.
Qed.
Proof. rewrite Forall_forall. setoid_rewrite elem_of_seq. auto with lia. Qed.
End seq.
(** ** Properties of the [seqZ] function *)
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment