Skip to content

Commit

Permalink
chore(Algebra/DirectLimit): drop some DecidableEq assumptions (#11288)
Browse files Browse the repository at this point in the history
... by moving `variable [DecidableEq ι]` to `section`s.
  • Loading branch information
urkud committed Mar 11, 2024
1 parent 0235206 commit cbd8ede
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions Mathlib/Algebra/DirectLimit.lean
Expand Up @@ -42,7 +42,7 @@ variable {R : Type u} [Ring R]

variable {ι : Type v}

variable [dec_ι : DecidableEq ι] [Preorder ι]
variable [Preorder ι]

variable (G : ι → Type w)

Expand Down Expand Up @@ -84,6 +84,7 @@ nonrec theorem DirectedSystem.map_map [DirectedSystem G fun i j h => f i j h] {i
#align module.directed_system.map_map Module.DirectedSystem.map_map

variable (G)
variable [DecidableEq ι]

/-- The direct limit of a directed system is the modules glued together along the maps. -/
def DirectLimit : Type max v w :=
Expand Down Expand Up @@ -365,11 +366,11 @@ end Module

namespace AddCommGroup

variable [∀ i, AddCommGroup (G i)]
variable [DecidableEq ι] [∀ i, AddCommGroup (G i)]

/-- The direct limit of a directed system is the abelian groups glued together along the maps. -/
def DirectLimit (f : ∀ i j, i ≤ j → G i →+ G j) : Type _ :=
@Module.DirectLimit ℤ _ ι _ _ G _ _ fun i j hij => (f i j hij).toIntLinearMap
@Module.DirectLimit ℤ _ ι _ G _ _ (fun i j hij => (f i j hij).toIntLinearMap) _
#align add_comm_group.direct_limit AddCommGroup.DirectLimit

namespace DirectLimit
Expand Down Expand Up @@ -708,8 +709,7 @@ variable {G f f'}
theorem of.zero_exact_aux [Nonempty ι] [IsDirected ι (· ≤ ·)] {x : FreeCommRing (Σi, G i)}
(H : (Ideal.Quotient.mk _ x : DirectLimit G fun i j h => f' i j h)
= (0 : DirectLimit G fun i j h => f' i j h)) :
∃ j s,
∃ H : ∀ k : Σi, G i, k ∈ s → k.1 ≤ j,
∃ j s, ∃ H : ∀ k : Σ i, G i, k ∈ s → k.1 ≤ j,
IsSupported x s ∧
lift (fun ix : s => f' ix.1.1 j (H ix ix.2) ix.1.2) (restriction s x) = (0 : G j) := by
refine' span_induction (Ideal.Quotient.eq_zero_iff_mem.1 H) _ _ _ _
Expand Down

0 comments on commit cbd8ede

Please sign in to comment.