Skip to content

Commit

Permalink
chore(Algebra/FilterBasis): use mul_mem_mul to improve readability (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Dec 22, 2023
1 parent eb17faa commit 0328934
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Topology/Algebra/FilterBasis.lean
Expand Up @@ -251,7 +251,7 @@ instance (priority := 100) isTopologicalGroup (B : GroupFilterBasis G) :
rcases mul U_in with ⟨V, V_in, hV⟩
refine' ⟨V, V, ⟨V_in, V_in⟩, _⟩
intro a b a_in b_in
exact hV ⟨a, b, a_in, b_in, rfl⟩
exact hV <| mul_mem_mul a_in b_in
· rw [basis.tendsto_iff basis]
intro U U_in
simpa using inv U_in
Expand Down Expand Up @@ -318,7 +318,7 @@ instance (priority := 100) isTopologicalRing {R : Type u} [Ring R] (B : RingFilt
rcases B.mul U_in with ⟨V, V_in, hV⟩
refine' ⟨V, V, ⟨V_in, V_in⟩, _⟩
intro a b a_in b_in
exact hV ⟨a, b, a_in, b_in, rfl⟩
exact hV <| mul_mem_mul a_in b_in
· intro x₀
rw [basis.tendsto_iff basis]
intro U
Expand Down

0 comments on commit 0328934

Please sign in to comment.