Skip to content

Commit

Permalink
chore: move some files to MeasureTheory/MeasurableSpace/ (#7045)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Sep 9, 2023
1 parent c69a99d commit e07e8dd
Show file tree
Hide file tree
Showing 9 changed files with 10 additions and 10 deletions.
6 changes: 3 additions & 3 deletions Mathlib.lean
Expand Up @@ -2357,7 +2357,6 @@ import Mathlib.Mathport.Attributes
import Mathlib.Mathport.Notation
import Mathlib.Mathport.Rename
import Mathlib.Mathport.Syntax
import Mathlib.MeasureTheory.CardMeasurableSpace
import Mathlib.MeasureTheory.Category.MeasCat
import Mathlib.MeasureTheory.Constructions.BorelSpace.Basic
import Mathlib.MeasureTheory.Constructions.BorelSpace.Complex
Expand Down Expand Up @@ -2451,8 +2450,9 @@ import Mathlib.MeasureTheory.Integral.SetToL1
import Mathlib.MeasureTheory.Integral.TorusIntegral
import Mathlib.MeasureTheory.Integral.VitaliCaratheodory
import Mathlib.MeasureTheory.Lattice
import Mathlib.MeasureTheory.MeasurableSpace
import Mathlib.MeasureTheory.MeasurableSpaceDef
import Mathlib.MeasureTheory.MeasurableSpace.Basic
import Mathlib.MeasureTheory.MeasurableSpace.Card
import Mathlib.MeasureTheory.MeasurableSpace.Defs
import Mathlib.MeasureTheory.Measure.AEDisjoint
import Mathlib.MeasureTheory.Measure.AEMeasurable
import Mathlib.MeasureTheory.Measure.Complex
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Function/AEMeasurableSequence.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Rémy Degenne. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Rémy Degenne
-/
import Mathlib.MeasureTheory.MeasurableSpace
import Mathlib.MeasureTheory.MeasurableSpace.Basic
import Mathlib.MeasureTheory.Measure.MeasureSpaceDef

#align_import measure_theory.function.ae_measurable_sequence from "leanprover-community/mathlib"@"d003c55042c3cd08aefd1ae9a42ef89441cdaaf3"
Expand Down
Expand Up @@ -7,7 +7,7 @@ import Mathlib.Algebra.IndicatorFunction
import Mathlib.Data.Prod.TProd
import Mathlib.GroupTheory.Coset
import Mathlib.Logic.Equiv.Fin
import Mathlib.MeasureTheory.MeasurableSpaceDef
import Mathlib.MeasureTheory.MeasurableSpace.Defs
import Mathlib.Order.Filter.SmallSets
import Mathlib.Order.Filter.CountableSeparatingOn
import Mathlib.Order.LiminfLimsup
Expand Down
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Sébastien Gouëzel. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Sébastien Gouëzel, Violeta Hernández Palacios
-/
import Mathlib.MeasureTheory.MeasurableSpaceDef
import Mathlib.MeasureTheory.MeasurableSpace.Defs
import Mathlib.SetTheory.Cardinal.Cofinality
import Mathlib.SetTheory.Cardinal.Continuum

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Measure/MeasureSpace.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Mario Carneiro
-/
import Mathlib.MeasureTheory.Measure.NullMeasurable
import Mathlib.MeasureTheory.MeasurableSpace
import Mathlib.MeasureTheory.MeasurableSpace.Basic
import Mathlib.Topology.Algebra.Order.LiminfLimsup

#align_import measure_theory.measure.measure_space from "leanprover-community/mathlib"@"343e80208d29d2d15f8050b929aa50fe4ce71b55"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean
Expand Up @@ -41,7 +41,7 @@ that two measure are equal.
A `MeasureSpace` is a class that is a measurable space with a canonical measure.
The measure is denoted `volume`.
This file does not import `MeasureTheory.MeasurableSpace`, but only `MeasurableSpaceDef`.
This file does not import `MeasureTheory.MeasurableSpace.Basic`, but only `MeasurableSpace.Defs`.
## References
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/PiSystem.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Martin Zinkevich, Rémy Degenne
-/
import Mathlib.Logic.Encodable.Lattice
import Mathlib.MeasureTheory.MeasurableSpaceDef
import Mathlib.MeasureTheory.MeasurableSpace.Defs

#align_import measure_theory.pi_system from "leanprover-community/mathlib"@"98e83c3d541c77cdb7da20d79611a780ff8e7d90"

Expand Down
2 changes: 1 addition & 1 deletion test/measurability.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Rémy Degenne
-/
import Mathlib.MeasureTheory.Tactic
import Mathlib.MeasureTheory.MeasurableSpace
import Mathlib.MeasureTheory.MeasurableSpace.Basic
import Mathlib.MeasureTheory.Constructions.BorelSpace.Basic
import Mathlib.MeasureTheory.Function.SpecialFunctions.Basic
import Mathlib.MeasureTheory.Function.SpecialFunctions.Inner
Expand Down

0 comments on commit e07e8dd

Please sign in to comment.