Skip to content

Commit f79581c

Browse files
sgouezelbjoernkjoshanssen
authored andcommitted
start
1 parent 2777305 commit f79581c

File tree

3 files changed

+6
-10
lines changed

3 files changed

+6
-10
lines changed

Mathlib/Algebra/Algebra/Operations.lean

+1-2
Original file line numberDiff line numberDiff line change
@@ -299,11 +299,10 @@ end
299299

300300
section DecidableEq
301301

302-
open scoped Classical
303-
304302
theorem mem_span_mul_finite_of_mem_span_mul {R A} [Semiring R] [AddCommMonoid A] [Mul A]
305303
[Module R A] {S : Set A} {S' : Set A} {x : A} (hx : x ∈ span R (S * S')) :
306304
∃ T T' : Finset A, ↑T ⊆ S ∧ ↑T' ⊆ S' ∧ x ∈ span R (T * T' : Set A) := by
305+
classical
307306
obtain ⟨U, h, hU⟩ := mem_span_finite_of_mem_span hx
308307
obtain ⟨T, T', hS, hS', h⟩ := Finset.subset_mul h
309308
use T, T', hS, hS'

Mathlib/Algebra/BigOperators/Finsupp.lean

+3-4
Original file line numberDiff line numberDiff line change
@@ -565,10 +565,9 @@ theorem Finsupp.sum_apply' : g.sum k x = g.sum fun i b => k i b x :=
565565

566566
section
567567

568-
open scoped Classical
569-
570-
theorem Finsupp.sum_sum_index' : (∑ x ∈ s, f x).sum t = ∑ x ∈ s, (f x).sum t :=
571-
Finset.induction_on s rfl fun a s has ih => by
568+
theorem Finsupp.sum_sum_index' : (∑ x ∈ s, f x).sum t = ∑ x ∈ s, (f x).sum t := by
569+
classical
570+
exact Finset.induction_on s rfl fun a s has ih => by
572571
simp_rw [Finset.sum_insert has, Finsupp.sum_add_index' h0 h1, ih]
573572

574573
end

Mathlib/Algebra/DirectLimit.lean

+2-4
Original file line numberDiff line numberDiff line change
@@ -249,10 +249,10 @@ end functorial
249249

250250
section Totalize
251251

252-
open scoped Classical
253252

254253
variable (G f)
255254

255+
open Classical in
256256
/-- `totalize G f i j` is a linear map from `G i` to `G j`, for *every* `i` and `j`.
257257
If `i ≤ j`, then it is the map `f i j` that comes with the directed system `G`,
258258
and otherwise it is the zero map. -/
@@ -592,8 +592,6 @@ theorem exists_of [Nonempty ι] [IsDirected ι (· ≤ ·)] (z : DirectLimit G f
592592

593593
section
594594

595-
open scoped Classical
596-
597595
open Polynomial
598596

599597
variable {f' : ∀ i j, i ≤ j → G i →+* G j}
@@ -948,8 +946,8 @@ theorem exists_inv {p : Ring.DirectLimit G f} : p ≠ 0 → ∃ y, p * y = 1 :=
948946

949947
section
950948

951-
open scoped Classical
952949

950+
open Classical in
953951
/-- Noncomputable multiplicative inverse in a direct limit of fields. -/
954952
noncomputable def inv (p : Ring.DirectLimit G f) : Ring.DirectLimit G f :=
955953
if H : p = 0 then 0 else Classical.choose (DirectLimit.exists_inv G f H)

0 commit comments

Comments
 (0)