Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2020-05-12 15:37 34a0c8c5

View on Github →

chore(*): unify use of left and right for injectivity lemmas (#2655) This is the evil twin of #2652 using the opposite convention: the name of a lemma stating that a function in two arguments is injective in one of the arguments refers to the argument that changes. Example:

lemma sub_right_inj : a - b = a - c ↔ b = c

See also the Zulip discussion. This PR renames lemmas following the other convention. The following lemmas were renamed: algebra/group/basic.lean:

  • mul_left_injectivemul_right_injective
  • mul_left_injmul_right_inj
  • sub_left_injsub_right_inj algebra/goup/units.lean:
  • mul_left_injmul_right_inj
  • divp_right_injdivp_left_inj algebra/group_power.lean:
  • pow_right_injpow_left_inj algebra/group_with_zero.lean:
  • div_right_inj' div_left_inj'
  • mul_right_inj'mul_left_inj' algebra/ring.lean:
  • domain.mul_right_injdomain.mul_left_inj data/finsupp.lean:
  • single_right_injsingle_left_inj data/list/basic.lean:
  • append_inj_leftappend_inj_right
  • append_inj_left'append_inj_right'
  • append_left_injappend_right_inj
  • prefix_append_left_injprefix_append_right_inj data/nat/basic.lean:
  • mul_left_injmul_right_inj data/real/ennreal.lean:
  • add_left_injadd_right_inj
  • sub_left_injsub_right_inj set_theory/ordinal.lean:
  • mul_left_injmul_right_inj

Estimated changes

modified theorem mul_left_inj
modified theorem mul_left_injective
modified theorem mul_right_inj
modified theorem mul_right_injective
modified theorem sub_left_inj
modified theorem sub_right_inj
added theorem divp_left_inj
deleted theorem divp_right_inj
modified theorem units.mul_left_inj
modified theorem units.mul_right_inj
added theorem div_left_inj'
deleted theorem div_right_inj'
added theorem mul_left_inj'
deleted theorem mul_right_inj'