File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed
Mathlib/Analysis/Normed/Group Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -667,14 +667,14 @@ theorem coe_nnnorm' (a : E) : (‖a‖₊ : ℝ) = ‖a‖ := rfl
667667theorem coe_comp_nnnorm' : (toReal : ℝ≥0 → ℝ) ∘ (nnnorm : E → ℝ≥0 ) = norm :=
668668 rfl
669669
670- @[to_additive norm_toNNReal]
670+ @[to_additive (attr := simp) norm_toNNReal]
671671theorem norm_toNNReal' : ‖a‖.toNNReal = ‖a‖₊ :=
672672 @Real.toNNReal_coe ‖a‖₊
673673
674- @[to_additive toReal_enorm]
674+ @[to_additive (attr := simp) toReal_enorm]
675675lemma toReal_enorm' (x : E) : ‖x‖ₑ.toReal = ‖x‖ := by simp [enorm]
676676
677- @[to_additive ofReal_norm]
677+ @[to_additive (attr := simp) ofReal_norm]
678678lemma ofReal_norm' (x : E) : .ofReal ‖x‖ = ‖x‖ₑ := by
679679 simp [enorm, ENNReal.ofReal, Real.toNNReal, nnnorm]
680680
You can’t perform that action at this time.
0 commit comments