Commit 2025-06-19 05:18 a978d177

View on Github →

chore(Tactic/Linarith): put linarith declarations into Mathlib.Tactic namespace (#25955) The Name.isMetaProgramming function is used to exclude lemmas from library search tactics. Thus, it is important that lemmas that are only meant for use in a tactic implementation have a name flagged by Name.isMetaProgramming. So, this PR renames everying in Mathlib/Tactic/Linarith to the namespace Mathlib.Tactic.Linarith (which previously was just Linarith)

Estimated changes

deleted def Linarith.Branch
deleted structure Linarith.CertificateOracle
deleted def Linarith.Comp.add
deleted def Linarith.Comp.cmp
deleted def Linarith.Comp.scale
deleted def Linarith.Comp.vars
deleted structure Linarith.Comp
deleted structure Linarith.GlobalPreprocessor
deleted def Linarith.Linexp.cmp
deleted def Linarith.Linexp.get
deleted structure Linarith.Preprocessor
deleted structure Linarith.PreprocessorBase
deleted theorem Linarith.add_neg
deleted theorem Linarith.add_nonpos
deleted theorem Linarith.eq_of_eq_of_eq
deleted theorem Linarith.le_of_eq_of_le
deleted theorem Linarith.le_of_le_of_eq
deleted theorem Linarith.lt_irrefl
deleted theorem Linarith.lt_of_eq_of_lt
deleted theorem Linarith.lt_of_lt_of_eq
deleted theorem Linarith.mul_eq
deleted theorem Linarith.mul_neg
deleted theorem Linarith.mul_nonpos
deleted theorem Linarith.mul_zero_eq
deleted theorem Linarith.natCast_nonneg
deleted theorem Linarith.sub_neg_of_lt
deleted theorem Linarith.sub_nonpos_of_le
deleted theorem Linarith.zero_lt_one
deleted theorem Linarith.zero_mul_eq
deleted inductive Linarith.CompSource
deleted structure Linarith.LinarithData
deleted def Linarith.PComp.add
deleted def Linarith.PComp.cmp
deleted structure Linarith.PComp
deleted def Linarith.elimVar
deleted def Linarith.elimVarM
deleted def Linarith.getMaxVar
deleted def Linarith.pelimVar
deleted def Linarith.update
deleted def Linarith.validate