Zulip Chat Archive

Stream: Berkeley Lean Seminar

Topic: Random intermediate_field.adjoin question


Patrick Lutz (Jan 12 2021 at 06:02):

Do we know that an FF-algebra homomorphism on F(S)F(S) is determined by its action on SS? For example do we have a lemma saying that if E/FE/F is a field extension with F(S)=F(S) = \top and if ff is an FF-algebra automorphism of EE then ff is the identity if and only if it's the identity on SS? For some reason I feel like we should have something like this but I don't see it

Thomas Browning (Jan 12 2021 at 06:12):

I've needed this too. I don't think that we have it.

Thomas Browning (Jan 12 2021 at 06:12):

A while ago I defined an equalizer subalgebra which allows you to do this for subalgebras

Thomas Browning (Jan 12 2021 at 06:12):

Could we define an equalizer intermediate field?

Thomas Browning (Jan 12 2021 at 06:14):

I guess, if E/F is a field extension and if you have two F-algebra homomorphisms E->A, then the equalizer is an intermediate field?

Patrick Lutz (Jan 12 2021 at 06:15):

yeah, I guess that's true

Patrick Lutz (Jan 12 2021 at 06:16):

actually I think I might really want it for subalgebras not intermediate fields. Since I guess most of the stuff in splitting_field.lean is about algebra adjoin not intermediate field adjoin

Patrick Lutz (Jan 12 2021 at 06:17):

is there a lemma saying exactly what I said above for subalgebras? (I realize it's pretty easy to prove using the equalizer but if it's already there I don't want to redo it)

Thomas Browning (Jan 12 2021 at 06:19):

I would guess that it's not stated explicitly for subalgebra adjoin

Thomas Browning (Jan 12 2021 at 06:19):

It would be a good lemma

Thomas Browning (Jan 12 2021 at 06:20):

It doesn't seem like it's in ring_theory/adjoin, which would be the natural place

Patrick Lutz (Jan 12 2021 at 06:21):

Actually, do you know why the gc and gi instances on algebra.adjoin are protected?

Thomas Browning (Jan 12 2021 at 06:23):

no, although there is api at the top of ring_theory/adjoin

Thomas Browning (Jan 12 2021 at 06:23):

adjoin_le_iff, for example

Patrick Lutz (Jan 12 2021 at 06:45):

actually, here's a possibly stupid question: does mathlib know that two algebra isomorphisms are equal if and only if they are equal as algebra homomorphisms?

Thomas Browning (Jan 12 2021 at 06:49):

not sure. it's a one-liner using the ext-lemmas though

Patrick Lutz (Jan 12 2021 at 06:52):

Thomas Browning said:

not sure. it's a one-liner using the ext-lemmas though

hmm, for me it's a very slow one-liner using simp and a faster two-linear using simp only with a bunch of little lemmas thrown in

Patrick Lutz (Jan 12 2021 at 06:55):

maybe "very" is an exaggeration

Thomas Browning (Jan 12 2021 at 06:56):

example {R A B : Type*} [comm_semiring R] [semiring A] [semiring B] [algebra R A] [algebra R B]
  (f g : A ≃ₐ[R] B) : f = g  f.to_alg_hom = g.to_alg_hom :=
λ h, by rw h, λ h, alg_equiv.ext $ λ x, alg_hom.ext_iff.mp h x

Last updated: Dec 20 2023 at 11:08 UTC