Skip to content

Commit

Permalink
feat(field_theory/adjoin): `intermediate_field.exists_finset_of_mem_s…
Browse files Browse the repository at this point in the history
…upr` (#15518)

This PR adds a lemma stating that an element of a compositum of intermediate fields lies in a finite compositum.
  • Loading branch information
tb65536 committed Jul 19, 2022
1 parent c55cadb commit 3563936
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/field_theory/adjoin.lean
Expand Up @@ -447,6 +447,14 @@ instance : is_compactly_generated (intermediate_field F E) :=
Sup_image.trans (le_antisymm (supr_le (λ i, supr_le (λ hi, adjoin_simple_le_iff.mpr hi)))
(λ x hx, adjoin_simple_le_iff.mp (le_supr_of_le x (le_supr_of_le hx le_rfl))))⟩⟩⟩

lemma exists_finset_of_mem_supr {ι : Type*} {f : ι → intermediate_field F E}
{x : E} (hx : x ∈ ⨆ i, f i) : ∃ s : finset ι, x ∈ ⨆ i ∈ s, f i :=
begin
have := (adjoin_simple_is_compact_element x).exists_finset_of_le_supr (intermediate_field F E) f,
simp only [adjoin_simple_le_iff] at this,
exact this hx,
end

end adjoin_simple
end adjoin_def

Expand Down

0 comments on commit 3563936

Please sign in to comment.