Skip to content
Snippets Groups Projects
Commit 3ab704f7 authored by Sergey Bozhko's avatar Sergey Bozhko :eyes:
Browse files

add lemmas to util/div_mod

Added a few lemmas to util/div_mod that are needed for POET
parent 84b68e3e
No related branches found
No related tags found
1 merge request!158Add lemmas to util/div_mod
Pipeline #54856 passed with warnings
Require Export prosa.util.nat prosa.util.subadditivity. Require Export prosa.util.nat prosa.util.subadditivity.
From mathcomp Require Export ssreflect ssrbool eqtype ssrnat seq fintype bigop div ssrfun. From mathcomp Require Export ssreflect ssrbool eqtype ssrnat seq fintype bigop div ssrfun.
(** First, we define functions [div_floor] and [div_ceil], which are (** Additional lemmas about [divn] and [modn]. *)
divisions rounded down and up, respectively. *) Section DivMod.
Definition div_floor (x y : nat) : nat := x %/ y.
Definition div_ceil (x y : nat) := if y %| x then x %/ y else (x %/ y).+1.
(** We start with an observation that [div_ceil 0 b] is equal to (** First, we show that if [t1 / h] is equal to [t2 / h] and [t1 <= t2],
[0] for any [b]. *) then [t1 mod h] is bounded by [t2 mod h]. *)
Lemma div_ceil0: Lemma eqdivn_leqmodn :
forall b, div_ceil 0 b = 0. forall t1 t2 h,
Proof. t1 <= t2 ->
intros b; unfold div_ceil. t1 %/ h = t2 %/ h ->
by rewrite dvdn0; apply div0n. t1 %% h <= t2 %% h.
Qed. Proof.
intros * LT EQ.
destruct (posnP h) as [Z | POSh].
{ by subst; rewrite !modn0. }
{ have EX: exists k, t1 + k = t2.
{ exists (t2 - t1); ssrlia. }
destruct EX as [k EX]; subst t2; clear LT.
rewrite modnD //; replace (h <= t1 %% h + k %% h) with false; first by ssrlia.
symmetry; apply/negP/negP; rewrite -ltnNge.
symmetry in EQ; rewrite divnD // in EQ; move: EQ => /eqP.
rewrite -{2}[t1 %/ h]addn0 -addnA eqn_add2l addn_eq0 => /andP [_ /eqP Z2].
by move: Z2 => /eqP; rewrite eqb0 -ltnNge.
}
Qed.
(** Next, we show that, given two positive integers [a] and [b], (** Given two natural numbers [x] and [y], the fact that
[div_ceil a b] is also positive. *) [x / y < (x + 1) / y] implies that [y] divides [x + 1]. *)
Lemma div_ceil_gt0: Lemma ltdivn_dvdn :
forall a b, forall x y,
a > 0 -> b > 0 -> x %/ y < (x + 1) %/ y ->
div_ceil a b > 0. y %| (x + 1).
Proof. Proof.
intros a b POSa POSb. intros ? ? LT.
unfold div_ceil. destruct (posnP y) as [Z | POS]; first by subst y.
destruct (b %| a) eqn:EQ; last by done. move: LT; rewrite divnD // -addn1 -addnA leq_add2l addn_gt0 => /orP [ONE | LE].
by rewrite divn_gt0 //; apply dvdn_leq. { by destruct y as [ | []]. }
Qed. { rewrite lt0b in LE.
destruct (leqP 2 y) as [LT2 | GE2]; last by destruct y as [ | []].
(** We show that [div_ceil] is monotone with respect to the first clear POS; rewrite [1 %% _]modn_small // in LE.
argument. *) move: LE; rewrite leq_eqVlt => /orP [/eqP EQ | LT].
Lemma div_ceil_monotone1: { rewrite [x](divn_eq x y) -addnA -EQ; apply dvdn_add.
forall d m n, - by apply dvdn_mull, dvdnn.
m <= n -> div_ceil m d <= div_ceil n d. - by apply dvdnn.
Proof. }
move => d m n LEQ. { by move: LT; rewrite -addn1 leq_add2r leqNgt ltn_pmod //; ssrlia. }
rewrite /div_ceil. }
have LEQd: m %/ d <= n %/ d by apply leq_div2r. Qed.
destruct (d %| m) eqn:Mm; destruct (d %| n) eqn:Mn => //; first by ssrlia.
rewrite ltn_divRL //. (** We prove an auxiliary lemma allowing us to change the order of
apply ltn_leq_trans with m => //. operations [_ + 1] and [_ %% h]. *)
move: (leq_trunc_div m d) => LEQm. Lemma addn1_modn_commute :
destruct (ltngtP (m %/ d * d) m) => //. forall x h,
move: e => /eqP EQ; rewrite -dvdn_eq in EQ. h > 0 ->
by rewrite EQ in Mm. x %/ h = (x + 1) %/ h ->
Qed. (x + 1) %% h = x %% h + 1 .
Proof.
intros x h POS EQ.
rewrite !addnS !addn0.
rewrite addnS divnS // addn0 in EQ.
destruct (h %| x.+1) eqn:DIV ; rewrite /= in EQ; first by ssrlia.
by rewrite modnS DIV.
Qed.
(** We show that for any two integers [a] and [b], (** We show that the fact that [x / h = (x + y) / h] implies that
[a] is less than [a %/ b * b + b] given that [b] is positive. *) [h] is larder than [x mod h + y mod h]. *)
Lemma div_floor_add_g: Lemma addmod_le_mod :
forall a b, forall x y h,
b > 0 -> h > 0 ->
a < a %/ b * b + b. x %/ h = (x + y) %/ h ->
Proof. h > x %% h + y %% h.
intros * POS. Proof.
specialize (divn_eq a b) => DIV. intros x y h POS EQ.
rewrite [in X in X < _]DIV. move: EQ => /eqP; rewrite divnD // -{1}[x %/ h]addn0 -addnA eqn_add2l eq_sym addn_eq0 => /andP [/eqP Z1 /eqP Z2].
rewrite ltn_add2l. by move: Z2 => /eqP; rewrite eqb0 -ltnNge => LT.
by apply ltn_pmod. Qed.
Qed.
End DivMod.
(** In this section, we define notions of [div_floor] and [div_ceil]
and prove a few basic lemmas. *)
Section DivFloorCeil.
(** Given [T] and [Δ] such that [Δ >= T > 0], we show that [div_ceil Δ T] (** We define functions [div_floor] and [div_ceil], which are
is strictly greater than [div_ceil (Δ - T) T]. *) divisions rounded down and up, respectively. *)
Lemma leq_div_ceil_add1: Definition div_floor (x y : nat) : nat := x %/ y.
forall Δ T, Definition div_ceil (x y : nat) := if y %| x then x %/ y else (x %/ y).+1.
T > 0 -> Δ >= T ->
div_ceil (Δ - T) T < div_ceil Δ T.
Proof.
intros * POS LE. rewrite /div_ceil.
have lkc: (Δ - T) %/ T < Δ %/ T.
{ rewrite divnBr; last by auto.
rewrite divnn POS.
rewrite ltn_psubCl //; try ssrlia.
by rewrite divn_gt0.
}
destruct (T %| Δ) eqn:EQ1.
{ have divck: (T %| Δ) -> (T %| (Δ - T)) by auto.
apply divck in EQ1 as EQ2.
rewrite EQ2; apply lkc.
}
by destruct (T %| Δ - T) eqn:EQ, (T %| Δ) eqn:EQ3; auto.
Qed.
(** We start with an observation that [div_ceil 0 b] is equal to [0]
for any [b]. *)
Lemma div_ceil0:
forall b, div_ceil 0 b = 0.
Proof.
intros b; unfold div_ceil.
by rewrite dvdn0; apply div0n.
Qed.
(** We show that the division with ceiling by a constant [T] is a subadditive function. *) (** Next, we show that, given two positive integers [a] and [b],
Lemma div_ceil_subadditive: [div_ceil a b] is also positive. *)
forall T, subadditive (div_ceil^~T). Lemma div_ceil_gt0:
Proof. forall a b,
move=> T ab a b SUM. a > 0 -> b > 0 ->
rewrite -SUM. div_ceil a b > 0.
destruct (T %| a) eqn:DIVa, (T %| b) eqn:DIVb. Proof.
- have DIVab: T %| a + b by apply dvdn_add. intros a b POSa POSb.
by rewrite /div_ceil DIVa DIVb DIVab divnDl. unfold div_ceil.
- have DIVab: T %| a+b = false by rewrite -DIVb; apply dvdn_addr. destruct (b %| a) eqn:EQ; last by done.
by rewrite /div_ceil DIVa DIVb DIVab divnDl //=; ssrlia. by rewrite divn_gt0 //; apply dvdn_leq.
- have DIVab: T %| a+b = false by rewrite -DIVa; apply dvdn_addl. Qed.
by rewrite /div_ceil DIVa DIVb DIVab divnDr //=; ssrlia.
- destruct (T %| a + b) eqn:DIVab. (** We show that [div_ceil] is monotone with respect to the first
+ rewrite /div_ceil DIVa DIVb DIVab. argument. *)
apply leq_trans with (a %/ T + b %/T + 1); last by ssrlia. Lemma div_ceil_monotone1:
by apply leq_divDl. forall d m n,
+ rewrite /div_ceil DIVa DIVb DIVab. m <= n -> div_ceil m d <= div_ceil n d.
apply leq_ltn_trans with (a %/ T + b %/T + 1); last by ssrlia. Proof.
by apply leq_divDl. move => d m n LEQ.
Qed. rewrite /div_ceil.
have LEQd: m %/ d <= n %/ d by apply leq_div2r.
destruct (d %| m) eqn:Mm; destruct (d %| n) eqn:Mn => //; first by ssrlia.
rewrite ltn_divRL //.
apply ltn_leq_trans with m => //.
move: (leq_trunc_div m d) => LEQm.
destruct (ltngtP (m %/ d * d) m) => //.
move: e => /eqP EQ; rewrite -dvdn_eq in EQ.
by rewrite EQ in Mm.
Qed.
(** Given [T] and [Δ] such that [Δ >= T > 0], we show that [div_ceil Δ T]
is strictly greater than [div_ceil (Δ - T) T]. *)
Lemma leq_div_ceil_add1:
forall Δ T,
T > 0 -> Δ >= T ->
div_ceil (Δ - T) T < div_ceil Δ T.
Proof.
intros * POS LE. rewrite /div_ceil.
have lkc: (Δ - T) %/ T < Δ %/ T.
{ rewrite divnBr; last by auto.
rewrite divnn POS.
rewrite ltn_psubCl //; try ssrlia.
by rewrite divn_gt0.
}
destruct (T %| Δ) eqn:EQ1.
{ have divck: (T %| Δ) -> (T %| (Δ - T)) by auto.
apply divck in EQ1 as EQ2.
rewrite EQ2; apply lkc.
}
by destruct (T %| Δ - T) eqn:EQ, (T %| Δ) eqn:EQ3; auto.
Qed.
(** We show that the division with ceiling by a constant [T] is a subadditive function. *)
Lemma div_ceil_subadditive:
forall T, subadditive (div_ceil^~T).
Proof.
move=> T ab a b SUM.
rewrite -SUM.
destruct (T %| a) eqn:DIVa, (T %| b) eqn:DIVb.
- have DIVab: T %| a + b by apply dvdn_add.
by rewrite /div_ceil DIVa DIVb DIVab divnDl.
- have DIVab: T %| a+b = false by rewrite -DIVb; apply dvdn_addr.
by rewrite /div_ceil DIVa DIVb DIVab divnDl //=; ssrlia.
- have DIVab: T %| a+b = false by rewrite -DIVa; apply dvdn_addl.
by rewrite /div_ceil DIVa DIVb DIVab divnDr //=; ssrlia.
- destruct (T %| a + b) eqn:DIVab.
+ rewrite /div_ceil DIVa DIVb DIVab.
apply leq_trans with (a %/ T + b %/T + 1); last by ssrlia.
by apply leq_divDl.
+ rewrite /div_ceil DIVa DIVb DIVab.
apply leq_ltn_trans with (a %/ T + b %/T + 1); last by ssrlia.
by apply leq_divDl.
Qed.
(** We show that for any two integers [a] and [b],
[a] is less than [a %/ b * b + b] given that [b] is positive. *)
Lemma div_floor_add_g:
forall a b,
b > 0 ->
a < a %/ b * b + b.
Proof.
intros * POS.
specialize (divn_eq a b) => DIV.
rewrite [in X in X < _]DIV.
rewrite ltn_add2l.
by apply ltn_pmod.
Qed.
(** We prove a technical lemma stating that for any three integers [a, (** We prove a technical lemma stating that for any three integers [a, b, c]
b, c] such that [c > b], [mod] can be swapped with subtraction in such that [c > b], [mod] can be swapped with subtraction in
the expression [(a + c - b) %% c]. *) the expression [(a + c - b) %% c]. *)
Lemma mod_elim: Lemma mod_elim:
forall a b c, forall a b c,
c > b -> c > b ->
(a + c - b) %% c = if a %% c >= b then (a %% c - b) else (a %% c + c - b). (a + c - b) %% c = if a %% c >= b then (a %% c - b) else (a %% c + c - b).
Proof. Proof.
intros * BC. intros * BC.
have POS : c > 0 by ssrlia. have POS : c > 0 by ssrlia.
have G : a %% c < c by apply ltn_pmod. have G : a %% c < c by apply ltn_pmod.
case (b <= a %% c) eqn:CASE; rewrite -addnBA; auto; rewrite -modnDml. case (b <= a %% c) eqn:CASE; rewrite -addnBA; auto; rewrite -modnDml.
- rewrite addnABC; auto. - rewrite addnABC; auto.
by rewrite -modnDmr modnn addn0 modn_small; auto; ssrlia. by rewrite -modnDmr modnn addn0 modn_small; auto; ssrlia.
- by rewrite modn_small; ssrlia. - by rewrite modn_small; ssrlia.
Qed. Qed.
End DivFloorCeil.
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