Skip to content

Commit

Permalink
add some comments (for example mathlib PR numbers)
Browse files Browse the repository at this point in the history
  • Loading branch information
kbuzzard committed Jan 7, 2025
1 parent e66b7d1 commit 35bb6ec
Show file tree
Hide file tree
Showing 3 changed files with 10 additions and 1 deletion.
1 change: 1 addition & 0 deletions FLT/Mathlib/NumberTheory/NumberField/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,7 @@ import Mathlib.NumberTheory.NumberField.Basic

open scoped NumberField

-- Mathlib PR #20544
theorem Rat.ringOfIntegersEquiv_eq_algebraMap (z : 𝓞 ℚ) :
(Rat.ringOfIntegersEquiv z : ℚ) = algebraMap (𝓞 ℚ) ℚ z := by
obtain ⟨z, rfl⟩ := Rat.ringOfIntegersEquiv.symm.surjective z
Expand Down
2 changes: 2 additions & 0 deletions FLT/NumberField/InfiniteAdeleRing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,13 +6,15 @@ open NumberField

variable [Algebra K (InfiniteAdeleRing L)] [IsScalarTower K L (InfiniteAdeleRing L)]

-- TODO should be →A[K]
/-- The canonical map from the infinite adeles of K to the infinite adeles of L -/
def NumberField.InfiniteAdeleRing.baseChange :
InfiniteAdeleRing K →ₐ[K] InfiniteAdeleRing L :=
sorry

open scoped TensorProduct

-- TODO should be ≃A[L]
/-- The canonical `L`-algebra isomorphism from `L ⊗_K K_∞` to `L_∞` induced by the
`K`-algebra base change map `K_∞ → L_∞`. -/
def NumberField.InfiniteAdeleRing.baseChangeIso :
Expand Down
8 changes: 7 additions & 1 deletion FLT/NumberField/IsTotallyReal.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,11 @@
import Mathlib.NumberTheory.NumberField.Basic
import Mathlib.Data.Complex.Basic

class NumberField.IsTotallyReal (F : Type*) [Field F] [NumberField F] : Prop where
namespace NumberField

-- #20542
class IsTotallyReal (F : Type*) [Field F] [NumberField F] : Prop where
isTotallyReal : ∀ τ : F →+* ℂ, ∀ f : F, ∃ r : ℝ, τ f = r

instance : IsTotallyReal ℚ where
isTotallyReal τ q := ⟨q, by simp⟩

0 comments on commit 35bb6ec

Please sign in to comment.