Zulip Chat Archive
Stream: new members
Topic: Fixed point of algebra equiv is the field itself.
Junjie Bai (Mar 05 2025 at 08:17):
I want to show that the fixed points of a AlgEquiv (L [M] L) is just M. But I don't know how to show that two fixed field of two subgroup is equal if the two subgroup is equvalance. Here is a #mwe :
import Mathlib
variable {M L : Type*} [Field M] [Field L] [Algebra M L] [Normal M L] [Algebra.IsSeparable M L]
open IntermediateField
example : fixedField (⊤ : Subgroup (L ≃ₐ[M] L)) = fixedField (fixingSubgroup (⊥ : IntermediateField M L)) := by sorry
Or it's there any better way to solve this problem?
Kevin Buzzard (Mar 05 2025 at 08:35):
simp
solves this. And this makes sense: statements like docs#IntermediateField.fixingSubgroup_bot are very natural simp
lemmas because the RHS is unambiguously simpler than the LHS.
Junjie Bai (Mar 05 2025 at 08:40):
Thanks a lot! It seems that the version I'm using is too old so I can't find it :sleeping:
Last updated: May 02 2025 at 03:31 UTC