Skip to content

Commit

Permalink
chore(measure_theory/probability_mass_function): avoid non-terminal s…
Browse files Browse the repository at this point in the history
…imp in coe_le_one (#10112)
  • Loading branch information
Ruben-VandeVelde committed Nov 2, 2021
1 parent 6df3143 commit 2d8be73
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion src/measure_theory/probability_mass_function.lean
Expand Up @@ -51,7 +51,8 @@ def support (p : pmf α) : set α := {a | p.1 a ≠ 0}
a ∈ p.support ↔ p a ≠ 0 := iff.rfl

lemma coe_le_one (p : pmf α) (a : α) : p a ≤ 1 :=
has_sum_le (by intro b; split_ifs; simp [h]; exact le_refl _) (has_sum_ite_eq a (p a)) p.2
has_sum_le (by { intro b, split_ifs; simp only [h, zero_le'] })
(has_sum_ite_eq a (p a)) (has_sum_coe_one p)

section pure

Expand Down

0 comments on commit 2d8be73

Please sign in to comment.