Commit 2025-02-24 10:06 ee225888

View on Github →

chore(Data/Complex): deprecate Complex.abs (#21995) in this PR:

  • Defines Complex.norm directly
  • Defines Complex.abs as Complex.norm and deprecate it
  • Change Complex.abs to norm in all definitions / statements / proofs
  • Delete Complex.norm_eq_abs and the file Data.Complex.Abs (its results are moved as deprecated aliases in Data.Complex.Norm)
  • Change the name of all results which refer to Complex.abs to use norm instead and deprecate the original names

Estimated changes

deleted theorem Complex.abs_I
deleted theorem Complex.abs_add_mul_I
deleted theorem Complex.abs_apply
deleted theorem Complex.abs_conj
deleted theorem Complex.abs_def
deleted theorem Complex.abs_im_eq_abs
deleted theorem Complex.abs_im_le_abs
deleted theorem Complex.abs_im_lt_abs
deleted theorem Complex.abs_intCast
deleted theorem Complex.abs_natCast
deleted theorem Complex.abs_ofNat
deleted theorem Complex.abs_ofReal
deleted theorem Complex.abs_prod
deleted theorem Complex.abs_re_eq_abs
deleted theorem Complex.abs_re_le_abs
deleted theorem Complex.abs_re_lt_abs
deleted theorem Complex.abs_zpow
deleted theorem Complex.equiv_limAux
deleted theorem Complex.im_le_abs
deleted theorem Complex.isCauSeq_abs
deleted theorem Complex.isCauSeq_conj
deleted theorem Complex.isCauSeq_im
deleted theorem Complex.isCauSeq_re
deleted theorem Complex.lim_abs
deleted theorem Complex.lim_conj
deleted theorem Complex.lim_im
deleted theorem Complex.lim_re
deleted theorem Complex.mul_self_abs
deleted theorem Complex.ne_zero_of_re_pos
deleted theorem Complex.normSq_eq_abs
deleted theorem Complex.range_abs
deleted theorem Complex.range_normSq
deleted theorem Complex.re_le_abs
deleted theorem Complex.sq_abs_sub_sq_im
deleted theorem Complex.sq_abs_sub_sq_re
added theorem Complex.abs_im_eq_norm
added theorem Complex.abs_im_le_norm
added theorem Complex.abs_im_lt_norm
added theorem Complex.abs_re_eq_norm
added theorem Complex.abs_re_le_norm
added theorem Complex.abs_re_lt_norm
modified theorem Complex.dist_eq
added theorem Complex.equiv_limAux
added theorem Complex.im_le_norm
added theorem Complex.isCauSeq_conj
added theorem Complex.isCauSeq_im
added theorem Complex.isCauSeq_norm
added theorem Complex.isCauSeq_re
added theorem Complex.lim_conj
added theorem Complex.lim_im
added theorem Complex.lim_norm
added theorem Complex.lim_re
modified theorem Complex.nnnorm_natCast
modified theorem Complex.nnnorm_nnratCast
modified theorem Complex.nnnorm_ofNat
modified theorem Complex.nnnorm_ratCast
modified theorem Complex.nnnorm_real
modified theorem Complex.norm_I
added theorem Complex.norm_add_mul_I
added theorem Complex.norm_conj
added theorem Complex.norm_def
deleted theorem Complex.norm_eq_abs
modified theorem Complex.norm_intCast
modified theorem Complex.norm_natCast
modified theorem Complex.norm_nnratCast
modified theorem Complex.norm_ofNat
modified theorem Complex.norm_ratCast
modified theorem Complex.norm_real
added theorem Complex.range_normSq
added theorem Complex.re_le_norm