Skip to content

Commit

Permalink
Manipulation of final bit of ARcoupl dunif rev
Browse files Browse the repository at this point in the history
  • Loading branch information
hei411 committed Mar 5, 2024
1 parent b97db5c commit d3b9a17
Showing 1 changed file with 14 additions and 2 deletions.
16 changes: 14 additions & 2 deletions theories/prob/couplings_app.v
Original file line number Diff line number Diff line change
Expand Up @@ -780,10 +780,15 @@ Proof.
+ admit.
}
apply (Rle_trans _ (SeriesC g + (N - M))); auto.
(* { (*?!*) *)
(* admit. } *)
rewrite Rplus_comm.
apply Rplus_le_compat_l.
assert (0<=SeriesC g) as Hpos.
{ apply SeriesC_ge_0'. naive_solver. }
rewrite Rmult_comm (Rmult_comm (/M)).
rewrite -Rdiv_def Rmult_div_assoc.
rewrite -Rle_div_r; last lra.
rewrite Rmult_comm.
apply Rmult_le_compat_r; lra.
Admitted.

Lemma ARcoupl_dunif_leq_rev_inj (N M : nat) h `{Inj (fin M) (fin N) (=) (=) h}:
Expand Down Expand Up @@ -812,6 +817,13 @@ Proof.
(* admit. } *)
rewrite Rplus_comm.
apply Rplus_le_compat_l.
assert (0<=SeriesC g) as Hpos.
{ apply SeriesC_ge_0'. naive_solver. }
rewrite Rmult_comm (Rmult_comm (/M)).
rewrite -Rdiv_def Rmult_div_assoc.
rewrite -Rle_div_r; last lra.
rewrite Rmult_comm.
apply Rmult_le_compat_r; lra.
Admitted.

Lemma ARcoupl_dunif_no_coll_l `{Countable A} (v : A) (N : nat) (x : fin N) :
Expand Down

0 comments on commit d3b9a17

Please sign in to comment.