Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2021-03-25 19:35 b299d144

View on Github →

feat(algebra/geom_sum): rename geom_series to geom_sum, adds a lemma for the geometric sum (#6828) Declarations with names including geom_series have been renamed to use geom_sum, instead. Also adds the lemma geom_sum₂_succ_eq: geom_sum₂ x y (n + 1) = x ^ n + y * (geom_sum₂ x y n)

Estimated changes

deleted def geom_series
deleted theorem geom_series_def
deleted theorem geom_series_one
deleted theorem geom_series_zero
deleted def geom_series₂
deleted theorem geom_series₂_def
deleted theorem geom_series₂_one
deleted theorem geom_series₂_self
deleted theorem geom_series₂_with_one
deleted theorem geom_series₂_zero
added def geom_sum
deleted theorem geom_sum
added theorem geom_sum_def
added theorem geom_sum_eq
added theorem geom_sum_one
added theorem geom_sum_zero
added def geom_sum₂
added theorem geom_sum₂_def
added theorem geom_sum₂_one
added theorem geom_sum₂_self
added theorem geom_sum₂_succ_eq
added theorem geom_sum₂_with_one
added theorem geom_sum₂_zero
deleted theorem op_geom_series
deleted theorem op_geom_series₂
added theorem op_geom_sum
added theorem op_geom_sum₂
deleted theorem ring_hom.map_geom_series
added theorem ring_hom.map_geom_sum