Skip to content

Commit

Permalink
fix(ring_theory/algebra): Fix typo "algbera" (#4337)
Browse files Browse the repository at this point in the history
Introduced in e57fc3d
  • Loading branch information
eric-wieser committed Sep 30, 2020
1 parent 05038da commit 9921fe7
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 5 deletions.
2 changes: 1 addition & 1 deletion src/field_theory/splitting_field.lean
Expand Up @@ -601,7 +601,7 @@ theorem splits_iff (f : polynomial α) [is_splitting_field α β f] :
let ⟨x, hxs, hxy⟩ := finset.mem_image.1 (by rwa multiset.to_finset_map at hy) in
hxy ▸ subalgebra.algebra_map_mem _ _),
λ h, @ring_equiv.to_ring_hom_refl α _ ▸
ring_equiv.trans_symm (ring_equiv.of_bijective _ $ algebra.bijective_algbera_map_iff.2 h) ▸
ring_equiv.trans_symm (ring_equiv.of_bijective _ $ algebra.bijective_algebra_map_iff.2 h) ▸
by { rw ring_equiv.to_ring_hom_trans, exact splits_comp_of_splits _ _ (splits β f) }⟩

theorem mul (f g : polynomial α) (hf : f ≠ 0) (hg : g ≠ 0) [is_splitting_field α β f]
Expand Down
8 changes: 4 additions & 4 deletions src/ring_theory/algebra.lean
Expand Up @@ -1163,15 +1163,15 @@ eq_top_iff.2 $ λ x, mem_top
def to_top : A →ₐ[R] (⊤ : subalgebra R A) :=
by refine_struct { to_fun := λ x, (⟨x, mem_top⟩ : (⊤ : subalgebra R A)) }; intros; refl

theorem surjective_algbera_map_iff :
theorem surjective_algebra_map_iff :
function.surjective (algebra_map R A) ↔ (⊤ : subalgebra R A) = ⊥ :=
⟨λ h, eq_bot_iff.2 $ λ y _, let ⟨x, hx⟩ := h y in hx ▸ subalgebra.algebra_map_mem _ _,
λ h y, algebra.mem_bot.1 $ eq_bot_iff.1 h (algebra.mem_top : y ∈ _)⟩

theorem bijective_algbera_map_iff {R A : Type*} [field R] [semiring A] [nontrivial A] [algebra R A] :
theorem bijective_algebra_map_iff {R A : Type*} [field R] [semiring A] [nontrivial A] [algebra R A] :
function.bijective (algebra_map R A) ↔ (⊤ : subalgebra R A) = ⊥ :=
⟨λ h, surjective_algbera_map_iff.1 h.2,
λ h, ⟨(algebra_map R A).injective, surjective_algbera_map_iff.2 h⟩⟩
⟨λ h, surjective_algebra_map_iff.1 h.2,
λ h, ⟨(algebra_map R A).injective, surjective_algebra_map_iff.2 h⟩⟩

/-- The bottom subalgebra is isomorphic to the base ring. -/
def bot_equiv_of_injective (h : function.injective (algebra_map R A)) :
Expand Down

0 comments on commit 9921fe7

Please sign in to comment.