Mathlib v3 is deprecated. Go to Mathlib v4

Commit 2021-05-03 17:06 048240e8

View on Github →

chore(*): update to lean 3.30.0c (#7264) There's quite a bit of breakage from no longer reducing acc.rec so aggressively. That is, a well-founded definition like nat.factors will no longer reduce definitionally. Where you could write rfl before, you might now need to write by rw nat.factors or by simp [nat.factors]. A more inconvenient side-effect of this change is that dec_trivial becomes less powerful, since it also relies on the definitional reduction. For example nat.factors 1 = [] is no longer true by dec_trivial (or rfl). Often you can replace dec_trivial by simp or norm_num. For extremely simple definitions that only use well-founded relations of rank ω, you could consider rewriting them to use structural recursion on a fuel parameter instead. The functions nat.mod and nat.div in core have been rewritten in this way, please consult the corresponding Lean PR for details on the implementation.

Estimated changes

deleted theorem le_imp_le_of_lt_imp_lt
deleted theorem le_of_not_lt
deleted theorem le_or_lt
deleted theorem lt_or_le
added theorem fin.coe_bit0
added theorem fin.coe_bit1
added theorem fin.succ_one_eq_two
added theorem fin.zero_succ_above
modified theorem nat.land_zero
modified theorem nat.lor_zero
modified theorem nat.lxor_zero
modified theorem nat.zero_land
modified theorem nat.zero_lor
modified theorem nat.zero_lxor
modified theorem nat.factors_one
modified theorem nat.factors_zero
modified theorem nat.not_prime_one
modified theorem nat.not_prime_zero
modified theorem nat.prime_three