Skip to content

Commit

Permalink
Bump mathlib
Browse files Browse the repository at this point in the history
  • Loading branch information
YaelDillies committed Dec 27, 2023
1 parent d798edd commit 1041902
Show file tree
Hide file tree
Showing 7 changed files with 3 additions and 72 deletions.
2 changes: 0 additions & 2 deletions LeanAPAP.lean
Original file line number Diff line number Diff line change
Expand Up @@ -33,15 +33,13 @@ import LeanAPAP.Mathlib.Analysis.NormedSpace.Ray
import LeanAPAP.Mathlib.Analysis.SpecialFunctions.Pow.Real
import LeanAPAP.Mathlib.Data.Complex.Basic
import LeanAPAP.Mathlib.Data.Complex.Order
import LeanAPAP.Mathlib.Data.Finset.Basic
import LeanAPAP.Mathlib.Data.Finset.Card
import LeanAPAP.Mathlib.Data.Finset.Image
import LeanAPAP.Mathlib.Data.Finset.Pi
import LeanAPAP.Mathlib.Data.Finset.Pointwise
import LeanAPAP.Mathlib.Data.Finset.Powerset
import LeanAPAP.Mathlib.Data.Fintype.Basic
import LeanAPAP.Mathlib.Data.Fintype.BigOperators
import LeanAPAP.Mathlib.Data.Fintype.Card
import LeanAPAP.Mathlib.Data.Fintype.Lattice
import LeanAPAP.Mathlib.Data.Fintype.Pi
import LeanAPAP.Mathlib.Data.FunLike.Basic
Expand Down
14 changes: 0 additions & 14 deletions LeanAPAP/Mathlib/Data/Finset/Basic.lean

This file was deleted.

7 changes: 1 addition & 6 deletions LeanAPAP/Mathlib/Data/Fintype/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,11 +7,6 @@ namespace Finset
@[simp]
lemma filter_mem_univ (s : Finset α) : univ.filter (· ∈ s) = s := by simp [filter_mem_eq_inter]

-- @[simp] --TODO: Unsimp `finset.univ_unique`
lemma singleton_eq_univ [Subsingleton α] (a : α) : ({a} : Finset α) = univ := by
ext b; simp [Subsingleton.elim a b]
-- TODO: Unsimp `Finset.univ_unique`

end Finset

instance {s : Set α} [DecidablePred (· ∈ s)] : Decidable s.Subsingleton :=
decidable_of_iff (∀ a ∈ s, ∀ b ∈ s, a = b) Iff.rfl
11 changes: 0 additions & 11 deletions LeanAPAP/Mathlib/Data/Fintype/Card.lean

This file was deleted.

2 changes: 1 addition & 1 deletion LeanAPAP/Prereqs/AddChar/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -293,7 +293,7 @@ noncomputable instance instFintype [Finite G] : Fintype (AddChar G R) :=

@[simp] lemma card_addChar_le [Fintype G] : card (AddChar G R) ≤ card G := by
simpa only [FiniteDimensional.finrank_fintype_fun_eq_card] using
FiniteDimensional.fintype_card_le_finrank_of_linearIndependent (AddChar.linearIndependent G R)
(AddChar.linearIndependent G R).fintype_card_le_finrank

end IsROrC

Expand Down
1 change: 0 additions & 1 deletion LeanAPAP/Prereqs/Dissociation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ import Mathlib.Data.Fintype.Pi
import Mathlib.Data.Set.Pointwise.Basic
import LeanAPAP.Mathlib.Algebra.BigOperators.Basic
import LeanAPAP.Mathlib.Algebra.GroupPower.Basic
import LeanAPAP.Mathlib.Data.Finset.Basic
import LeanAPAP.Mathlib.Data.Finset.Powerset
import LeanAPAP.Mathlib.Data.Fintype.Basic
import LeanAPAP.Mathlib.Data.Set.Function
Expand Down
38 changes: 1 addition & 37 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -49,47 +49,11 @@
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"rev": "be0b59d276020004e21109a79cab71f259755349",
"rev": "7a302eb97c8a48fef146f33f55eb00fc7a5541e3",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
"inherited": false,
"configFile": "lakefile.lean"},
{"url": "https://github.com/xubaiw/CMark.lean",
"type": "git",
"subDir": null,
"rev": "0077cbbaa92abf855fc1c0413e158ffd8195ec77",
"name": "CMark",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/fgdorais/lean4-unicode-basic",
"type": "git",
"subDir": null,
"rev": "280d75fdfe7be8eb337be7f1bf8479b4aac09f71",
"name": "UnicodeBasic",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/hargonix/LeanInk",
"type": "git",
"subDir": null,
"rev": "2447df5cc6e48eb965c3c3fba87e46d353b5e9f1",
"name": "leanInk",
"manifestFile": "lake-manifest.json",
"inputRev": "doc-gen",
"inherited": true,
"configFile": "lakefile.lean"},
{"url": "https://github.com/leanprover/doc-gen4",
"type": "git",
"subDir": null,
"rev": "86d5c219a9ad7aa686c9e0e704af030e203c63a1",
"name": "«doc-gen4»",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
"inherited": false,
"configFile": "lakefile.lean"}],
"name": "LeanAPAP",
"lakeDir": ".lake"}

0 comments on commit 1041902

Please sign in to comment.