Skip to content

Commit

Permalink
lint(topology/algebra/order/basic): use finite instead of fintype (
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Jul 10, 2022
1 parent f51aaab commit 4b6ec60
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/topology/algebra/order/basic.lean
Expand Up @@ -1261,7 +1261,7 @@ sometimes Lean fails to unify different instances while trying to apply the depe
e.g., `ι → ℝ`.
-/

variables {ι : Type*} {π : ι → Type*} [fintype ι] [Π i, linear_order (π i)]
variables {ι : Type*} {π : ι → Type*} [finite ι] [Π i, linear_order (π i)]
[Π i, topological_space (π i)] [∀ i, order_topology (π i)] {a b x : Π i, π i} {a' b' x' : ι → α}

lemma pi_Iic_mem_nhds (ha : ∀ i, x i < a i) : Iic a ∈ 𝓝 x :=
Expand All @@ -1277,7 +1277,7 @@ lemma pi_Ici_mem_nhds' (ha : ∀ i, a' i < x' i) : Ici a' ∈ 𝓝 x' :=
pi_Ici_mem_nhds ha

lemma pi_Icc_mem_nhds (ha : ∀ i, a i < x i) (hb : ∀ i, x i < b i) : Icc a b ∈ 𝓝 x :=
pi_univ_Icc a b ▸ set_pi_mem_nhds (set.to_finite _) (λ i _, Icc_mem_nhds (ha _) (hb _))
pi_univ_Icc a b ▸ set_pi_mem_nhds finite_univ (λ i _, Icc_mem_nhds (ha _) (hb _))

lemma pi_Icc_mem_nhds' (ha : ∀ i, a' i < x' i) (hb : ∀ i, x' i < b' i) : Icc a' b' ∈ 𝓝 x' :=
pi_Icc_mem_nhds ha hb
Expand Down

0 comments on commit 4b6ec60

Please sign in to comment.