Skip to content

Commit

Permalink
chore(ring_theory/ideal): some simp attributes (#9487)
Browse files Browse the repository at this point in the history
  • Loading branch information
PatrickMassot committed Oct 2, 2021
1 parent e60dc2b commit a97e86a
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/ring_theory/ideal/operations.lean
Expand Up @@ -400,16 +400,16 @@ mul_one r ▸ hst ▸ (mul_add r s t).symm ▸ ideal.add_mem (I * J) (mul_mem_mu
(mul_mem_mul hri htj)

variables (I)
theorem mul_bot : I * ⊥ = ⊥ :=
@[simp] theorem mul_bot : I * ⊥ = ⊥ :=
submodule.smul_bot I

theorem bot_mul : ⊥ * I = ⊥ :=
@[simp] theorem bot_mul : ⊥ * I = ⊥ :=
submodule.bot_smul I

theorem mul_top : I * ⊤ = I :=
@[simp] theorem mul_top : I * ⊤ = I :=
ideal.mul_comm ⊤ I ▸ submodule.top_smul I

theorem top_mul : ⊤ * I = I :=
@[simp] theorem top_mul : ⊤ * I = I :=
submodule.top_smul I
variables {I}

Expand Down

0 comments on commit a97e86a

Please sign in to comment.