Skip to content

Commit

Permalink
feat: port MeasureTheory.Measure.OuterMeasure (#3674)
Browse files Browse the repository at this point in the history
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
Co-authored-by: Komyyy <pol_tta@outlook.jp>
Co-authored-by: Johan Commelin <johan@commelin.net>
  • Loading branch information
4 people committed May 3, 2023
1 parent 2d97555 commit b7bda09
Show file tree
Hide file tree
Showing 3 changed files with 1,773 additions and 2 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -1521,6 +1521,7 @@ import Mathlib.Mathport.Syntax
import Mathlib.MeasureTheory.CardMeasurableSpace
import Mathlib.MeasureTheory.MeasurableSpace
import Mathlib.MeasureTheory.MeasurableSpaceDef
import Mathlib.MeasureTheory.Measure.OuterMeasure
import Mathlib.MeasureTheory.PiSystem
import Mathlib.ModelTheory.Basic
import Mathlib.ModelTheory.Encoding
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Algebra/Tower.lean
Expand Up @@ -156,8 +156,8 @@ instance (priority := 999) subsemiring (U : Subsemiring S) : IsScalarTower U S A
#align is_scalar_tower.subsemiring IsScalarTower.subsemiring

-- Porting note: @[nolint instance_priority]
instance of_ring_hom {R A B : Type _} [CommSemiring R] [CommSemiring A] [CommSemiring B]
[Algebra R A] [Algebra R B] (f : A →ₐ[R] B) :
instance (priority := 999) of_ring_hom {R A B : Type _} [CommSemiring R] [CommSemiring A]
[CommSemiring B] [Algebra R A] [Algebra R B] (f : A →ₐ[R] B) :
@IsScalarTower R A B _ f.toRingHom.toAlgebra.toSMul _ :=
letI := (f : A →+* B).toAlgebra
of_algebraMap_eq fun x => (f.commutes x).symm
Expand Down

0 comments on commit b7bda09

Please sign in to comment.