Skip to content

Commit

Permalink
style: remove three double spaces (#11186)
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg authored and utensil committed Mar 26, 2024
1 parent 30452cd commit 951decc
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 4 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Data/List/NodupEquivFin.lean
Original file line number Diff line number Diff line change
Expand Up @@ -19,8 +19,8 @@ Given a list `l`,
sending `⟨x, hx⟩` to `⟨indexOf x l, _⟩`;
* if `l` has no duplicates and contains every element of a type `α`, then
`List.Nodup.getEquivOfForallMemList` defines an equivalence between
`Fin (length l)` and `α`; if `α` does not have decidable equality, then
`List.Nodup.getEquivOfForallMemList` defines an equivalence between `Fin (length l)` and `α`;
if `α` does not have decidable equality, then
there is a bijection `List.Nodup.getBijectionOfForallMemList`;
* if `l` is sorted w.r.t. `(<)`, then `List.Sorted.getIso` is the same bijection reinterpreted
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/Submonoid/Membership.lean
Original file line number Diff line number Diff line change
Expand Up @@ -371,7 +371,7 @@ theorem card_le_one_iff_eq_bot : card S ≤ 1 ↔ S = ⊥ :=

@[to_additive]
lemma eq_bot_iff_card : S = ⊥ ↔ card S = 1 :=
by rintro rfl; exact card_bot, eq_bot_of_card_eq⟩
by rintro rfl; exact card_bot, eq_bot_of_card_eq⟩

end Submonoid

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Order/PartialSups.lean
Original file line number Diff line number Diff line change
Expand Up @@ -61,7 +61,7 @@ theorem partialSups_succ (f : ℕ → α) (n : ℕ) :
#align partial_sups_succ partialSups_succ

lemma partialSups_iff_forall {f : ℕ → α} (p : α → Prop)
(hp : ∀ {a b}, p (a ⊔ b) ↔ p a ∧ p b) : ∀ {n : ℕ}, p (partialSups f n) ↔ ∀ k ≤ n, p (f k)
(hp : ∀ {a b}, p (a ⊔ b) ↔ p a ∧ p b) : ∀ {n : ℕ}, p (partialSups f n) ↔ ∀ k ≤ n, p (f k)
| 0 => by simp
| (n + 1) => by simp [hp, partialSups_iff_forall, ← Nat.lt_succ_iff, ← Nat.forall_lt_succ]

Expand Down

0 comments on commit 951decc

Please sign in to comment.