Merge pull request #68 from HEPLean/Mathematics
feat: Create a Mathematics directory
This commit is contained in:
commit
84df731c16
7 changed files with 5 additions and 10 deletions
|
@ -1,6 +1,5 @@
|
|||
import HepLean.AnomalyCancellation.Basic
|
||||
import HepLean.AnomalyCancellation.GroupActions
|
||||
import HepLean.AnomalyCancellation.LinearMaps
|
||||
import HepLean.AnomalyCancellation.MSSMNu.B3
|
||||
import HepLean.AnomalyCancellation.MSSMNu.Basic
|
||||
import HepLean.AnomalyCancellation.MSSMNu.HyperCharge
|
||||
|
@ -59,7 +58,8 @@ import HepLean.FlavorPhysics.CKMMatrix.Relations
|
|||
import HepLean.FlavorPhysics.CKMMatrix.Rows
|
||||
import HepLean.FlavorPhysics.CKMMatrix.StandardParameterization.Basic
|
||||
import HepLean.FlavorPhysics.CKMMatrix.StandardParameterization.StandardParameters
|
||||
import HepLean.GroupTheory.SO3.Basic
|
||||
import HepLean.Mathematics.LinearMaps
|
||||
import HepLean.Mathematics.SO3.Basic
|
||||
import HepLean.SpaceTime.AsSelfAdjointMatrix
|
||||
import HepLean.SpaceTime.Basic
|
||||
import HepLean.SpaceTime.CliffordAlgebra
|
||||
|
|
|
@ -3,7 +3,7 @@ Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
|
|||
Released under Apache 2.0 license.
|
||||
Authors: Joseph Tooby-Smith
|
||||
-/
|
||||
import HepLean.AnomalyCancellation.LinearMaps
|
||||
import HepLean.Mathematics.LinearMaps
|
||||
import Mathlib.Algebra.Module.Basic
|
||||
import Mathlib.LinearAlgebra.FiniteDimensional
|
||||
/-!
|
||||
|
|
|
@ -224,7 +224,6 @@ lemma ubOnePhaseCond_shift_solution {V : CKMMatrix} (h1 : a + f = - arg [V]ub)
|
|||
subst hc
|
||||
ring
|
||||
|
||||
-- rename
|
||||
lemma fstRowThdColRealCond_holds_up_to_equiv (V : CKMMatrix) :
|
||||
∃ (U : CKMMatrix), V ≈ U ∧ FstRowThdColRealCond U:= by
|
||||
obtain ⟨τ, hτ⟩ := V.uRow_cross_cRow_eq_tRow
|
||||
|
@ -319,7 +318,6 @@ lemma ubOnePhaseCond_hold_up_to_equiv_of_ub_one {V : CKMMatrix} (hb : ¬ ([V]ud
|
|||
ring
|
||||
rw [hcs, hUV, cs_of_ud_us_zero hb]
|
||||
|
||||
|
||||
lemma cd_of_fstRowThdColRealCond {V : CKMMatrix} (hb : [V]ud ≠ 0 ∨ [V]us ≠ 0)
|
||||
(hV : FstRowThdColRealCond V) :
|
||||
[V]cd = (- VtbAbs ⟦V⟧ * VusAbs ⟦V⟧ / (VudAbs ⟦V⟧ ^2 + VusAbs ⟦V⟧ ^2)) +
|
||||
|
|
|
@ -4,7 +4,7 @@ Released under Apache 2.0 license.
|
|||
Authors: Joseph Tooby-Smith
|
||||
-/
|
||||
import HepLean.SpaceTime.LorentzGroup.Basic
|
||||
import HepLean.GroupTheory.SO3.Basic
|
||||
import HepLean.Mathematics.SO3.Basic
|
||||
import Mathlib.Topology.Constructions
|
||||
/-!
|
||||
# Rotations
|
||||
|
|
|
@ -22,11 +22,9 @@ The functions
|
|||
|
||||
are adapted from `batteries.scripts.check_imports.lean` authored by Joe Hendrix.
|
||||
|
||||
|
||||
-/
|
||||
open Lean System Meta
|
||||
|
||||
|
||||
/-- Recursively finds files in directory. -/
|
||||
partial def addModulesIn (recurse : Bool) (prev : Array Name) (root : Name := .anonymous)
|
||||
(path : FilePath) : IO (Array Name) := do
|
||||
|
@ -41,7 +39,6 @@ partial def addModulesIn (recurse : Bool) (prev : Array Name) (root : Name := .a
|
|||
r := r.push (root.mkStr mod)
|
||||
pure r
|
||||
|
||||
|
||||
/-- Compute imports expected by `HepLean.lean` by looking at file structure. -/
|
||||
def expectedHepLeanImports : IO (Array Name) := do
|
||||
let mut needed := #[]
|
||||
|
@ -80,7 +77,7 @@ def checkMissingImports (modData : ModuleData) (reqImports : Array Name) :
|
|||
def main (_ : List String) : IO UInt32 := do
|
||||
initSearchPath (← findSysroot)
|
||||
let mods : Name := `HepLean
|
||||
let imp : Import := {module := mods}
|
||||
let imp : Import := {module := mods}
|
||||
let mFile ← findOLean imp.module
|
||||
unless (← mFile.pathExists) do
|
||||
throw <| IO.userError s!"object file '{mFile}' of module {imp.module} does not exist"
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue