Skip to content

Commit

Permalink
fix build
Browse files Browse the repository at this point in the history
  • Loading branch information
riccardobrasca committed Nov 27, 2023
1 parent 5e0e357 commit 02fef3c
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions FltRegular/NumberTheory/KummersLemma/KummersLemma.lean
Original file line number Diff line number Diff line change
Expand Up @@ -64,6 +64,9 @@ theorem exists_units_eq_div_root_of_isUnramified
rw [← RingHom.coe_comp, ← IsScalarTower.algebraMap_eq, IsScalarTower.algebraMap_eq A K L]
exact (algebraMap K L).injective.comp (IsFractionRing.injective _ _)
rw [← NoZeroSMulDivisors.iff_algebraMap_injective] at hAB
letI : Algebra (FractionRing A) (FractionRing B) := FractionRing.liftAlgebra _ _
have : IsScalarTower A (FractionRing A) (FractionRing B) :=
FractionRing.isScalarTower_liftAlgebra _ _
have H : RingHom.comp (algebraMap (FractionRing A) (FractionRing B))
↑(FractionRing.algEquiv A K).symm.toRingEquiv =
RingHom.comp ↑(FractionRing.algEquiv B L).symm.toRingEquiv (algebraMap K L)
Expand Down

0 comments on commit 02fef3c

Please sign in to comment.