Skip to content

Commit bacd2ec

Browse files
tobiasgrosserJamesGallicchiokim-emeric-wieserdigama0
committed
chore: update std4 to b197bd2, catching up to leanprover-community/batteries#427 (#8888)
Co-authored-by: James <jamesgallicchio@gmail.com> Co-authored-by: Scott Morrison <scott.morrison@gmail.com> Co-authored-by: Eric Wieser <wieser.eric@gmail.com> Co-authored-by: Mario Carneiro <di.gama@gmail.com> Co-authored-by: Siddharth Bhat <siddu.druid@gmail.com>
1 parent 7df4ff9 commit bacd2ec

File tree

9 files changed

+15
-22
lines changed

9 files changed

+15
-22
lines changed

Mathlib/Combinatorics/SetFamily/Shadow.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -211,7 +211,7 @@ theorem upShadow_monotone : Monotone (upShadow : Finset (Finset α) → Finset (
211211

212212
/-- `t` is in the upper shadow of `𝒜` iff there is a `s ∈ 𝒜` from which we can remove one element
213213
to get `t`. -/
214-
lemma mem_upShadow_iff : t ∈ ∂⁺ 𝒜 ↔ ∃ s ∈ 𝒜, ∃ a, a ∉ s insert a s = t := by
214+
lemma mem_upShadow_iff : t ∈ ∂⁺ 𝒜 ↔ ∃ s ∈ 𝒜, ∃ a ∉ s, insert a s = t := by
215215
simp_rw [upShadow, mem_sup, mem_image, mem_compl]
216216
#align finset.mem_up_shadow_iff Finset.mem_upShadow_iff
217217

Mathlib/Data/Finset/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1230,7 +1230,7 @@ theorem insert_inj_on (s : Finset α) : Set.InjOn (fun a => insert a s) sᶜ :=
12301230
(insert_inj h).1
12311231
#align finset.insert_inj_on Finset.insert_inj_on
12321232

1233-
theorem ssubset_iff : s ⊂ t ↔ ∃ a, a ∉ sinsert a s ⊆ t := mod_cast @Set.ssubset_iff_insert α s t
1233+
theorem ssubset_iff : s ⊂ t ↔ ∃ a ∉ s, insert a s ⊆ t := mod_cast @Set.ssubset_iff_insert α s t
12341234
#align finset.ssubset_iff Finset.ssubset_iff
12351235

12361236
theorem ssubset_insert (h : a ∉ s) : s ⊂ insert a s :=

Mathlib/Data/Finset/Grade.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -104,13 +104,13 @@ lemma covby_insert (ha : a ∉ s) : s ⋖ insert a s :=
104104

105105
@[simp] lemma erase_covby (ha : a ∈ s) : s.erase a ⋖ s := ⟨erase_ssubset ha, (erase_wcovby _ _).2
106106

107-
lemma _root_.Covby.exists_finset_insert (h : s ⋖ t) : ∃ a, a ∉ s insert a s = t := by
107+
lemma _root_.Covby.exists_finset_insert (h : s ⋖ t) : ∃ a ∉ s, insert a s = t := by
108108
simpa using h.exists_finset_cons
109109

110110
lemma _root_.Covby.exists_finset_erase (h : s ⋖ t) : ∃ a ∈ t, t.erase a = s := by
111111
simpa only [← coe_inj, coe_erase] using h.finset_coe.exists_set_sdiff_singleton
112112

113-
lemma covby_iff_exists_insert : s ⋖ t ↔ ∃ a, a ∉ s insert a s = t := by
113+
lemma covby_iff_exists_insert : s ⋖ t ↔ ∃ a ∉ s, insert a s = t := by
114114
simp only [← coe_covby_coe, Set.covby_iff_exists_insert, ← coe_inj, coe_insert, mem_coe]
115115

116116
lemma covby_iff_card_sdiff_eq_one : t ⋖ s ↔ t ⊆ s ∧ (s \ t).card = 1 := by

Mathlib/Data/List/Perm.lean

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -229,7 +229,6 @@ lemma subperm_iff : l₁ <+~ l₂ ↔ ∃ l, l ~ l₂ ∧ l₁ <+ l := by
229229
obtain ⟨l', h₂⟩ := h₂.exists_perm_append
230230
exact ⟨l₁ ++ l', (h₂.trans (h₁.append_right _)).symm, (prefix_append _ _).sublist⟩
231231

232-
233232
-- This is now in `Std`, but apparently misnamed as `List.subperm_singleton_iff`.
234233
lemma singleton_subperm_iff : [a] <+~ l ↔ a ∈ l :=
235234
fun ⟨s, hla, h⟩ ↦ by rwa [perm_singleton.1 hla, singleton_sublist] at h,

Mathlib/Data/Set/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1179,7 +1179,7 @@ theorem subset_insert_iff_of_not_mem (ha : a ∉ s) : s ⊆ insert a t ↔ s ⊆
11791179
forall₂_congr <| fun _ hb => or_iff_right <| ne_of_mem_of_not_mem hb ha
11801180
#align set.subset_insert_iff_of_not_mem Set.subset_insert_iff_of_not_mem
11811181

1182-
theorem ssubset_iff_insert {s t : Set α} : s ⊂ t ↔ ∃ a, a ∉ s insert a s ⊆ t := by
1182+
theorem ssubset_iff_insert {s t : Set α} : s ⊂ t ↔ ∃ a ∉ s, insert a s ⊆ t := by
11831183
simp only [insert_subset_iff, exists_and_right, ssubset_def, not_subset]
11841184
aesop
11851185
#align set.ssubset_iff_insert Set.ssubset_iff_insert

Mathlib/MeasureTheory/Integral/Marginal.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -103,9 +103,7 @@ theorem _root_.Measurable.lmarginal (hf : Measurable f) : Measurable (∫⋯∫
103103

104104
/-- The marginal distribution is independent of the variables in `s`. -/
105105
theorem lmarginal_congr {x y : ∀ i, π i} (f : (∀ i, π i) → ℝ≥0∞)
106-
-- TODO: change back from `∀ i, i ∉ s →` to `∀ i ∉ s,` after bumping past
107-
-- https://github.com/leanprover/std4/pull/427
108-
(h : ∀ i, i ∉ s → x i = y i) :
106+
(h : ∀ i ∉ s, x i = y i) :
109107
(∫⋯∫⁻_s, f ∂μ) x = (∫⋯∫⁻_s, f ∂μ) y := by
110108
dsimp [lmarginal, updateFinset_def]; rcongr; exact h _ ‹_›
111109

Mathlib/Order/Cover.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -501,7 +501,7 @@ variable {s t : Set α} {a : α}
501501
@[simp] lemma sdiff_singleton_covby (ha : a ∈ s) : s \ {a} ⋖ s :=
502502
⟨sdiff_lt (singleton_subset_iff.2 ha) $ singleton_ne_empty _, (sdiff_singleton_wcovby _ _).2
503503

504-
lemma _root_.Covby.exists_set_insert (h : s ⋖ t) : ∃ a, a ∉ s insert a s = t :=
504+
lemma _root_.Covby.exists_set_insert (h : s ⋖ t) : ∃ a ∉ s, insert a s = t :=
505505
let ⟨a, ha, hst⟩ := ssubset_iff_insert.1 h.lt
506506
⟨a, ha, (hst.eq_of_not_ssuperset $ h.2 $ ssubset_insert ha).symm⟩
507507

@@ -510,7 +510,7 @@ lemma _root_.Covby.exists_set_sdiff_singleton (h : s ⋖ t) : ∃ a ∈ t, t \ {
510510
⟨a, ha, (hst.eq_of_not_ssubset fun h' ↦ h.2 h' $
511511
sdiff_lt (singleton_subset_iff.2 ha) $ singleton_ne_empty _).symm⟩
512512

513-
lemma covby_iff_exists_insert : s ⋖ t ↔ ∃ a, a ∉ s insert a s = t :=
513+
lemma covby_iff_exists_insert : s ⋖ t ↔ ∃ a ∉ s, insert a s = t :=
514514
⟨Covby.exists_set_insert, by rintro ⟨a, ha, rfl⟩; exact covby_insert ha⟩
515515

516516
lemma covby_iff_exists_sdiff_singleton : s ⋖ t ↔ ∃ a ∈ t, t \ {a} = s :=

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
[{"url": "https://github.com/leanprover/std4",
55
"type": "git",
66
"subDir": null,
7-
"rev": "63c387daa50f6d651effa5c7cf47647d5424f850",
7+
"rev": "b197bd218dbab248ad8899404334d41da04f5d13",
88
"name": "std",
99
"manifestFile": "lake-manifest.json",
1010
"inputRev": "main",

test/delaborators.lean

Lines changed: 6 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -45,11 +45,9 @@ variable (P : Nat → Prop) (α : Nat → Type) (s : Set ℕ)
4545
#guard_msgs in
4646
#check ∀ x, x ∈ s → P x
4747

48-
-- TODO: uncomment after bumping past
49-
-- https://github.com/leanprover/std4/pull/427
50-
-- /-- info: ∀ x ∉ s, P x : Prop -/
51-
-- #guard_msgs in
52-
-- #check ∀ x ∉ s,P x
48+
/-- info: ∀ x ∉ s, P x : Prop -/
49+
#guard_msgs in
50+
#check ∀ x ∉ s,P x
5351

5452
/-- info: ∀ x ∉ s, P x : Prop -/
5553
#guard_msgs in
@@ -149,11 +147,9 @@ section existential
149147

150148
variable (s : Set ℕ) (P : ℕ → Prop) (Q : Set ℕ → Prop)
151149

152-
-- TODO: uncomment after bumping past
153-
-- https://github.com/leanprover/std4/pull/427
154-
-- /-- info: ∃ x ∉ s, P x : Prop -/
155-
-- #guard_msgs in
156-
-- #check ∃ x ∉ s, P x
150+
/-- info: ∃ x ∉ s, P x : Prop -/
151+
#guard_msgs in
152+
#check ∃ x ∉ s, P x
157153

158154
/-- info: ∃ x ∉ s, P x : Prop -/
159155
#guard_msgs in

0 commit comments

Comments
 (0)