Skip to content

Commit 92e1606

Browse files
committed
chore: bump Std to Std#340 (#8104)
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 8befe9d commit 92e1606

File tree

15 files changed

+17
-20
lines changed

15 files changed

+17
-20
lines changed

Archive/MiuLanguage/DecisionNec.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -145,7 +145,7 @@ theorem goodm_of_rule2 (xs : Miustr) (_ : Derivable (M :: xs)) (h₂ : Goodm (M
145145
· cases' h₂ with mhead mtail
146146
contrapose! mtail
147147
rw [cons_append] at mtail
148-
exact (or_self_iff _).mp (mem_append.mp mtail)
148+
exact or_self_iff.mp (mem_append.mp mtail)
149149
#align miu.goodm_of_rule2 Miu.goodm_of_rule2
150150

151151
theorem goodm_of_rule3 (as bs : Miustr) (h₁ : Derivable (as ++ ↑[I, I, I] ++ bs))

Mathlib/Algebra/Group/Commute/Units.lean

Lines changed: 1 addition & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -94,8 +94,7 @@ theorem isUnit_mul_iff (h : Commute a b) : IsUnit (a * b) ↔ IsUnit a ∧ IsUni
9494

9595
@[to_additive (attr := simp)]
9696
theorem _root_.isUnit_mul_self_iff : IsUnit (a * a) ↔ IsUnit a :=
97-
(Commute.refl a).isUnit_mul_iff.trans (and_self_iff _)
98-
-- porting note: `and_self_iff` now has an implicit argument instead of an explicit one.
97+
(Commute.refl a).isUnit_mul_iff.trans and_self_iff
9998
#align is_unit_mul_self_iff isUnit_mul_self_iff
10099
#align is_add_unit_add_self_iff isAddUnit_add_self_iff
101100

Mathlib/Algebra/Hom/Centroid.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -509,7 +509,7 @@ def commRing (h : ∀ a b : α, (∀ r : α, a * r * b = 0) → a = 0 ∨ b = 0)
509509
{ CentroidHom.instRing with
510510
mul_comm := fun f g ↦ by
511511
ext
512-
refine' sub_eq_zero.1 ((or_self_iff _).1 <| (h _ _) fun r ↦ _)
512+
refine' sub_eq_zero.1 (or_self_iff.1 <| (h _ _) fun r ↦ _)
513513
rw [mul_assoc, sub_mul, sub_eq_zero, ← map_mul_right, ← map_mul_right, coe_mul, coe_mul,
514514
comp_mul_comm] }
515515
#align centroid_hom.comm_ring CentroidHom.commRing

Mathlib/Data/Finset/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1658,7 +1658,7 @@ theorem inter_right_comm (s₁ s₂ s₃ : Finset α) : s₁ ∩ s₂ ∩ s₃ =
16581658

16591659
@[simp]
16601660
theorem inter_self (s : Finset α) : s ∩ s = s :=
1661-
ext fun _ => mem_inter.trans <| and_self_iff _
1661+
ext fun _ => mem_inter.trans <| and_self_iff
16621662
#align finset.inter_self Finset.inter_self
16631663

16641664
@[simp]

Mathlib/Data/Finset/Sym.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -100,7 +100,7 @@ theorem sym2_singleton (a : α) : ({a} : Finset α).sym2 = {Sym2.diag a} := by
100100
@[simp]
101101
theorem diag_mem_sym2_mem_iff : (∀ b, b ∈ Sym2.diag a → b ∈ s) ↔ a ∈ s := by
102102
rw [← mem_sym2_iff]
103-
exact mk'_mem_sym2_iff.trans <| and_self_iff _
103+
exact mk'_mem_sym2_iff.trans <| and_self_iff
104104

105105
theorem diag_mem_sym2_iff : Sym2.diag a ∈ s.sym2 ↔ a ∈ s := by simp [diag_mem_sym2_mem_iff]
106106
#align finset.diag_mem_sym2_iff Finset.diag_mem_sym2_iff

Mathlib/Data/Set/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -763,7 +763,7 @@ theorem mem_union (x : α) (a b : Set α) : x ∈ a ∪ b ↔ x ∈ a ∨ x ∈
763763

764764
@[simp]
765765
theorem union_self (a : Set α) : a ∪ a = a :=
766-
ext fun _ => or_self_iff _
766+
ext fun _ => or_self_iff
767767
#align set.union_self Set.union_self
768768

769769
@[simp]
@@ -917,7 +917,7 @@ theorem mem_of_mem_inter_right {x : α} {a b : Set α} (h : x ∈ a ∩ b) : x
917917

918918
@[simp]
919919
theorem inter_self (a : Set α) : a ∩ a = a :=
920-
ext fun _ => and_self_iff _
920+
ext fun _ => and_self_iff
921921
#align set.inter_self Set.inter_self
922922

923923
@[simp]

Mathlib/GroupTheory/Perm/Support.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -142,7 +142,7 @@ theorem nodup_of_pairwise_disjoint {l : List (Perm α)} (h1 : (1 : Perm α) ∉
142142
suffices (σ : Perm α) = 1 by
143143
rw [this] at h_mem
144144
exact h1 h_mem
145-
exact ext fun a => (or_self_iff _).mp (h_disjoint a)
145+
exact ext fun a => or_self_iff.mp (h_disjoint a)
146146
#align equiv.perm.nodup_of_pairwise_disjoint Equiv.Perm.nodup_of_pairwise_disjoint
147147

148148
theorem pow_apply_eq_self_of_apply_eq_self {x : α} (hfx : f x = x) : ∀ n : ℕ, (f ^ n) x = x

Mathlib/Init/CCLemmas.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -31,7 +31,7 @@ theorem and_eq_of_eq_false_right {a b : Prop} (h : b = False) : (a ∧ b) = Fals
3131
h.symm ▸ propext (and_false_iff _)
3232

3333
theorem and_eq_of_eq {a b : Prop} (h : a = b) : (a ∧ b) = a :=
34-
h ▸ propext (and_self_iff _)
34+
h ▸ propext and_self_iff
3535

3636
theorem or_eq_of_eq_true_left {a b : Prop} (h : a = True) : (a ∨ b) = True :=
3737
h.symm ▸ propext (true_or_iff _)
@@ -46,7 +46,7 @@ theorem or_eq_of_eq_false_right {a b : Prop} (h : b = False) : (a ∨ b) = a :=
4646
h.symm ▸ propext (or_false_iff _)
4747

4848
theorem or_eq_of_eq {a b : Prop} (h : a = b) : (a ∨ b) = a :=
49-
h ▸ propext (or_self_iff _)
49+
h ▸ propext or_self_iff
5050

5151
theorem imp_eq_of_eq_true_left {a b : Prop} (h : a = True) : (a → b) = b :=
5252
h.symm ▸ propext ⟨fun h ↦ h trivial, fun h₁ _ ↦ h₁⟩

Mathlib/Init/Logic.lean

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -152,7 +152,6 @@ theorem false_and_iff : False ∧ p ↔ False := iff_of_eq (false_and _)
152152
#align false_and false_and_iff
153153
#align not_and_self not_and_self_iff
154154
#align and_not_self and_not_self_iff
155-
theorem and_self_iff : p ∧ p ↔ p := iff_of_eq (and_self _)
156155
#align and_self and_self_iff
157156

158157
#align or.imp Or.impₓ -- reorder implicits
@@ -187,7 +186,6 @@ theorem false_or_iff : False ∨ p ↔ p := iff_of_eq (false_or _)
187186
#align false_or false_or_iff
188187
theorem or_false_iff : p ∨ False ↔ p := iff_of_eq (or_false _)
189188
#align or_false or_false_iff
190-
theorem or_self_iff : p ∨ p ↔ p := iff_of_eq (or_self _)
191189
#align or_self or_self_iff
192190

193191
theorem not_or_of_not : ¬a → ¬b → ¬(a ∨ b) := fun h1 h2 ↦ not_or.2 ⟨h1, h2⟩

Mathlib/NumberTheory/PythagoreanTriples.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -374,13 +374,13 @@ private theorem coprime_sq_sub_mul_of_even_odd {m n : ℤ} (h : Int.gcd m n = 1)
374374
-- Porting note: norm_num is not enough to close this
375375
field_simp [sq, Int.sub_emod, Int.mul_emod, hm, hn]
376376
apply mt (Int.dvd_gcd (Int.coe_nat_dvd_left.mpr hpm)) hnp
377-
apply (or_self_iff _).mp
377+
apply or_self_iff.mp
378378
apply Int.Prime.dvd_mul' hp
379379
rw [(by ring : n * n = -(m ^ 2 - n ^ 2) + m * m)]
380380
exact hp1.neg_right.add ((Int.coe_nat_dvd_left.2 hpm).mul_right _)
381381
rw [Int.gcd_comm] at hnp
382382
apply mt (Int.dvd_gcd (Int.coe_nat_dvd_left.mpr hpn)) hnp
383-
apply (or_self_iff _).mp
383+
apply or_self_iff.mp
384384
apply Int.Prime.dvd_mul' hp
385385
rw [(by ring : m * m = m ^ 2 - n ^ 2 + n * n)]
386386
apply dvd_add hp1

0 commit comments

Comments
 (0)