Mathlib Changelog
v4
Changelog
About
Github
Commit
2022-12-17 23:54
4e2a7237
View on Github →
chore: tidy various files (
#1086
)
Estimated changes
Modified
Mathlib/Algebra/EuclideanDomain/Basic.lean
Modified
Mathlib/Algebra/Field/Basic.lean
added
theorem
ofDual_rat_cast
added
theorem
ofLex_rat_cast
deleted
theorem
of_dual_rat_cast
deleted
theorem
of_lex_rat_cast
added
theorem
toDual_rat_cast
added
theorem
toLex_rat_cast
deleted
theorem
to_dual_rat_cast
deleted
theorem
to_lex_rat_cast
Modified
Mathlib/Algebra/Group/Opposite.lean
added
theorem
AddOpposite.opMulEquiv_toEquiv
deleted
theorem
AddOpposite.op_mul_equiv_to_equiv
added
theorem
MulOpposite.opAddEquiv_toEquiv
deleted
theorem
MulOpposite.op_add_equiv_to_equiv
added
theorem
MulOpposite.semiconjBy_op
added
theorem
MulOpposite.semiconjBy_unop
deleted
theorem
MulOpposite.semiconj_by_op
deleted
theorem
MulOpposite.semiconj_by_unop
added
theorem
Units.coe_opEquiv_symm
deleted
theorem
Units.coe_op_equiv_symm
added
theorem
Units.coe_unop_opEquiv
deleted
theorem
Units.coe_unop_op_equiv
Modified
Mathlib/Algebra/Hom/Equiv/TypeTags.lean
Modified
Mathlib/Algebra/Hom/Ring.lean
added
theorem
NonUnitalRingHom.coe_toMulHom
deleted
theorem
NonUnitalRingHom.coe_to_mulHom
added
theorem
RingHom.coe_addMonoidHom_id
deleted
theorem
RingHom.coe_add_monoid_hom_id
added
theorem
RingHom.coe_monoidHom_id
deleted
theorem
RingHom.coe_monoid_hom_id
added
theorem
RingHom.isUnit_map
deleted
theorem
RingHom.is_unit_map
Modified
Mathlib/Algebra/Order/AbsoluteValue.lean
added
theorem
AbsoluteValue.coe_toMonoidHom
deleted
theorem
AbsoluteValue.coe_to_monoid_hom
Modified
Mathlib/Algebra/Order/Hom/Monoid.lean
added
theorem
strictAnti_iff_map_neg
added
theorem
strictAnti_iff_map_pos
added
theorem
strictMono_iff_map_neg
added
theorem
strictMono_iff_map_pos
deleted
theorem
strict_anti_iff_map_neg
deleted
theorem
strict_anti_iff_map_pos
deleted
theorem
strict_mono_iff_map_neg
deleted
theorem
strict_mono_iff_map_pos
Modified
Mathlib/Algebra/Order/Invertible.lean
Modified
Mathlib/Algebra/Order/Monoid/ToMulBot.lean
added
theorem
WithZero.toMulBot_coe_ofAdd
deleted
theorem
WithZero.toMulBot_coe_of_add
Modified
Mathlib/Algebra/Ring/Opposite.lean
Modified
Mathlib/Control/Traversable/Lemmas.lean
added
theorem
Traversable.pureTransformation_apply
deleted
theorem
Traversable.pure_transformation_apply
Modified
Mathlib/Data/Bool/Basic.lean
added
theorem
Bool.ofNat_le_ofNat
added
theorem
Bool.ofNat_toNat
deleted
theorem
Bool.of_nat_le_of_nat
deleted
theorem
Bool.of_nat_to_nat
added
theorem
Bool.toNat_le_toNat
deleted
theorem
Bool.to_nat_le_to_nat
Modified
Mathlib/Data/Int/Cast/Lemmas.lean
added
theorem
Int.castAddHom_int
added
theorem
Int.castRingHom_int
deleted
theorem
Int.cast_add_hom_int
deleted
theorem
Int.cast_ring_hom_int
added
theorem
Int.cast_strictMono
deleted
theorem
Int.cast_strict_mono
added
theorem
Int.coe_castAddHom
added
theorem
Int.coe_castRingHom
deleted
theorem
Int.coe_cast_add_hom
deleted
theorem
Int.coe_cast_ring_hom
added
theorem
Sum.elim_intCast_intCast
deleted
theorem
Sum.elim_int_cast_int_cast
added
theorem
ofDual_int_cast
added
theorem
ofLex_int_cast
deleted
theorem
of_dual_int_cast
deleted
theorem
of_lex_int_cast
added
theorem
toDual_int_cast
added
theorem
toLex_int_cast
deleted
theorem
to_dual_int_cast
deleted
theorem
to_lex_int_cast
Modified
Mathlib/Data/Int/Div.lean
added
theorem
Int.eq_of_mod_eq_of_natAbs_sub_lt_natAbs
deleted
theorem
Int.eq_of_mod_eq_of_nat_abs_sub_lt_nat_abs
added
theorem
Int.natAbs_le_of_dvd_ne_zero
deleted
theorem
Int.nat_abs_le_of_dvd_ne_zero
Modified
Mathlib/Data/Int/LeastGreatest.lean
modified
theorem
Int.exists_greatest_of_bdd
modified
theorem
Int.exists_least_of_bdd
Modified
Mathlib/Data/Int/Order/Basic.lean
added
theorem
Int.lt_of_toNat_lt
deleted
theorem
Int.lt_of_to_nat_lt
added
theorem
Int.lt_toNat
deleted
theorem
Int.lt_to_nat
added
theorem
Int.toNat_eq_zero
added
theorem
Int.toNat_le
added
theorem
Int.toNat_le_toNat
added
theorem
Int.toNat_lt_toNat
added
theorem
Int.toNat_pred_coe_of_pos
added
theorem
Int.toNat_sub_of_le
deleted
theorem
Int.to_nat_eq_zero
deleted
theorem
Int.to_nat_le
deleted
theorem
Int.to_nat_le_to_nat
deleted
theorem
Int.to_nat_lt_to_nat
deleted
theorem
Int.to_nat_pred_coe_of_pos
deleted
theorem
Int.to_nat_sub_of_le
Modified
Mathlib/Data/Nat/Cast/Basic.lean
added
theorem
NeZero.nat_of_neZero
deleted
theorem
NeZero.nat_of_ne_zero
Modified
Mathlib/Data/Nat/Factorial/Basic.lean
Modified
Mathlib/Data/Nat/Pow.lean
added
theorem
Nat.pow_left_strictMono
deleted
theorem
Nat.pow_left_strict_mono
added
theorem
Nat.pow_right_strictMono
deleted
theorem
Nat.pow_right_strict_mono
Modified
Mathlib/Data/PEquiv.lean
added
theorem
PEquiv.injective_of_forall_isSome
deleted
theorem
PEquiv.injective_of_forall_is_some
added
theorem
PEquiv.isSome_symm_get
deleted
theorem
PEquiv.is_some_symm_get
Modified
Mathlib/Data/Set/BoolIndicator.lean
Modified
Mathlib/Data/Set/Function.lean
Modified
Mathlib/Data/Set/Image.lean
added
theorem
Set.preimage_setOf_eq
deleted
theorem
Set.preimage_set_of_eq
Modified
Mathlib/Data/Set/Intervals/ProjIcc.lean
added
theorem
Set.projIcc_of_right_le
deleted
theorem
Set.proj_Icc_of_right_le
Modified
Mathlib/Data/Set/Intervals/SurjOn.lean
Modified
Mathlib/Data/Set/NAry.lean
Modified
Mathlib/Data/TwoPointing.lean
Modified
Mathlib/Data/Vector.lean
added
theorem
Vector.toList_append
added
theorem
Vector.toList_cons
added
theorem
Vector.toList_drop
added
theorem
Vector.toList_length
added
theorem
Vector.toList_nil
added
theorem
Vector.toList_take
deleted
theorem
Vector.to_list_append
deleted
theorem
Vector.to_list_cons
deleted
theorem
Vector.to_list_drop
deleted
theorem
Vector.to_list_length
deleted
theorem
Vector.to_list_nil
deleted
theorem
Vector.to_list_take
Modified
Mathlib/Logic/Embedding/Set.lean
Modified
Mathlib/Logic/Equiv/Embedding.lean
Modified
Mathlib/Logic/Equiv/Set.lean
Modified
Mathlib/Order/Bounds/Basic.lean
added
theorem
isGLB_Icc
added
theorem
isGLB_Ico
added
theorem
isGLB_Ioc
added
theorem
isGLB_Ioo
added
theorem
isGLB_univ
deleted
theorem
is_glb_Icc
deleted
theorem
is_glb_Ico
deleted
theorem
is_glb_Ioc
deleted
theorem
is_glb_Ioo
deleted
theorem
is_glb_univ
Modified
Mathlib/Order/Directed.lean
added
theorem
directedOn_image
added
theorem
directedOn_of_inf_mem
deleted
theorem
directed_on_image
deleted
theorem
directed_on_of_inf_mem
added
theorem
isDirected_mono
deleted
theorem
is_directed_mono
Modified
Mathlib/Order/InitialSeg.lean
added
theorem
InitialSeg.codRestrict_apply
deleted
theorem
InitialSeg.cod_restrict_apply
added
theorem
InitialSeg.leLt_apply
deleted
theorem
InitialSeg.le_lt_apply
added
theorem
InitialSeg.ltOrEq_apply_left
added
theorem
InitialSeg.ltOrEq_apply_right
deleted
theorem
InitialSeg.lt_or_eq_apply_left
deleted
theorem
InitialSeg.lt_or_eq_apply_right
added
theorem
PrincipalSeg.codRestrict_apply
added
theorem
PrincipalSeg.codRestrict_top
deleted
theorem
PrincipalSeg.cod_restrict_apply
deleted
theorem
PrincipalSeg.cod_restrict_top
added
theorem
PrincipalSeg.equivLt_apply
added
theorem
PrincipalSeg.equivLt_top
deleted
theorem
PrincipalSeg.equiv_lt_apply
deleted
theorem
PrincipalSeg.equiv_lt_top
added
theorem
PrincipalSeg.ofElement_apply
added
theorem
PrincipalSeg.ofElement_top
added
theorem
PrincipalSeg.ofIsEmpty_top
deleted
theorem
PrincipalSeg.of_element_apply
deleted
theorem
PrincipalSeg.of_element_top
deleted
theorem
PrincipalSeg.of_is_empty_top
Modified
Mathlib/Order/LatticeIntervals.lean
Modified
Mathlib/Order/WellFounded.lean
Modified
Mathlib/Tactic/ModCases.lean