Skip to content

Commit

Permalink
cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
semorrison committed Mar 13, 2024
1 parent 33eaca8 commit 7bdcaa7
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 5 deletions.
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicTopology/SimplicialSet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -291,7 +291,7 @@ def primitiveTriangle {n : ℕ} (i : Fin (n+4))
use Fin.last (n+3)
simp only [hₙ.ne, not_false_eq_true, Fin.zero_eta, zero_add, true_and]
intro j
fin_cases j <;> simp [Fin.ext_iff] <;> omega
fin_cases j <;> simp [Fin.ext_iff]
· use 0
simp only [h₀.ne', not_false_eq_true, true_and]
intro j
Expand Down
7 changes: 3 additions & 4 deletions Mathlib/Data/Nat/Factorization/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -891,16 +891,15 @@ def recOnPrimeCoprime {P : ℕ → Sort*} (h0 : P 0) (hp : ∀ p n : ℕ, Prime
@[elab_as_elim]
def recOnMul {P : ℕ → Sort*} (h0 : P 0) (h1 : P 1) (hp : ∀ p, Prime p → P p)
(h : ∀ a b, P a → P b → P (a * b)) : ∀ a, P a :=
let rec hp'' (p n : ℕ) (hp' : Prime p) : P (p ^ n) :=
let rec
/-- The predicate holds on prime powers -/
hp'' (p n : ℕ) (hp' : Prime p) : P (p ^ n) :=
match n with
| 0 => h1
| n + 1 => h _ _ (hp'' p n hp') (hp p hp')
recOnPrimeCoprime h0 hp'' fun a b _ _ _ => h a b
#align nat.rec_on_mul Nat.recOnMul

--Adaptation note: as of `nightly-2024-03-11`, this is exposed to docBlame
attribute [nolint docBlame] recOnMul.hp''

/-- For any multiplicative function `f` with `f 1 = 1` and any `n ≠ 0`,
we can evaluate `f n` by evaluating `f` at `p ^ k` over the factorization of `n` -/
theorem multiplicative_factorization {β : Type*} [CommMonoid β] (f : ℕ → β)
Expand Down

0 comments on commit 7bdcaa7

Please sign in to comment.