Skip to content

Commit 8f1b057

Browse files
committed
chore: make ‖x‖ₑ.toReal = ‖x‖ simp (#21327)
From LeanAPAP
1 parent 702f356 commit 8f1b057

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

Mathlib/Analysis/Normed/Group/Basic.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -667,14 +667,14 @@ theorem coe_nnnorm' (a : E) : (‖a‖₊ : ℝ) = ‖a‖ := rfl
667667
theorem coe_comp_nnnorm' : (toReal : ℝ≥0 → ℝ) ∘ (nnnorm : E → ℝ≥0) = norm :=
668668
rfl
669669

670-
@[to_additive norm_toNNReal]
670+
@[to_additive (attr := simp) norm_toNNReal]
671671
theorem norm_toNNReal' : ‖a‖.toNNReal = ‖a‖₊ :=
672672
@Real.toNNReal_coe ‖a‖₊
673673

674-
@[to_additive toReal_enorm]
674+
@[to_additive (attr := simp) toReal_enorm]
675675
lemma toReal_enorm' (x : E) : ‖x‖ₑ.toReal = ‖x‖ := by simp [enorm]
676676

677-
@[to_additive ofReal_norm]
677+
@[to_additive (attr := simp) ofReal_norm]
678678
lemma ofReal_norm' (x : E) : .ofReal ‖x‖ = ‖x‖ₑ := by
679679
simp [enorm, ENNReal.ofReal, Real.toNNReal, nnnorm]
680680

0 commit comments

Comments
 (0)