Skip to content

Commit

Permalink
wip
Browse files Browse the repository at this point in the history
  • Loading branch information
Ruben-VandeVelde committed Sep 9, 2024
1 parent 38c98ef commit c62f63e
Showing 1 changed file with 15 additions and 1 deletion.
16 changes: 15 additions & 1 deletion FLT/ForMathlib/Algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -134,7 +134,21 @@ lemma left_distrib' (a b c : A[S⁻¹]) :
simp only [OreLocalization.mul_def]
rcases oreDivAddChar' (a * b) (a * c) (t * s) (u * s) with ⟨r₂, s₂, h₂, q⟩; rw [q]; clear q
rw [oreDiv_eq_iff]
sorry
change ∃ w, _
use s₁ * t * s, s₂ * t * s
simp [mul_add]
constructor
· congr 1
· sorry
calc (s₁ * t * s) • r₂ • (a * c)
_ = (s₁ * t * s : R) • r₂ • (a * c) := by rw [@Submonoid.smul_def]; simp
_ = (r₁ * u * s : R) • r₂ • (a * c) := by rw [h₁]
_ = (r₂ * u * s : R) • r₁ • (a * c) := sorry
_ = (r₂ * ↑(u * s) : R) • r₁ • (a * c) := sorry
_ = (s₂ * ↑(t * s) : R) • r₁ • (a * c) := by rw [h₂]
_ = (s₂ * t * s : R) • r₁ • (a * c) := by simp [mul_assoc]
_ = (s₂ * t * s : R) • (a * r₁ • c) := sorry
· simp [mul_assoc, mul_comm, mul_left_comm]

instance : CommSemiring A[S⁻¹] where
__ := commMonoid
Expand Down

0 comments on commit c62f63e

Please sign in to comment.