Skip to content

Commit

Permalink
chore: move pointwise set files to Algebra._.Pointwise
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies committed Nov 16, 2024
1 parent 2aeb155 commit 586e58a
Show file tree
Hide file tree
Showing 17 changed files with 18 additions and 45 deletions.
9 changes: 4 additions & 5 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -289,7 +289,10 @@ import Mathlib.Algebra.Group.Pi.Lemmas
import Mathlib.Algebra.Group.Pointwise.Finset.Basic
import Mathlib.Algebra.Group.Pointwise.Finset.Interval
import Mathlib.Algebra.Group.Pointwise.Set.Basic
import Mathlib.Algebra.Group.Pointwise.Set.BigOperators
import Mathlib.Algebra.Group.Pointwise.Set.Card
import Mathlib.Algebra.Group.Pointwise.Set.Finite
import Mathlib.Algebra.Group.Pointwise.Set.ListOfFn
import Mathlib.Algebra.Group.Prod
import Mathlib.Algebra.Group.Semiconj.Basic
import Mathlib.Algebra.Group.Semiconj.Defs
Expand Down Expand Up @@ -648,6 +651,7 @@ import Mathlib.Algebra.Order.Group.OrderIso
import Mathlib.Algebra.Order.Group.PiLex
import Mathlib.Algebra.Order.Group.Pointwise.Bounds
import Mathlib.Algebra.Order.Group.Pointwise.CompleteLattice
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.Algebra.Order.Group.PosPart
import Mathlib.Algebra.Order.Group.Prod
import Mathlib.Algebra.Order.Group.Synonym
Expand Down Expand Up @@ -2797,12 +2801,7 @@ import Mathlib.Data.Set.Operations
import Mathlib.Data.Set.Opposite
import Mathlib.Data.Set.Pairwise.Basic
import Mathlib.Data.Set.Pairwise.Lattice
import Mathlib.Data.Set.Pointwise.BigOperators
import Mathlib.Data.Set.Pointwise.BoundedMul
import Mathlib.Data.Set.Pointwise.Finite
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.Data.Set.Pointwise.Iterate
import Mathlib.Data.Set.Pointwise.ListOfFn
import Mathlib.Data.Set.Pointwise.SMul
import Mathlib.Data.Set.Pointwise.Support
import Mathlib.Data.Set.Prod
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,9 @@ Authors: Kenny Lau
import Mathlib.Algebra.Algebra.Bilinear
import Mathlib.Algebra.Algebra.Opposite
import Mathlib.Algebra.Group.Pointwise.Finset.Basic
import Mathlib.Algebra.Group.Pointwise.Set.BigOperators
import Mathlib.Algebra.GroupWithZero.NonZeroDivisors
import Mathlib.Algebra.Module.Submodule.Pointwise
import Mathlib.Data.Set.Pointwise.BigOperators
import Mathlib.Data.Set.Semiring
import Mathlib.GroupTheory.GroupAction.SubMulAction.Pointwise

Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,11 +5,11 @@ Authors: Floris van Doorn, Yaël Dillies
-/
import Mathlib.Algebra.BigOperators.Group.Finset
import Mathlib.Algebra.Group.Action.Pi
import Mathlib.Algebra.Group.Pointwise.Set.Finite
import Mathlib.Data.Finset.Density
import Mathlib.Data.Finset.Max
import Mathlib.Data.Finset.NAry
import Mathlib.Data.Set.Pointwise.Finite
import Mathlib.Data.Set.Pointwise.ListOfFn
import Mathlib.Algebra.Group.Pointwise.Set.ListOfFn
import Mathlib.Data.Set.Pointwise.SMul

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Group/Pointwise/Finset/Interval.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: Eric Wieser
-/
import Mathlib.Algebra.Group.Pointwise.Finset.Basic
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.Order.Interval.Finset.Defs

/-! # Pointwise operations on intervals
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Group/Pointwise/Set/Card.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2024 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.Data.Set.Pointwise.Finite
import Mathlib.Algebra.Group.Pointwise.Set.Finite
import Mathlib.SetTheory.Cardinal.Finite

/-!
Expand Down
File renamed without changes.
File renamed without changes.
2 changes: 2 additions & 0 deletions Mathlib/Algebra/Order/Group/Pointwise/Bounds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -48,6 +48,8 @@ lemma BddAbove.mul (hs : BddAbove s) (ht : BddAbove t) : BddAbove (s * t) :=
lemma BddBelow.mul (hs : BddBelow s) (ht : BddBelow t) : BddBelow (s * t) :=
(Nonempty.mul hs ht).mono (subset_lowerBounds_mul s t)

@[to_additive (attr := deprecated (since := "2024-11-13"))] alias Set.BddAbove.mul := BddAbove.mul

@[to_additive]
lemma BddAbove.range_mul (hf : BddAbove (range f)) (hg : BddAbove (range g)) :
BddAbove (range fun i ↦ f i * g i) :=
Expand Down
File renamed without changes.
4 changes: 2 additions & 2 deletions Mathlib/Analysis/Normed/Field/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,10 +5,10 @@ Authors: Patrick Massot, Johannes Hölzl
-/
import Mathlib.Algebra.Algebra.NonUnitalSubalgebra
import Mathlib.Algebra.Algebra.Subalgebra.Basic
import Mathlib.Algebra.Field.Subfield.Defs
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.Analysis.Normed.Group.Constructions
import Mathlib.Analysis.Normed.Group.Submodule
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.Algebra.Field.Subfield.Defs

/-!
# Normed fields
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Real/Cardinality.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,9 @@ Copyright (c) 2019 Floris van Doorn. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Floris van Doorn
-/
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.Analysis.SpecificLimits.Basic
import Mathlib.Data.Rat.Denumerable
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.SetTheory.Cardinal.Continuum

/-!
Expand Down
28 changes: 0 additions & 28 deletions Mathlib/Data/Set/Pointwise/BoundedMul.lean

This file was deleted.

2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/Finiteness.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2021 Riccardo Brasca. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Riccardo Brasca
-/
import Mathlib.Algebra.Group.Pointwise.Set.Finite
import Mathlib.Algebra.Group.Subgroup.Pointwise
import Mathlib.Data.Set.Pointwise.Finite
import Mathlib.GroupTheory.QuotientGroup.Defs
import Mathlib.SetTheory.Cardinal.Finite

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Joseph Myers. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Myers
-/
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.LinearAlgebra.AffineSpace.Basic
import Mathlib.LinearAlgebra.BilinearMap
import Mathlib.LinearAlgebra.Pi
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Algebra/Order/Field.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Benjamin Davidson. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Benjamin Davidson, Devon Tuma, Eric Rodriguez, Oliver Nash
-/
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.Order.Filter.AtTopBot.Field
import Mathlib.Topology.Algebra.Field
import Mathlib.Topology.Algebra.Order.Group
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/MetricSpace/Pseudo/Real.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2015, 2017 Jeremy Avigad. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jeremy Avigad, Robert Y. Lewis, Johannes Hölzl, Mario Carneiro, Sébastien Gouëzel
-/
import Mathlib.Data.Set.Pointwise.Interval
import Mathlib.Algebra.Order.Group.Pointwise.Interval
import Mathlib.Topology.MetricSpace.Pseudo.Pi

/-!
Expand Down

0 comments on commit 586e58a

Please sign in to comment.