Skip to content

Commit

Permalink
tiny simplification of gcd_rec proof
Browse files Browse the repository at this point in the history
  • Loading branch information
dwrensha committed Jul 1, 2021
1 parent 5ef8f93 commit fd1c568
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions Mathlib/Data/Nat/Gcd.lean
Original file line number Diff line number Diff line change
Expand Up @@ -144,8 +144,7 @@ Exists.elim H (λ l H1 => by rw [Nat.mul_assoc] at H1
theorem gcd_rec (m n : ℕ) : gcd m n = gcd (n % m) m :=
match m with
| 0 => by have := (mod_zero n).symm
simp
exact this
rwa [gcd_zero_right]
| pm + 1 => by simp [gcd_succ]

theorem gcd.induction
Expand Down

0 comments on commit fd1c568

Please sign in to comment.