Skip to content

Commit

Permalink
chore(MeasureTheory): move Measure/OuterMeasure to `OuterMeasure/Basi…
Browse files Browse the repository at this point in the history
…c` (#10916)

I'm going to generalize some constructions
from measures to outer measures and this file is already too large.
  • Loading branch information
urkud committed Feb 24, 2024
1 parent a25ebf0 commit d3dbfd9
Show file tree
Hide file tree
Showing 4 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion Mathlib.lean
Expand Up @@ -2810,7 +2810,6 @@ import Mathlib.MeasureTheory.Measure.MeasureSpaceDef
import Mathlib.MeasureTheory.Measure.MutuallySingular
import Mathlib.MeasureTheory.Measure.NullMeasurable
import Mathlib.MeasureTheory.Measure.OpenPos
import Mathlib.MeasureTheory.Measure.OuterMeasure
import Mathlib.MeasureTheory.Measure.Portmanteau
import Mathlib.MeasureTheory.Measure.ProbabilityMeasure
import Mathlib.MeasureTheory.Measure.Regular
Expand All @@ -2825,6 +2824,7 @@ import Mathlib.MeasureTheory.Measure.WithDensity
import Mathlib.MeasureTheory.Measure.WithDensityVectorMeasure
import Mathlib.MeasureTheory.Order.Group.Lattice
import Mathlib.MeasureTheory.Order.Lattice
import Mathlib.MeasureTheory.OuterMeasure.Basic
import Mathlib.MeasureTheory.PiSystem
import Mathlib.MeasureTheory.SetSemiring
import Mathlib.MeasureTheory.Tactic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2017 Johannes Hölzl. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johannes Hölzl, Mario Carneiro
-/
import Mathlib.MeasureTheory.Measure.OuterMeasure
import Mathlib.MeasureTheory.OuterMeasure.Basic
import Mathlib.Order.Filter.CountableInter

#align_import measure_theory.measure.measure_space_def from "leanprover-community/mathlib"@"c14c8fcde993801fca8946b0d80131a1a81d1520"
Expand Down
2 changes: 1 addition & 1 deletion scripts/style-exceptions.txt
Expand Up @@ -100,8 +100,8 @@ Mathlib/MeasureTheory/Integral/Lebesgue.lean : line 1 : ERR_NUM_LIN : 2000 file
Mathlib/MeasureTheory/Integral/SetToL1.lean : line 1 : ERR_NUM_LIN : 2000 file contains 1817 lines, try to split it up
Mathlib/MeasureTheory/MeasurableSpace/Basic.lean : line 1 : ERR_NUM_LIN : 2400 file contains 2250 lines, try to split it up
Mathlib/MeasureTheory/Measure/MeasureSpace.lean : line 1 : ERR_NUM_LIN : 2300 file contains 2191 lines, try to split it up
Mathlib/MeasureTheory/Measure/OuterMeasure.lean : line 1 : ERR_NUM_LIN : 1900 file contains 1785 lines, try to split it up
Mathlib/MeasureTheory/Measure/Typeclasses.lean : line 1 : ERR_NUM_LIN : 1700 file contains 1564 lines, try to split it up
Mathlib/MeasureTheory/OuterMeasure/Basic.lean : line 1 : ERR_NUM_LIN : 1900 file contains 1785 lines, try to split it up
Mathlib/Order/Basic.lean : line 1 : ERR_NUM_LIN : 1700 file contains 1547 lines, try to split it up
Mathlib/Order/Bounds/Basic.lean : line 1 : ERR_NUM_LIN : 1900 file contains 1714 lines, try to split it up
Mathlib/Order/CompleteLattice.lean : line 1 : ERR_NUM_LIN : 2200 file contains 2091 lines, try to split it up
Expand Down

0 comments on commit d3dbfd9

Please sign in to comment.