Skip to content

Commit

Permalink
chore: rename PushNeg.lean to Push.lean (#22108)
Browse files Browse the repository at this point in the history
This PR renames the file `PushNeg.lean` to `Push.lean`, to help reviewing #21965.

It also removes an import of PushNeg where it is already transitively imported
  • Loading branch information
JovanGerb committed Feb 20, 2025
1 parent c97217f commit 7921910
Show file tree
Hide file tree
Showing 10 changed files with 8 additions and 9 deletions.
2 changes: 1 addition & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5292,7 +5292,7 @@ import Mathlib.Tactic.ProdAssoc
import Mathlib.Tactic.ProjectionNotation
import Mathlib.Tactic.Propose
import Mathlib.Tactic.ProxyType
import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push
import Mathlib.Tactic.Qify
import Mathlib.Tactic.RSuffices
import Mathlib.Tactic.Recall
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Data/Nat/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,6 @@ import Mathlib.Logic.Function.Basic
import Mathlib.Logic.Nontrivial.Defs
import Mathlib.Tactic.Contrapose
import Mathlib.Tactic.GCongr.CoreAttrs
import Mathlib.Tactic.PushNeg
import Mathlib.Util.AssertExists

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/BoundedOrder/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl
-/
import Mathlib.Order.Max
import Mathlib.Order.ULift
import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push
import Mathlib.Tactic.Finiteness.Attr
import Mathlib.Util.AssertExists

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -206,7 +206,7 @@ import Mathlib.Tactic.ProdAssoc
import Mathlib.Tactic.ProjectionNotation
import Mathlib.Tactic.Propose
import Mathlib.Tactic.ProxyType
import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push
import Mathlib.Tactic.Qify
import Mathlib.Tactic.RSuffices
import Mathlib.Tactic.Recall
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic/ByContra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kevin Buzzard
-/
import Batteries.Tactic.Init
import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push

/-!
# The `by_contra` tactic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic/Common.lean
Original file line number Diff line number Diff line change
Expand Up @@ -76,7 +76,7 @@ import Mathlib.Tactic.OfNat
-- import Mathlib.Tactic.Positivity
import Mathlib.Tactic.ProjectionNotation
import Mathlib.Tactic.Propose
import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push
import Mathlib.Tactic.RSuffices
import Mathlib.Tactic.Recover
import Mathlib.Tactic.Relation.Rfl
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Tactic/Contrapose.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jireh Loreaux
-/

import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push

/-! # Contrapose
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion MathlibTest/push_neg.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Alice Laroche, Frédéric Dupuis, Jireh Loreaux
-/

import Mathlib.Order.Defs.LinearOrder
import Mathlib.Tactic.PushNeg
import Mathlib.Tactic.Push

private axiom test_sorry : ∀ {α}, α
set_option autoImplicit true
Expand Down
2 changes: 1 addition & 1 deletion scripts/noshake.json
Original file line number Diff line number Diff line change
Expand Up @@ -143,7 +143,7 @@
"Mathlib.Tactic.Positivity.Basic",
"Mathlib.Tactic.Positivity.Finset",
"Mathlib.Tactic.ProjectionNotation",
"Mathlib.Tactic.PushNeg",
"Mathlib.Tactic.Push",
"Mathlib.Tactic.Qify",
"Mathlib.Tactic.RSuffices",
"Mathlib.Tactic.Recover",
Expand Down

0 comments on commit 7921910

Please sign in to comment.