Skip to content
Snippets Groups Projects
Commit f3d1c76f authored by Björn Brandenburg's avatar Björn Brandenburg
Browse files

do not rely on simpl_sum_const tactic

parent f7550c93
No related branches found
No related tags found
No related merge requests found
......@@ -164,8 +164,8 @@ Section UnitService.
Proof.
unfold service_during; intros t delta.
apply leq_trans with (n := \sum_(t <= t0 < t + delta) 1);
last by simpl_sum_const; rewrite addKn leqnn.
by apply: leq_sum => t' _; apply: service_at_most_one.
last by rewrite sum_of_ones.
by apply: leq_sum => t' _; apply: service_at_most_one.
Qed.
Section ServiceIsAStepFunction.
......
......@@ -248,7 +248,7 @@ Section ExtraLemmas.
\sum_(t <= x < t + Δ) 1 = Δ.
Proof.
intros.
simpl_sum_const.
rewrite big_const_nat iter_addn_0 mul1n.
rewrite addnC -addnBA; last by done.
by rewrite subnn addn0.
Qed.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment