Skip to content

Commit

Permalink
feat: port Topology.ContinuousFunction.Ideals (#4852)
Browse files Browse the repository at this point in the history
Co-authored-by: Moritz Firsching <firsching@google.com>
Co-authored-by: Jireh Loreaux <loreaujy@gmail.com>
  • Loading branch information
3 people committed Jun 14, 2023
1 parent 0f286b0 commit 9c20de9
Show file tree
Hide file tree
Showing 3 changed files with 474 additions and 3 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -2800,6 +2800,7 @@ import Mathlib.Topology.ContinuousFunction.Basic
import Mathlib.Topology.ContinuousFunction.Bounded
import Mathlib.Topology.ContinuousFunction.CocompactMap
import Mathlib.Topology.ContinuousFunction.Compact
import Mathlib.Topology.ContinuousFunction.Ideals
import Mathlib.Topology.ContinuousFunction.LocallyConstant
import Mathlib.Topology.ContinuousFunction.Ordered
import Mathlib.Topology.ContinuousFunction.Polynomial
Expand Down
9 changes: 6 additions & 3 deletions Mathlib/Topology/Algebra/Ring/Ideal.lean
Expand Up @@ -38,10 +38,13 @@ theorem Ideal.coe_closure (I : Ideal R) : (I.closure : Set R) = closure I :=
rfl
#align ideal.coe_closure Ideal.coe_closure

@[simp]
theorem Ideal.closure_eq_of_isClosed (I : Ideal R) [hI : IsClosed (I : Set R)] : I.closure = I :=
-- porting note: removed `@[simp]` because we make the instance argument explicit since otherwise
-- it causes timeouts as `simp` tries and fails to generated an `IsClosed` instance.
-- we also `alignₓ` because of the change in argument type
-- https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/!4.234852.20heartbeats.20of.20the.20linter
theorem Ideal.closure_eq_of_isClosed (I : Ideal R) (hI : IsClosed (I : Set R)) : I.closure = I :=
SetLike.ext' hI.closure_eq
#align ideal.closure_eq_of_is_closed Ideal.closure_eq_of_isClosed
#align ideal.closure_eq_of_is_closed Ideal.closure_eq_of_isClosedₓ

end Ring

Expand Down

0 comments on commit 9c20de9

Please sign in to comment.