Skip to content

Commit

Permalink
minor cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
markusdemedeiros committed Nov 6, 2024
1 parent 0399d5a commit aef1458
Showing 1 changed file with 1 addition and 3 deletions.
Original file line number Diff line number Diff line change
Expand Up @@ -9,8 +9,7 @@ import SampCert.DifferentialPrivacy.Queries.UnboundedMax.Properties
import SampCert.DifferentialPrivacy.Pure.System

noncomputable section
set_option pp.coercions false
-- set_option pp.all true

open Classical

namespace SLang
Expand Down Expand Up @@ -269,7 +268,6 @@ lemma DSN (N : ℕ) (H : Neighbour L1 L2) : ((exactDiffSum N L1) : ℝ) - (exact
simp only [not_le] at hd
rw [min_eq_right_iff.mpr ?G1]
case G1 =>
-- #check Nat.add_one_le_iff
have X : (1 : ℝ) = ((1 : ℕ) : ℝ) := by simp
rw [X]
rw [← Nat.cast_add]
Expand Down

0 comments on commit aef1458

Please sign in to comment.