Commit 2020-05-15 21:05 1b85e3c2
View on Github →chore(*): bump to lean-3.12.0 (#2681)
Changes to bracket notation
{a}now requires an instancehas_singleton;insert a ∅ = {a}is calledinsert_emptyc_eq, provided by anis_lawful_singletoninstance;a ∈ ({b} : set α)is now defeqa = b, nota = b ∨ false;({a} : set α)is no longer defeqinsert a ∅;({a} : finset α)now means⟨⟨[a]⟩, _⟩(used to be calledfinset.singleton a), notinsert a ∅;- removed
finset.singleton; {a, b}is nowinsert a {b}, notinsert b {a}.finset.univ : finset boolis now{tt, ff};(({a} : finset α) : set α)is no longer defeq{a}.
Tactic norm_num
The interactive tactic norm_num was recently rewritten in Lean. The non-interactive tactic.norm_num has been removed in Lean 3.12 so that we can migrate the algebraic hierarchy to mathlib in 3.13.
Tactic combinators
https://github.com/leanprover-community/lean/pull/212 renames a bunch of tactic combinators. We change to using the new names.
Tactic case
https://github.com/leanprover-community/lean/pull/228 slightly changes the semantics of the case tactic. We fix the resulting breakage to be conform the new semantics.