From 674152da7a98acf3cc177438dd7180b10ca102ce Mon Sep 17 00:00:00 2001
From: leanprover-community-bot In 1. The Irrationality of the Square Root
+
@@ -77,7 +77,7 @@ 2. Fundamental Theorem of Algebra
(hf : 0 < Polynomial.degree f)
:
3. The Denumerability of the Rational N
+
@@ -117,7 +117,7 @@ 4. Pythagorean Theorem
(p3 : P)
:
7. Law of Quadratic Reciprocity
(hpq : p ≠ q)
:
10. Euler’s Generalization of Fermat
(h : Nat.Coprime x n)
:
+
@@ -191,7 +191,7 @@ 11. The Infinitude of Primes Nat.exists_infinite_primes
(n : ℕ)
:
-
+
@@ -202,7 +202,7 @@ 14. Euler’s Summation of 1 + (1/2)^2
-
+
@@ -235,7 +235,7 @@ 15. Fundamental Theorem of Integral Ca
(hb : Filter.Tendsto f (nhds b ⊓ MeasureTheory.Measure.ae MeasureTheory.volume) (nhds c))
:
+
15. Fundamental Theorem of Integral Ca
(f'int : IntervalIntegrable f' MeasureTheory.volume a b)
:
17. De Moivre’s Formula
(z : ℂ)
:
18. Liouville’s Theorem and the Cons
(lx : Liouville x)
:
-
+
@@ -313,7 +313,7 @@ 19. Four Squares Theorem Nat.sum_four_squares
(n : ℕ)
:
-
+
@@ -330,7 +330,7 @@ 20. All Primes (1 mod 4) Equal the Sum
(hp : p % 4 ≠ 3)
:
-
+
@@ -341,7 +341,7 @@ 22. The Non-Denumerability of the Cont
+
@@ -359,7 +359,7 @@ 23. Formula for Pythagorean Triples {z : ℤ}
:
-
+
@@ -389,7 +389,7 @@ 25. Schroeder-Bernstein Theorem
(hg : Function.Injective g)
:
26. Leibniz’s Series for Pi
27. Sum of the Angles of a Triangle
(h3 : p3 ≠ p1)
:
34. Divergence of the Harmonic Series
+
@@ -484,7 +484,7 @@ 35. Taylor’s Theorem (hf' : DifferentiableOn ℝ (iteratedDerivWithin n f (Set.Icc x₀ x)) (Set.Ioo x₀ x))
:
35. Taylor’s Theorem (hf' : DifferentiableOn ℝ (iteratedDerivWithin n f (Set.Icc x₀ x)) (Set.Ioo x₀ x))
:38. Arithmetic Mean/Geometric Mean
(hz : ∀ (i : ι), i ∈ s → 0 ≤ z i)
:
39. Solutions to Pell’s Equation
(hp : x * x - Pell.d a1 * y * y = 1)
:
-
+
pell.eq_pell
, d
is defined to be a*a - 1
for an arbitrary a > 1
.
Automatically generated when defining the natural numbers
@@ -1142,7 +1142,7 @@it also has a generalized version, by showing that every Euclidean domain is a unique factorization domain, and showing that the integers form a Euclidean domain.
@@ -1377,7 +1377,7 @@Without some kind of structure like this -- for example, if students receive bare .lean files -- it is hard to ensure that they all use the same version of Lean. It is also a good way to provide a "library" file or files -containing basic definitions, tactics, and such that are useful for your course. -[if you are distributing bare Lean files...]
+containing basic definitions, tactics, and such that are useful for your course.These projects are often hosted on GitHub. Students are asked to clone the project, or create a Codespace or Gitpod instance, at the start of the course.