Skip to content

Commit

Permalink
feat(field_theory/adjoin): add dim_bot, finrank_bot (#10964)
Browse files Browse the repository at this point in the history
Added two simp lemmas, showing that the dimension and finrank respectively of bottom intermediate fields are 1. 

Co-authored-by: Sebastian-Monnet <54352341+Sebastian-Monnet@users.noreply.github.com>
  • Loading branch information
Sebastian-Monnet and Sebastian-Monnet committed Dec 23, 2021
1 parent f4e46fd commit 08b13ec
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/field_theory/adjoin.lean
Expand Up @@ -375,6 +375,12 @@ by rw [← to_subalgebra_eq_iff, ← dim_eq_dim_subalgebra,
by rw [← to_subalgebra_eq_iff, ← finrank_eq_finrank_subalgebra,
subalgebra.finrank_eq_one_iff, bot_to_subalgebra]

@[simp] lemma dim_bot : module.rank F (⊥ : intermediate_field F E) = 1 :=
by rw dim_eq_one_iff

@[simp] lemma finrank_bot : finrank F (⊥ : intermediate_field F E) = 1 :=
by rw finrank_eq_one_iff

lemma dim_adjoin_eq_one_iff : module.rank F (adjoin F S) = 1 ↔ S ⊆ (⊥ : intermediate_field F E) :=
iff.trans dim_eq_one_iff adjoin_eq_bot_iff

Expand Down

0 comments on commit 08b13ec

Please sign in to comment.