Skip to content

Commit

Permalink
Delete now-unused code
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies committed Dec 20, 2024
1 parent a0946a5 commit fbfdecb
Show file tree
Hide file tree
Showing 11 changed files with 5 additions and 143 deletions.
10 changes: 2 additions & 8 deletions LeanCamCombi.lean
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ import LeanCamCombi.GrowthInGroups.ApproximateSubgroup
import LeanCamCombi.GrowthInGroups.Chevalley
import LeanCamCombi.GrowthInGroups.ChevalleyComplex
import LeanCamCombi.GrowthInGroups.Constructible
import LeanCamCombi.GrowthInGroups.ConstructiblePrimeSpectrum
import LeanCamCombi.GrowthInGroups.ConstructibleSetData
import LeanCamCombi.GrowthInGroups.Lecture1
import LeanCamCombi.GrowthInGroups.Lecture2
Expand Down Expand Up @@ -47,24 +46,18 @@ import LeanCamCombi.Mathlib.Analysis.Convex.Exposed
import LeanCamCombi.Mathlib.Analysis.Convex.Extreme
import LeanCamCombi.Mathlib.Analysis.Convex.Independence
import LeanCamCombi.Mathlib.Analysis.Convex.SimplicialComplex.Basic
import LeanCamCombi.Mathlib.Analysis.Normed.Group.Basic
import LeanCamCombi.Mathlib.Combinatorics.Additive.VerySmallDoubling
import LeanCamCombi.Mathlib.Combinatorics.Schnirelmann
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Basic
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Density
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Finite
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Maps
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Multipartite
import LeanCamCombi.Mathlib.Combinatorics.SimpleGraph.Subgraph
import LeanCamCombi.Mathlib.Data.Finset.Basic
import LeanCamCombi.Mathlib.Data.Finset.PosDiffs
import LeanCamCombi.Mathlib.Data.Finset.Powerset
import LeanCamCombi.Mathlib.Data.List.DropRight
import LeanCamCombi.Mathlib.Data.Multiset.Basic
import LeanCamCombi.Mathlib.Data.Nat.Defs
import LeanCamCombi.Mathlib.Data.Prod.Lex
import LeanCamCombi.Mathlib.Data.Set.Basic
import LeanCamCombi.Mathlib.Data.Set.Pairwise.Lattice
import LeanCamCombi.Mathlib.Data.Set.Pointwise.SMul
import LeanCamCombi.Mathlib.GroupTheory.OrderOfElement
import LeanCamCombi.Mathlib.LinearAlgebra.AffineSpace.FiniteDimensional
Expand All @@ -76,16 +69,17 @@ import LeanCamCombi.Mathlib.Order.Partition.Finpartition
import LeanCamCombi.Mathlib.Order.RelIso.Group
import LeanCamCombi.Mathlib.Probability.ProbabilityMassFunction.Constructions
import LeanCamCombi.Mathlib.RingTheory.FinitePresentation
import LeanCamCombi.Mathlib.RingTheory.Ideal.Span
import LeanCamCombi.Mathlib.RingTheory.LocalRing.ResidueField.Ideal
import LeanCamCombi.Mathlib.RingTheory.Localization.Integral
import LeanCamCombi.Mathlib.RingTheory.PrimeSpectrum
import LeanCamCombi.MetricBetween
import LeanCamCombi.MinkowskiCaratheodory
import LeanCamCombi.Multipartite
import LeanCamCombi.PhD.VCDim.Basic
import LeanCamCombi.PlainCombi.LittlewoodOfford
import LeanCamCombi.PlainCombi.OrderShatter
import LeanCamCombi.PlainCombi.VanDenBergKesten
import LeanCamCombi.PosDiffs
import LeanCamCombi.SimplicialComplex.Basic
import LeanCamCombi.SimplicialComplex.Finite
import LeanCamCombi.SimplicialComplex.Pure
Expand Down
5 changes: 2 additions & 3 deletions LeanCamCombi/GrowthInGroups/Chevalley.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ import LeanCamCombi.Mathlib.Algebra.Polynomial.Degree.Lemmas
import LeanCamCombi.Mathlib.AlgebraicGeometry.PrimeSpectrum.Basic
import LeanCamCombi.Mathlib.Data.Prod.Lex
import LeanCamCombi.Mathlib.RingTheory.FinitePresentation
import LeanCamCombi.Mathlib.RingTheory.Ideal.Span
import LeanCamCombi.Mathlib.RingTheory.Localization.Integral
import LeanCamCombi.GrowthInGroups.PrimeSpectrumPolynomial

Expand Down Expand Up @@ -51,15 +50,15 @@ lemma foo_induction
obtain ⟨n, e, rfl⟩ : ∃ (n : ℕ) (e : Fin (n + 1) → R[X]), I = Ideal.span (Set.range e) := by
obtain ⟨s, rfl⟩ := hI
exact ⟨s.card, Fin.cons 0 (Subtype.val ∘ s.equivFin.symm),
by simp [← Set.union_singleton, Ideal.span_union]⟩
by simp [← Set.union_singleton, Ideal.span_union, Set.singleton_zero]⟩
clear hI
set v : (Fin (n + 1) → WithBot ℕ) ×ₗ Prop := toLex
(degree ∘ e, ¬ ∃ i, IsUnit (e i).leadingCoeff ∧ ∀ j, e j ≠ 0
(e i).degree ≤ (e j).degree) with hv
clear_value v
induction' v using WellFoundedLT.induction with v H_IH generalizing R
by_cases he0 : e = 0
· rw [he0, Set.range_zero, Ideal.span_singleton_zero]; exact hP₁ R
· simpa [he0, Set.range_zero, Set.singleton_zero] using hP₁ R
cases subsingleton_or_nontrivial R
· rw [Subsingleton.elim (Ideal.span (Set.range e)) ⊥]; exact hP₁ R
simp only [funext_iff, Pi.zero_apply, not_forall] at he0
Expand Down
44 changes: 0 additions & 44 deletions LeanCamCombi/GrowthInGroups/ConstructiblePrimeSpectrum.lean

This file was deleted.

13 changes: 0 additions & 13 deletions LeanCamCombi/Mathlib/Analysis/Normed/Group/Basic.lean

This file was deleted.

18 changes: 0 additions & 18 deletions LeanCamCombi/Mathlib/Data/Finset/Basic.lean

This file was deleted.

19 changes: 0 additions & 19 deletions LeanCamCombi/Mathlib/Data/Finset/Powerset.lean

This file was deleted.

8 changes: 0 additions & 8 deletions LeanCamCombi/Mathlib/Data/Set/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,12 +6,4 @@ variable {α : Type*} {s : Set α} {a : α}
lemma diff_inter_right_comm (s t u : Set α) : s \ t ∩ u = (s ∩ u) \ t := by
ext; simp [and_right_comm]

lemma insert_diff_self_of_mem (ha : a ∈ s) : insert a (s \ {a}) = s := by aesop

lemma insert_erase_invOn :
InvOn (insert a) (fun s ↦ s \ {a}) {s : Set α | a ∈ s} {s : Set α | a ∉ s} :=
fun _s ha ↦ insert_diff_self_of_mem ha, fun _s ↦ insert_diff_self_of_not_mem⟩

@[gcongr] protected alias ⟨_, GCongr.singleton_subset_singleton⟩ := singleton_subset_singleton

end Set
24 changes: 0 additions & 24 deletions LeanCamCombi/Mathlib/Data/Set/Pairwise/Lattice.lean

This file was deleted.

5 changes: 0 additions & 5 deletions LeanCamCombi/Mathlib/RingTheory/Ideal/Span.lean

This file was deleted.

File renamed without changes.
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2023 Yaël Dillies. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yaël Dillies
-/
import Mathlib.Combinatorics.SetFamily.Compression.Down
import Mathlib.Algebra.Group.Pointwise.Finset.Basic
import Mathlib.Combinatorics.SetFamily.Compression.Down
import Mathlib.Data.Finset.Sups
import Mathlib.Order.Interval.Set.OrdConnected
import Mathlib.Order.UpperLower.Basic
Expand Down

0 comments on commit fbfdecb

Please sign in to comment.