Commit 2024-12-20 20:23 75faccb7
View on Github →feat: some more properties of linearly disjoint (#19614) Major new results:
*.LinearDisjoint.map
: linear disjointness is preserved by injective ring homomorphism.rank_sup_of_isAlgebraic
->rank_sup
at the expense of importingAlgebraicIndependent
.IntermediateField.LinearDisjoint.algEquiv_of_isAlgebraic
: linear disjointness is preserved by isomorphisms, provided that one of the field is algebraic. Regarding https://mathoverflow.net/questions/8324:Subalgebra.LinearDisjoint.isDomain_of_injective
,Subalgebra.LinearDisjoint.exists_field_of_isDomain_of_injective
:IntermediateField.LinearDisjoint.isDomain'
,IntermediateField.LinearDisjoint.exists_field_of_isDomain
: under some flatness and injectivity conditions, ifA
andB
areR
-algebras (resp. fields), thenA ⊗[R] B
is a domain if and only if there exists a field such thatA
andB
inject into it and their images are linearly disjoint.IntermediateField.LinearDisjoint.isField_of_forall
,IntermediateField.LinearDisjoint.of_isField'
: ifA
andB
are field extensionsF
, thenA ⊗[F] B
is a field if and only if for any field such thatA
andB
map to it, their images are linearly disjoint.Algebra.TensorProduct.not_isField_of_transcendental
,Algebra.TensorProduct.isAlgebraic_of_isField
: ifA
andB
are flatR
-algebras, both of them are transcendental, thenA ⊗[R] B
cannot be a field, equivalently, ifA ⊗[R] B
is a field, then one of them is algebraic.Algebra.TensorProduct.isField_of_isAlgebraic
: ifE
andK
are field extensions ofF
, one of them is algebraic, such thatE ⊗[F] K
is a domain, thenE ⊗[F] K
is also a field.