Skip to content

Commit

Permalink
Proved composition and mechanism with additinoal properties
Browse files Browse the repository at this point in the history
  • Loading branch information
jtristan committed May 2, 2024
1 parent bec4178 commit c5fcdc5
Show file tree
Hide file tree
Showing 4 changed files with 386 additions and 23 deletions.
20 changes: 12 additions & 8 deletions SampCert/DiffPrivacy/BoundedAvg.lean
Original file line number Diff line number Diff line change
Expand Up @@ -33,13 +33,17 @@ theorem BoundedSumQueryDP (L U : ℤ) (h : L < U) (ε₁ ε₂ : ℕ+) : DP (Noi
unfold NoisedBoundedAvgQuery'
simp only

have A := @NoisedCountingQueryDP ℤ ε₁ (2 * ε₂)
have B := @NoisedBoundedSumQueryDP L U h ε₁ (2 * ε₂)
have C := DPCompose B A
simp at C
ring_nf at C
rw [← division_def] at C
have D := DPPostProcess C (fun z => z.1 / z.2)
exact D
have A₁ := @NoisedCountingQueryDP ℤ ε₁ (2 * ε₂)
have A₂ := @NoisedCountingQuery_NonZeroNQ ℤ ε₁ (2 * ε₂)
have A₃ := @NoisedCountingQuery_NonTopNQ ℤ ε₁ (2 * ε₂)
have A₄ := @NoisedCountingQuery_NonTopRDNQ ℤ ε₁ (2 * ε₂)
sorry
-- have B := @NoisedBoundedSumQueryDP L U h ε₁ (2 * ε₂)
-- have C := DPCompose B A
-- simp at C
-- ring_nf at C
-- rw [← division_def] at C
-- have D := DPPostProcess C (fun z => z.1 / z.2)
-- exact D

end SLang
3 changes: 0 additions & 3 deletions SampCert/DiffPrivacy/ConcentratedBound.lean
Original file line number Diff line number Diff line change
Expand Up @@ -548,8 +548,5 @@ theorem RenyiDivergenceBound' {σ α : ℝ} (h : σ ≠ 0) (h' : 1 < α) (μ ν
apply RenyiSumSG_nonneg h
. apply RenyiSumSG_nonneg h
. apply SummableRenyiGauss h



rw [A]
apply RenyiDivergenceBound_pre h h'
15 changes: 14 additions & 1 deletion SampCert/DiffPrivacy/Count.lean
Original file line number Diff line number Diff line change
Expand Up @@ -34,8 +34,21 @@ theorem CountingQuery1Sensitive :
def NoisedCountingQuery (ε₁ ε₂ : ℕ+) (l : List T) : SLang ℤ := do
NoisedQuery CountingQuery 1 ε₁ ε₂ l

theorem NoisedCountingQueryDP (ε₁ ε₂ : ℕ+) : @DP T ℤ (NoisedCountingQuery ε₁ ε₂) ((ε₁ : ℝ) / ε₂) := by
theorem NoisedCountingQueryDP (ε₁ ε₂ : ℕ+) :
@DP T ℤ (NoisedCountingQuery ε₁ ε₂) ((ε₁ : ℝ) / ε₂) := by
apply NoisedQueryDP
apply CountingQuery1Sensitive

theorem NoisedCountingQuery_NonZeroNQ (ε₁ ε₂ : ℕ+) :
@NonZeroNQ T ℤ (NoisedCountingQuery ε₁ ε₂) := by
apply NoisedQuery_NonZeroNQ

theorem NoisedCountingQuery_NonTopNQ (ε₁ ε₂ : ℕ+) :
@NonTopNQ T ℤ (NoisedCountingQuery ε₁ ε₂) := by
apply NoisedQuery_NonTopNQ

theorem NoisedCountingQuery_NonTopRDNQ (ε₁ ε₂ : ℕ+) :
@NonTopRDNQ T ℤ (NoisedCountingQuery ε₁ ε₂) := by
apply NoisedQuery_NonTopRDNQ

end SLang
Loading

0 comments on commit c5fcdc5

Please sign in to comment.