Skip to content

Commit

Permalink
lemma3_counter_prob_choice
Browse files Browse the repository at this point in the history
  • Loading branch information
bmtrager committed Dec 8, 2024
1 parent 51e44f8 commit 4b5edce
Showing 1 changed file with 15 additions and 1 deletion.
16 changes: 15 additions & 1 deletion coq/QLearn/jaakkola_vector.v
Original file line number Diff line number Diff line change
Expand Up @@ -3367,6 +3367,20 @@ Section jaakola_vector2.
apply H10.
Qed.

Lemma lemma3_counter_prob_choice (d1 d2 : R) :
d1 > 1 ->
d2 < 1 ->
exists p, 0 < p < 1 /\ p * d1 + (1-p)*d2 = 1.
Proof.
exists ((1-d2)/(d1-d2)).
split.
- split.
+ apply Rdiv_lt_0_compat; lra.
+ rewrite <- Rdiv_lt_1; lra.
- field_simplify; try lra.
apply Rdiv_diag; lra.
Qed.

Lemma vecrvclip_max_bound (rvec : Ts -> vector R (S N)) (C : posreal) :
forall a,
Rvector_max_abs (vecrvclip (S N) rvec (pos_to_nneg C) a) <= C.
Expand Down Expand Up @@ -7044,7 +7058,7 @@ Proof.
((FiniteConditionalVariance_new prts (filt_sub k) (vecrvnth i pf (XF k)) (rv := vecrvnth_rv i pf (XF k) (rv := vec_rvXF_I filt_sub XF k))) ω)
<= (C * (1 + scaled_norm(X k ω) W)^2)))) ->

(**r X (k + 1) = (1 - α_κ) * Χ (k) + β_k * XF (k) *)
(**r X (k + 1) = (1 - α_κ) * Χ (k) + β_k * XF (k) defined componentwise *)
(forall k, rv_eq (X (S k))
(vecrvplus (vecrvminus (X k) (vecrvmult (α k) (X k))) (vecrvmult (β k) (XF k) ))) ->

Expand Down

0 comments on commit 4b5edce

Please sign in to comment.