MA243 Notes
MA243 Notes
Let me know if you find any typos in these note, or have any questions!
1
MA243 December 8, 2023 2
||z||
Proof. If y = 0, we get 0 ≤ 0, which is true. Now assume y 6= 0.
||
||x
Recall from A-level maths, if the angle between x and y is θ, then:
y
hx, yi = ||x|| · ||y|| cos(θ). λy
||y||
The result follows since cos θ ≤ 1.
0
For a proof from first principles: Let z := x − hx,yi
||y||2
y. Using bilinearity, y
x, ||y||
λ =
we have
hx, yi hx, yi hx, yi hx, yi hx, yi
2
0 ≤ ||z|| = x − y, x − y = hx, xi − 2 x, y + y, y
||y||2 ||y||2 ||y||2 ||y||2 ||y||2
2 2 2
hx, yi hx, yi hx, yi hx, yi
2 2
= ||x|| − 2 hx, yi + hy, yi = ||x|| − 2 + .
||y||2 ||y||2 ||y|| ||y||
2
Rearranged, this is ||x||2 ≥ hx,yi
||y|| , which gives the required result.
Equality is acheived if and only if ||z|| = 0. Because the norm is non-degenerate ||z|| = 0 if and only if
z = 0, which is the case if and only if
hx, yi
x = λy where λ =
||y||2
To save on notation, we prove that the Euclidean metric is translation invariant.
Lemma 3 (Translation invariance of Euclidean metric). For x, y, z ∈ Rm we have d(x, y) = d(x−z, y−z).
Proof. d(x, y) = ||x − y|| = ||(x − z) − (y − z)|| = d(x − z, y − z).
Lemma 4 (Triangle inequality for the Euclidean metric). For all x, y, x ∈ Rn we have d(x, y) ≤ d(x, z) +
d(z, y), with equality if and only if either z = x, or y − z is a positive scalar multiple of z − x.
We want to show that d(x, y) ≤ d(x, z)+d(z, y). By translation invariance
Triangle inequality in Rm
(Lemma 3), we can replace x, y, z by 0, y0 = y − x and z0 = z − x z
respectively. (because the distances between these points are the same as
the distances between x, y, z. The only reason to change is to cut down ||y
on notation.) So by definition of the metric, it is sufficient to prove
−
z|
||
|
||y0 || ≤ ||z0 || + ||y0 − z0 ||.
−z
This is equivalent to ||y0 ||2 ≤ (||z0 || + ||y0 − z0 ||)2 . Using the Cauchy
||x
y
Schwartz inequality, we have ||z0 ||·||y0 −z0 || ≥ | hz0 , y0 − z0 i | ≥ hz0 , y0 − z0 i.
So
(||z0 || + ||y0 − z0 ||)2 = ||z0 ||2 + 2||z0 || · ||y0 − z0 || + ||y0 − z0 ||2 y||
||x −
x
(1) ≥ ||z0 ||2 + 2| z0 , y0 − z0 | + ||y0 − z0 ||2
||x − y|| ≤ ||x − z|| + ||z − y||
(2) ≥ ||z0 ||2 + 2 z0 , y0 − z0 + ||y0 − z0 ||2
= z0 , z0 + 2 z0 , y0 − z0 + y0 − z0 , y0 − z0 = z0 − (y0 − z0 ), z0 − (y0 − z0 ) = y0 , y0 = ||y0 ||2 ,
as required. Looking at the lines (1) and (2), we see equality is obtained if and only if both: z0 = 0 or
y 0 − z0 is a multiple of z0 , and hz0 , y0 − z0 i is positive. In terms of the original x, y, z, this is if and only
if z − x = 0 or y − z is a positive multiple of z − x.
MA243 December 8, 2023 4
Note that adding points on L does not make sense: If the points are added together using addition in R2 ,
then the result is not on L. We can make addition on L make sense, but we would have to choose a zero.
Definition 4. A motion, also called a Euclidean isometry, is an isometry of a Euclidean space.
Note: A motion does not move.
MA243 December 8, 2023 5
u v
So we can scale by 1/u3 , and so replace (u1 , u2 , u3 ) by (−λ1 , −λ2 , 1) for some λ1 , λ2 ∈ R.
Now multiplying both sides of Equation 3 by (−λ1 , −λ2 , 1)T , we get:
−λ1
(4) x y z −λ2 = 0
1
Rearranged, z = λ1 x + λ2 y. Since (−λ1 , −λ2 , 1) is in the kernel of M , we must have λ1 + λ2 = 1. This
implies that we also have
−λ1
(5) z z z −λ2 = 0
1
Subtracting Equation 5 from Equation 4 gives
−λ1
x−z y−z 0 −λ2 = 0
1
I.e., λ1 (x − z) = −λ2 (y − z) So
|λ1 |||x − z|| = |λ2 |||y − z||.
Picture on desmos (https://www.desmos.com/calculator/lcgtswvxgm):
MA243 December 8, 2023 7
z
(6) d(x, y) = d(x, z) + d(z, y) then d(x, y) = d(x, z) + d(z, y)
x
up to permuting x, y, z.
Proof. Easy case: If y = z, the last term is zero and the others are equal, so the result is true. Since
we are proving the result up to permutaion of the points, we now assume that all points are distinct.
⇐: In the proof of the triangle inequality, we saw that there is equality in (6) if and only if z = x (which
we are now assuming is not the case) or y − z is a positive multiple of z − x. I.e., for some λ ∈ R≥0 ,
y − z = λ(z − x). Rearranged,
(7) y = z − λ(x − z)
which by Lemma 5 implies x, y, z are collinear. (λ happens to be positive, so we don’t yet have ⇒.)
⇒: If x, y, z are collinear, and distinct, then by Lemma 5, and following discussion, we can permute
(rename) x, y, z so that z = λ1 x + λ2 y with λ1 , λ2 ≥ 0, λ1 + λ2 = 1. Then
1 λ1 λ1
y= z − x = z + (z − x)
λ2 λ2 λ2
So y − z is a positive multiple of z − x, and so by Lemma 4 (triangle inequality) Equation (6) holds.
MA243 December 8, 2023 8
4.2. Isometries and Collinearity. We’re going to show that isometries map lines to lines, and use
this to write isometries in terms of matrices. Previously you have seen that vectors and matrices can be
used to define “motions”, but now we show that all isometries have this form.
Isometry in latex tikzpicture: T (c)
[shift = (7,-1), rotate=45]
N (b)
b
T (b)
c N (a)
a Apply an isometry N (c)
Not the result of an isometry
T (a)
Proposition 2. If T is an isometry of Em , then T maps lines to lines, i.e., x, y, z are collinear then
T (x), T (y), T (z) are also collinear. Moreover, if z = (1 − λ)x + λy, then T (z) = (1 − λ)T (x) + λT (y).
Proof. By Propsition 1, and since T is distance preserving,
x, y, z are collinear ⇒ d(x, y) = d(x, z) + d(z, y) after possible permutation of x, y, z
⇒ d(T (x), T (y)) = d(T (x), T (z)) + d(T (z), T (y))
⇒ T (x), T (y), T (z) are collinear by Proposition 1
If λ ∈ [0, 1], the final statement follows from Lemma 5, which implies (1 − λ) : λ = d(z, y) : d(x, z) =
d(T (z), T (y)) : d(T (x), T (z)). Cases λ 6∈ [0, 1] are obtained by reordering x, y, z appropriately.
Definition 7. A linear map is a function L : V → W between two vector spaces over k, such that
L(λv + µw) = λL(v) + µL(w)
for all v, w ∈ V , and for all λ, µ ∈ k. For us, the field k is almost always R; we might extend to C
sometimes.
Definition 8 (Affine maps). A map T : Rn → Rk is affine if it is of the form T (x) = L(x) + b for all
x ∈ Rn for some linear map L : Rn → Rk linear and b ∈ Rk . Note that b = T (0).
From linear algebra, you know that a linear map L : Rn → Rk is described by a k by n matrix A.
Notation: For a k × n matrix A and b ∈ Rk , write T(A,b) for the map
T(A,b) (x) = Ax + b
for x ∈ Rn .
Theorem 2. The set of all invertible affine maps from Rn to Rn ,
n o
Aff(n) := T(A,b) : A is an n × n invertible matrix, b ∈ Rn
is a group. The composition law is
T(A1 ,b1 ) ◦ T(A2 ,b2 ) = T(A1 A2 ,A1 b2 +b1 )
Proof. Exercise.
This group law is denoted
Aff(n) ∼= GL(n) n Rn .
The notation n is just a way of saying that this is a special kind of product, called the “semi direct
product”, not the direct product of two groups.
Exercise: What is the inverse of TA,b ?
Note that the GL(n) is a subgroup of Aff(n) – this is the subgroup of affine maps that fix the origin.
Rn is the subgroup of Aff(n) consisting of the translations.
Exercise: GL(n) and Stab(v) (maps fixing v) are normal subgroups of Aff(n). Show by example that the
subgroup of translations is not normal.
We are going to show that Euclidean isometries are affine. But not just any old affine map.
MA243 December 8, 2023 9
So by Equation ∗, with λ = 12 ,
2λx (F)
1 1
T ( λx + µy ) = T ( 2λx ) + T ( 2µy ).
2 2
λx λx + µy 0, x and 2λx are collinear, with
x 2λx = 2λ x + (1 − 2λ) 0
5.1. Linear isometries have orthogonal matrices. We now find a characterisation of linear
isometries L in terms of the matrix A corresponding to L. We need a result, which expresses the inner
product in terms of the norm:
||x
||x
−
y|
1 1
|
hx, yi = ||x + y||2 − ||x − y||2
4 4
Proposition 4. let L : Rn → Rn be a linear map with matrix A with respect to the standard basis. Then
the following are equivalent:
(1) L is an isometry
(2) ||L(x)|| = ||x|| for all x ∈ Rn , i.e., L is norm preserving
(3) hL(x), L(y)i = hx, yi ∀x, y ∈ Rn i.e., L preserves the inner product
(4) The matrix A is orthogonal, i.e., AT A = I
Proof. (1)⇒(2): Using definition of the metric, defining property of isometries, and linearity of L:
||x|| = d(x, 0) = d(L(x), L(0)) = d(L(x), 0) = ||L(x)||.
(2)⇒(3): This follows from the polarisation inequality in Lemma 6.
(3)⇒(4): Now compute the elements of AT A. By the formula for matrix multiplication
n
X n
X n
X
T T
(A A)ij = (A )ik Akj = Aki Akj = L(ei )k L(ej )k = hL(ei ), L(ej )i
k=1 k=1 k=1
So the entries of AT A are the inner products of the columns of A. Since the ei are the standard basis,
and by hypothesis (3), L preserves the inner product, we have
(
T 1 if i = j
(A A)ij = hL(ei ), L(ej )i = hei , ej i =
0 6 j
if i =
These are the elements of the identity matrix, so A is orthogonal.
(4)⇒ (1): Assuming (4), A is invertible with inverse AT , so L is a bijection. So we just need to check L
is distance preserving. First check that L is norm preserving:
||L(x)||2 = hL(x), L(x)i
= (L(x))T L(x) using matrix notation for dot product
= (Ax)T (Ax) writing L(x) = Ax
= xT AT Ax property of transpose
= xT x since A is orthogonal
= hx, xi , by definition of inner product
= ||x||2 , by definition of norm.
6.1. Isometries of R2 . Recall the matrices for rotations and reflections are defined as follows:
π
2
−θ
π − 2θ
(0, 1) (0, 1)
(− sin θ), cos(θ)) (cos(2θ), sin(2θ))
(cos(θ), sin(θ))
(sin(2θ), − cos(2θ))
θ
θ (1, 0)
θ (1, 0)
Theorem 3. Let T : E2 → E2 be an isometry. Then T (x) = Ax + b where, with respect to the standard
basis, A = Bθ or ρθ and b ∈ R2 , so, T is a rotation or reflection, followed by a translation.
Proof. By Corollary 2, T (x) = Ax + b, with A orthogonal. Write A as a column matrix, A = [v, w].
Then AT A = I implies ||v|| = ||w|| = 1 and hv, wi = 0. Let v = (a, b). Since a2 + b2 = 1, and a, b ∈ R,
for some θ, (a, b) = (cos θ, sin θ). Since hv, wi = 0, and ||w|| = 1, w = ±(−b, a). These give the two
cases.
6.2. Frieze groups: examples of isometries of R2 . The motives in the following frieze patterns
are related by translations, rotations, reflections or glide reflections - can you identify which of these
isometries are involved in the following frieze pattern?
[0, 1]2
sketch of S 1 × [0, 1]2 , representing motions
S1 mapping 0 to a point in [0, 1]2
MA243 December 8, 2023 13
7.1. Extending a linear map from Rn to Cn . In order to prove results about orthogonal matrices,
it’s useful to work over C.
If L : Rn → Rm is a linear map, we can extend it to a map from L : Rn → Rm , by mapping u + iv to
L(u) + iL(v), for u, v ∈ Rn . The matrix describing the transformation is the same.
7.2. sesquilinear inner product. For z,w ∈ Cn we define the sesquilinear inner product by
m
X
hz, wi := z i · wi = z T · w
i=1
Where a is the complex conjugate of a. Note that ||v|| is a real number, and Cauchy-Schwartz still holds.
Lemma 8. If L is a linear isometry of Rn , with matrix A then the extension of L to Cn preserves the
sesquilinear inner product.
Proof. Take z, w ∈ Cn . Then by definition,
hL(z), L(w)i = hAz, Awi = (Az)T · (Aw) = (zT AT )(Aw) = zT AT Aw = zIn w = zT w = hz, wi
7.3. Direct sum. If W is a vector space containing subspaces U and V , then we say W is the direct
sum of U and and V , written W = U ⊕ V if U ∩ V = {0} and every element of W can be written uniquely
as a sum of an element of U and an element of V . E.g., R2 = (Re1 ) ⊕ (Re2 ), where e1 , e2 is a basis for
R2 . We can extend this concept, writing W = U1 ⊕ U2 ⊕ · · · ⊕ Un where Ui are subspaces of a vector
space V , Ui ∩ Uj = {0} for i 6= j, and any element of W can be written uniquely as w = u1 + · · · + un
with ui ∈ Ui .
7.4. Orthogonal complement. If V is a vector space, with a subspace W , then the orthogonal
complement of W in V is the vector subspace:
W ⊥ := {v ∈ V : hv, wi = 0 ∀w ∈ W }
If V is a complex vector space, the inner product here means the sesquilinear inner product. In MA251
you will see a proof that V = W ⊕ W ⊥ . This involves finding an orthonormal basis for W .
Lemma 9. If L is an isometry of Rn , and W is a subspace of Rn such that L(W ) = W , then also
L(W ⊥ ) = W ⊥ . This result also holds for L extended to Cn and W a subspace of Cn .
Proof. Note that since L is an isometry, it is a bijection, so has an inverse L−1 .
9. Lecture 9: Reflections
Definition 11. A hyperplane of Rn is an affine subspace of dimension n − 1, which has the form
Π = V + b = {b + v : v ∈ V } = {b + λ1 v1 + · · · + λm−1 vn−1 |λi ∈ R} = (Rvn )⊥ + b.
= {v ∈ Rn : hv, vn i = β}
where b ∈ Rn and V ⊆ Rn is a vector subspace of dimension n − 1, with basis v1 , . . . , vn−1 , and vn is
orthogonal to V , and β = hvn , bi.
For any c ∈ Rn , Π + c = V + (b + c). (Π is a coset of V as an additive subgroup of Rn .)
Definition 12. For a map T : Rn → Rn , the set of fixed points of T is
Fix(T ) := {x ∈ Rn : T (x) = x}
Definition 13. Let Π be a hyperplane. A reflection in Π is a Euclidean isometry ρΠ : Rn → Rn such
that Fix(ρΠ ) = Π.
P | hP
b
V +
−b
Π=
rp l ane
hype
, vi
re f
lect
|
b+v
ion
viv
b P −b, The reflection ρΠ in the hyperplane Π
b−h
P− exists and is unique, and is given by:
ρΠ : P 7→ P − 2 hP − b, vi v,
where Π = b + (Rv)⊥ and ||v|| = 1
ρΠ (P)
Stuff that I would have covered in week 3 if there was more time
Lemma 11. ρΠ (P) = P − 2 hP − b, vi v, where Π = b + (Rv)⊥ and ||v|| = 1.
Proof. Exercise.
Lemma 12. Given distinct points P and Q ∈ Rn , there exists a reflection ρ with ρ(P) = Q.
Lemma 13. If W = U ⊕ V for some vector spaces U, V and W , and R : U → U is a linear reflection,
then R ⊕ I : W → W is also a reflection.
Proof. This result hold when n = 1, since by Lemma 10 in this case λ = ±1, corresponding to 0 or 1
reflections. Now suppose n > 1. If T 6= I, we’re done. If T 6= I, there is some P 6= 0 with T (P) = Q 6= P.
By Lemma 12, there is a reflection R1 with R1 (Q) = P, so R1 ◦ T fixes P.
Now note that R1 is linear. Not all reflections are linear (they are all affine). In general, a reflection might
be in a plane which is not through the origin. However, in this case, the hyperplane perpendicular to
the line from P to Q and midway between them does pass through the origin. From previous discussion,
the plane that you have to reflect in to get from P to Q is perpendicular to the vector P − Q. I.e., it
is a subspace V , plus some vector b. And the mid point between P and Q is b = (P + Q)/2. So the
mirror plane is V + b. If we can show that P + Q is perpendicular to P − Q, then P + Q lies in the
reflection hyperplane, i.e., b is in V , and so then V + b = V . And reflecting in a hyperplane through
the origin is linear, because the hyperplane is fixed, and so 0 is fixed. We know reflections are affine
(linear plus constant), so if 0 maps to 0, then the reflection is linear. So we just have to check that
hP + Q, P − Qi = 0. But hP + Q, P − Qi = hP, P i − hQ, Qi = ||P ||2 − ||Q||2 . But isometries preserve
length, so since Q = T (P ), we have ||Q|| = ||T (P )|| = ||P ||, so P + Q is perpendicular to P − Q, as
required, and R1 is linear.
Since R1 and T are both linear, R1 ◦ T is linear. And the space W = RP is also fixed by R1 ◦ T . By
Lemma 9 W ⊥ is fixed by R1 ◦ T . By induction (R1 ◦ T )|W ⊥ is a product of at most n − 1 reflections,
(R1 ◦ T )|W ⊥ = R2 ◦ · · · ◦ Rk with k ≤ n. By Lemma 13, these reflections can be considered as reflections
of Rn , which all fix W .
Now we have (Rk ◦ · · · ◦ R2 ◦ R1 ◦ T )|W ⊥ = I|W ⊥ , but since R1 ◦ T |W = I|W , and all Ri are trivial on
W , then also (Rk ◦ · · · ◦ R2 ◦ R1 ◦ T )|W = I|W , So since this map is trivial on both W and W ⊥ , it is the
identity, and so Rk ◦ · · · ◦ R2 ◦ R1 ◦ T = I from which we obtain the result
T = R1 ◦ R2 ◦ · · · ◦ Rk .
Proof. Suppose T (0) 6= 0. Then by Lemma 12, there is some reflection R1 with R1 (T (0)) = 0, so
R1 ◦ T fixes 0, and so is a linear isometry. By Proposition 7, R1 ◦ T is the product of at most n reflections,
and hence T is the product of at most n reflections.
MA243 December 8, 2023 18
Example 3. Let T be a rotation through 90◦ about the origin of R2 . Then T has
0 −1 A2
matrix A = . Take any point which is not fixed, e.g., P = (1, 0). There is
1 0
a reflection mapping (1, 0) to T (1, 0) = (1, 0), which has matrix
0 1
A1 = .
1 0
Now A2 := A1 ◦ A must fix the line (1, 0)R pointwise. The orthogonal complement,
(0, 1)R must also be fixed by A1 ◦ A, so either is the identity, which would imply
A1 = A, which is not the case, or A1 ◦ A is a reflection; we can check A1
0 −1
0 1 1 0
A1 ◦ A = = .
1 0 1 0 0 −1
So A2 is a reflection in the x-axis, and A = A1 ◦ A2 . So T can be acheieved by a
reflection in y = 0 followed by a reflection in x = y. If we choose a different point
P, we will get a different decomposition.
9.1. Classification of isometries of R3 . Using the Normal form theorem, all isometries of R3 are
one of the following:
(1) Translation, by a vector v ∈ R3 .
(2) Rotation about some axis
(3) Twist: A rotation about some axis, followed by a translation in the direction of this axis
(4) Reflection in some plane
(5) Glide: Reflection in a plane, followed by a translation by a vector parallel to the plane.
(6) Rotary relection: Rotation followed by a reflection in a plane perpendicular to the rotation axis.
Proof is omitted. See course text book, [RS].
MA243 December 8, 2023 19
10. Lecture 10: Spherical geometry: The sphere and the spherical metric
Definition 15. The n-dimensional sphere of radius r ≥ 0 is defined by
Srn := {(x1 , . . . , xn+1 ) ∈ Rn+1 : x21 + · · · + x2n+1 = r2 }
= {x ∈ Rn+1 : ||x|| = r}
S n := S1n
Example 4. Spheres S n for n = 0, 1, 2:
−1 1
Definition 16. A spherical line or great circle is the intersection of Srn with a 2-dimensional vector
subspace of Rn+1 .
z
P
Lemma 15. If P and Q ∈ Srn are not antipodal, then there is a
unique great circle containing both of them
O Proof. P and Q have length r and so are non-zero. If
they are not antipodal, then they are not multiples of each
other, since a line Rv only intersects Srn at the points λv
x Q y where ||λv|| = |λ|||v|| = R, which has only two solutions,
λ = ±R/||v||. Thus the only two dimensional vector subspace
containing P and Q is
RP ⊕ RQ = {αP + βQ : α, β ∈ R}
MA243 December 8, 2023 21
z
Definition 18. The spherical distance between two points
P, Q ∈ Srn is the length of the shortest arc of a great circle join-
ing them. We will show that this distance is a metric, called P
the spherical metric, which we can also define by
D E
P, Q
dSrn (P, Q) := r cos−1
θ O
r2
rθ
Proof. Note that the distance on the sphere, in Definition 18, is given in terms of the inner product. By
Proposition 4, any linear isometry of R3 preserves the inner product, so, if we apply a linear isometry of
R3 to the sphere and the points on it, the distances between the points will be unchanged. Therefore, we
may apply an isometry to map the vertices of the triangle to more convenient positions.
P = (0, 0, 1)
γ
β)
Q = (sin(β), 0, cos(β))
sin(
sin(a
)
z-axis
sin(β)
Q = (sin(β), 0, cos(β))
cos(β)
sin(γ)
cos(γ)
β
γ
0
R0 = (cos(a), sin(a), 0)
Q0 = (1, 0, 0)
P = (0, 0, 1)
Q0 = (1, 0, 0)
Q = ( sin β, 0, cos β)
R0 = ( sin a, cos a, 0)
R = (sin γ cos a, sin γ sin a, cos γ)
Cut out the circle, and fold along the vertical axis. As you “open or close” the circle, the angles a, which
is the dihedral angle between the two planes (the plane containing 0, P and R and the plane containing
0, P, Q), and the angle α, which is the angle between the two vectors Q and R will vary.
The minimum possible value of cos(a) is −1, which is obtained before the paper is folded, ie., lying flat,
unfolded. In this case, either α = β + γ, when β + γ ≤ π, or, if β + γ > π, as in this little picture, then
if a = π, we still have cos(α) = cos(β + γ), so β + γ = 2π − α.
β γ
MA243 December 8, 2023 25
Lemma 16. The spherical distance satisfies the triangle inequality. That is, with P, Q, R, α, β, γ and a
as in Proposition 9, we have α ≤ β + γ, with equality, or with α + β + γ = 2π ⇐⇒ a = π. Furthermore,
a = 0 ⇐⇒ α = |β − γ|.
Proof. Since P, Q, R are contained in a vector space V of dimension 3, and so lie on the unit sphere
S2 ∼
= V ∩ S n , it is enough to prove the result for n = 2. We may assume P, Q, R are distinct, since
otherwise the result is easy.
By definition, α, β, γ ∈ [0, π], so sin α, sin β ≥ 0. Since cos a ≥ −1, by
f (x)
Proposition 9 1
(††) cos α = cos β · cos γ + sin β · sin γ · cos a
cos α
≥ cos β · cos γ − sin β · sin γ = cos(β + γ)
Case β + γ ≤ π: By definition, α ∈ [0, π]. On [0, π], cos(x) is strictly x
decreasing, so cos α ≥ cos(β + γ) ⇒ α ≤ β + γ. There is equality in (††) α π β+γ π
2
if and only if cos(a) = −1, which is if and only if a = π.
Case β + γ > π: Since α ∈ [0, π], the inequality is immediate. Equality in
(††) occurs ⇐⇒ a = π, but now β + γ > π so cos(β + γ) = cos(α) ⇐⇒ cos(β+γ)
α = 2π − (β + γ) ⇐⇒ α + β + γ = 2π. The final statement follows −1 f (x) = cos x
similarly, since a = 0 ⇐⇒ cos(α) = cos(β − γ).
Proposition 10. The spherical distance dS n is a metric on S n
Proof. Symmetry follows from symmetry of the inner product on Rn . Non-degeneracy follows since
cos−1 ∈ [0, π], so d(P, Q) = 0 ⇐⇒ hP, Qi = 1, and since ||P|| = ||Q|| = 1, this implies P = Q. The
triangle inequality is proved in Lemma 16.
MA243 December 8, 2023 26
Proposition 11. If T is an isometry of S n , then T extends to a Euclidean isometry Tb of Rn+1 , that is,
there is a Euclidean isometry Tb of Rn+1 , and Tb|S n = T .
Proof. Given an isometry T of S n , define Tb by radial extension, i.e., by
0 if x = 0
(8) Tb(x) =
x
T
||x|| ||x|| if x =
6 0
Tb(x)
x
x
T ||x||
x Tb
||x||
We will show that Tb is an isometry of Rn+1 . First, Tb is a bijection, because Td−1 is the inverse of T
b:
First, note that since T and T −1 n
preserve the S , only 0 maps to 0, so we assume x 6= 0. Then, using
the fact that ||T (y)|| = 1 for all y ∈ S n , we have
x z x
−1 −1 −1
T
d T (x) = T
b d T ||x|| = T ||z||, where z = T ||x||
||x|| ||z|| ||x||
x
= T −1 T ||x||, since ||z|| = ||x||
||x||
x
= ||x|| = x.
||x||
Now we show Tb preserves the inner product on Rn+1 . Since T preserves the spherical metric, for x, y ∈ S n ,
hx, yi = cos (dS n (x, y)) = cos(dS n (T (x), T (y)) = hT (x), T (y)i, so T preserves the inner product restricted
MA243 December 8, 2023 27
We will make some assumptions about area, in particular, assume that you will learn about a rigourous
definition of area in terms of integration in analysis.
Assumptions:
(1) The total surface area of a unit sphere is 4π.
(2) The area of a region of S 2 is invariant under application of θ
any isometry of S 2 .
(3) If X and Y are two non intersecting regions on S 2 , then
area(X ∪ Y ) = area(X) + area(Y )
(4) The segment of a sphere, σθ that lies between two semi- Segment σθ
θ
circular segments of great circles, from P to −P, meeting area 2π 4π
at angle θ has area 2θ.
Let Σθ be the union of σθ and −σθ . So Σθ has area 4θ.
Theorem 8. (Girard’s theorem) Let ∆PQR be a spherical triangle on S 2 , with P, Q, R distinct points,
and such that the interior of ∆PQR does not intersect the great circles which contain the sides of ∆PQR,
and with non-zero area. Then
area (∆PQR) = a + b + c − π
Proof. Notice that area(∆PQR) = area(−∆PQR), since x 7→ −x
is an isometry, and area is preserved by isometries. Also notice
that since we assume that the triangle does not contain any of the
extended edges in its interior, these triangles are disjoint. Notice
P that S 2 is the union of Σa , Σb and Σc , and that
a σa ∩ σb = σb ∩ σc = σa ∩ σb = ∆PQR
and similarly for the images of these areas under x 7→ −x.
b c Let
Q R Sa = σa \ ∆PQR
Sb = σb \ ∆PQR
Sc = σc \ ∆PQR
Then we have a disjoint union:
S 2 = Sa ∪ Sb ∪ Sc ∪ (−Sa ) ∪ (−Sb ) ∪ (−Sc ) ∪ ∆PQR ∪ (−∆PQR).
MA243 December 8, 2023 29
Since we have a disjoint union σa = Sa ∪ ∆PQR), we have area(σθ ) = area(Sθ ) + area(∆PQR), for
θ = a, b, c, so
area(S 2 ) = area(Σa ) + area(Σa ) + area(Σa ) − 4 area(∆PQR)).
By assumption Σθ has area 2θ so
4π = 4(a + b + c) − 4 area(∆PQR),
and the result follows.
Remark: This result also holds if we do not make the restriction that the triangle does not contain
the extensions of its edges in its interior, but then ∆PQR and (−∆PQR) can not be guaranteed to be
disjoint, and so we need to consider several different cases. To save time, I will not prove the general
case, which is not needed for the following result.
Corollary 5. The sum of the angles of a spherical triangle, satisfying the hypothesis of Theorem 8, is
strictly greater than π.
Proof. This follows from Theorem 8.
Schwarz triangles: Suppose ∆ is a spherical triangle, and G
is the group generated by reflections in the sides of ∆. Suppose
these reflections result in a tiling of the sphere – this means that
S 2 = ∪T ∈G T (∆) and T1 (∆)◦ ∩ T2 (∆)◦ 6= ∅ ⇐⇒ T1 = T2 ,
where X ◦ means the interior of X. Then the angles must divide
π. This means that if ∆ tiles S 2 through reflections, then the
angles are πp , πq , πr for positive integers p, q, r such that
1 1 1
+ + >1
p q r
The only solutions are (p, 2, 2), (3, 3, 2), (4, 3, 2), (5, 3, 2). The
later is shown on the right.
(You will probably see more of this if you take the third year course on reflection groups.)
MA243 December 8, 2023 30
Distortion. There is no way to draw the sphere on the plane without some distortion. This gives
rise to various different map projections. (Possibly topic for a second year essay).
Example, of a non isometric map from S 2 to R2 :
imagine a 3D sphere flat version of the sphere
distortion
Hyperbolic space
We will use the model of hyperbolic space defined as follows. An advantage of this definition is that
results are very similar to results in the case of the sphere, just with a “twist”, which is to replace the
usual Euclidean metric hx, yi = xT y with the the Lorentz inner product. We define
−1
0
Jn :=
0 In−1
Note that Jn has n rows and columns and acts on Rn . If x, y ∈ Rn , then xT Jy means xT Jn y.
Definition 20. The Lorentz inner product of two vectors x, y ∈ Rn is defined by:
hx, yiL := −x1 y1 + x2 y2 + x3 y3 + · · · xn yn
= xT Jy
Definition 21. The Lorentz norm of a vector x ∈ Rn is given by
q
||x||L := hx, xiL
We always take this root to be positive or positive imaginary, or zero. WARNING: hx, xi may be negative,
so ||x||L may be imaginary, so is not a norm.
Definition 22. The n-dimensional hyperbolic space is the metric space with underlying set
n o
Hn := (x1 , x2 , . . . , xn+1 ) ∈ Rn+1 : −x21 + x22 + x23 + · · · + x2n+1 = −1 and x1 > 0
n o
= x ∈ Rn+1 : ||x||L = i and x1 > 0
parametrization:
(sinh(t), cosh(t)) 2
1
x2
−4 −2 2 4
−1
−2
−4
ahttps://www.geogebra.org/m/xqnc3sdm
exp(θ)−exp(−θ) exp(θ)+exp(−θ)
sinh(θ) = 2 = −i sin(iθ) cosh(θ) = 2 = cos(iθ)
2 y 2 y
1 1
x x
−2 −1 1 2 −2 −1 1 2
−1 −1
cosh(x)
sinh(x) cosh−1 (x)
−2 −2
2 2
cosh (a) − sinh (a) = 1
erb
le
ng
hyp
th
circle
trigonometric area = θ
θ
θ
area = 2
cos(a + b) = cos(a) cos(b) − sin(a) sin(b) 2
sin(a + b) = sin(a) cos(b) + cos(a) sin(b)
1 1
cos0 (a) = − sin(a) sin0 (a) = cos(a)
2 2 hyperbola
cos (a) + sin (a) = 1
where R2 is given with polar coordinates, and H2 with the Cartesian coordinates of R3 .
Proof. For the first parameterisation, we use
the fact that cosh(t)2 −sinh(t)2 = 1, and that cosh(t)
is strictly increasing on [0, ∞), and symmetric, and
that sinh(−t) = − sinh(t).
For the parameterisation of H2 , this is the inverse
of the projection from R3 given by (x1 , x2 , x3 ) →
(x2 , x3 ). This is a bijection between H2 and R2 , since
for any (x2 , x3 ) there is a unique solution to
(?) − x21 + x22 + x23 = −1 and x1 > 0.
In polar coordinates,
(x2 , x3 ) = (r cos(θ), r sin(θ)),
so (?) becomes
−x21 + r2 = −1, x1 > 0,
the equation for H1 , parametrised by
(x1 , r) = (cosh(t), sinh(t)),
from which the result follows by substitution.
where the norm on the right is the Euclidean norm. So we have by the Cauchy-Schwartz inequality for
the Euclidean norm, Lemma 2,
hx b i2 ≤ ||x
b, y b ||2 ||y
b ||2 = (x1 y1 )2
i.e.,
(10) |1 + x2 y2 + x3 y3 + . . . xn yn | ≤ |x1 y1 |
so
1 + x2 y2 + x3 y3 + . . . xn yn ≤ |x1 y1 | = x1 y1
where we have used that x1 , y1 are positive, since x, y ∈ Hn . Rearranged, we get
hx, yiL = −x1 y1 + x2 y2 + x3 y3 + · · · + xn yn ≤ −1,
which multiplying through by −1 gives the first inequality.
MA243 December 8, 2023 34
on the cone
light like;
||x||L = 0 inside cone:
positive time like H2 = surface of hyperboloid
outside cone: = {x : ||x||L = i, z > 0}
space like region
x2 (“space”)
x3 (“space”)
inside cone:
negative time like Lorentz transoformations fix H2
MA243 December 8, 2023 35
Lemma 21. If T : Rn+1 → Rn+1 is a positive, bijective Lorentz transformation, then T |Hn ∈ Isom(Hn , dHn ).
Proof. Since Hn = {x ∈ Rn : hx, xiL = −1 and x is positive}, T preserves Hn . Since T is bijective,
it has a bijective inverse, which is also a positive Lorentz transformation, and so T |Hn is a bijection.
Distance on Hn is given in terms of the Lorentz inner product, so T is distance preserving. Hence T |Hn
is an isometry.
Euclidean isometries correspond to orthogonal matrices. The Lorentzian analogy is given by:
Definition 26. An n × n real matrix A is Lorentz orthogonal if
−1
T 0
A JA = J :=
0 In−1
Definition 27. The Lorentz group is the group of Lorentz orthogonal n + 1 × n + 1 matrices, denoted
By Lemma 24 this means that the columns of this matrix form a Lorentz orthonormal basis for R2 .
Lorentz translation
cosh γ sinh γ
More generally for any γ ∈ R, Aγ = defines an element of O+ (1, 1), which we can think
sinh γ cosh γ
of as inducing a translation on H1 , since we have
cosh γ sinh γ cosh x sinh γ sinh x + cosh γ cosh x cosh(x + γ)
= =
sinh γ cosh γ sinh x cosh γ sinh x + sinh γ cosh x sinh(x + γ)
The spaces (E1 , dE1 ) and (H1 , dH1 ) are isometric, via the paramterisation x 7→ (sinh x, cosh x).
MA243 December 8, 2023 36
To Do:
Important results we hope to have time to prove later:
• The hyperbolic metric is a metric
• All isometries of Hn are given by elements of O(1, n).
• For a hyperbolic triangle with angles a, b, c and area A, we have A = π − a − b − c.
Things we will actually do:
• Think about lines in the hyperbolic plane, by projection to the plane x1 = 0.
• Think about what are all the isometries of the hyperbolic plane, e.g., translation, rotation, etc
MA243 December 8, 2023 37
Some different views of the hyperbolic line. The hyperbolic line is isometric to R with the
Euclidean metric, under the map t 7→ (cosh(t), sinh(t)). So the simplest way to think about H1 would be
to imagine the usual Euclidean line.
However, H2 can not be embedded smoothly and isometrically in R3 , so is harder to imagine. There are
several common models to work with. Since these models are easier to understand in the analogous one
dimensional cases, the following picture shows 4 different ways to view H1 .
If a plane does not contain a time like vector, it can’t intersect H2 , as for example in this case:
Any plane has the form (Rv)⊥ for some vector v. As long as v is space line, we’re guaranteed that
H2 ∩ (Rv)⊥ is non empty.
You can move the point P in the following geogebra graph to see this for yourself:
https://www.geogebra.org/3d/tu9fgsgj
https://www.geogebra.org/3d/jz6j8cc4
https://www.geogebra.org/3d/jz6j8cc4
step 2:
• Pick a point v in Π that is space like.
• This can be any point, but to be spe-
cific, let’s take a non zero point on
the line where Π intersects the plane
{x1 = 0}.
• Since the two planes Π and {x1 = 0}
are two different two dimensional sub-
spaces of R3 , they must intersect in a
line, which is spanned by some vector
v.
• Since we’ve chosen v = (0, v2 , v3 ) 6=
(0, 0, 0) we must have hv, viL = v22 +
v32 > 0, so v is a space like point on Π
https://www.geogebra.org/3d/faf89g7m
step 4
Note that
• v is space like, and
• u is time like. https://www.geogebra.org/3d/xfsqjeq5
• And there is a continuous function g(t)
from [0, 1] to R mapping t to g(t) :=
hPt , Pt iL
• Since g(0) = hv, viL = α > 0 and
g(0) = hu, uiL = −1, for any value of
a ∈ (0, α), by the intermediate value
theorem, there is some point Pta ∈
[0, 1) with g(ta ) = a, i.e., Pta is a space
like point on Π, and since these points
all have different values of their Lorentz
norm, they are different points. So we
have infinitely many space like points
in Π on this line segment.
We can add the light cone to emphasise that
points on S which are not in the light cone are
space like points on Π.
It’s not that easy to see, but the green area is
the light cone.
https://www.geogebra.org/3d/bxhgbkf2
step 5
Now consider one of the space like points Pt , and
the point x on H.
MA243 December 8, 2023 41
https://www.geogebra.org/3d/uakw5h7p
step 6
• Now consider one of the space like
points Pt , and the point x on H.
• We let the plane Πt be the span of the
vectors x and Pt .
• This plane intersects Π in the subspace
RPt spanned by the vector Pt .
• This is because Π contains Pt , since Pt
was chosen to be on Π and Πt contains
Pt since Πt was defined to be the span
of Pt and x.
• Since RPt ⊂ Π ∩ Πt , we must have
RPt = Π ∩ Πt , since otherwise they
would be equal, but x is in Πt by con-
struction, but is not in L, and thus not
in Π by assumption.
Let Lt = H ∩ Πt . Since this contains the time like point x, it is a line. (not empty).
We’re now going to double check that the Lt lines are the infinite collection of lines we’re looking for. A
projected to R2 picture looks like:
• The lines Lt and L are disjoint, since the intersection is Lt ∩ L = Πt ∩ H ∩ Π ∩ H = Πt ∩ Π ∩ H =
RPt ∩ H = ∅, where the final step is because all points on RPt are space like (or light like at
the origin), but all points on H are time like. So the intersection is empty.
• Now we just have to check that the lines Lt are all different. I.e., if t1 6= t1 then Lt1 6= Lt2 . This
is because the planes Πt1 and Πt2 are different, which is because the vectors Pt1 and Pt2 are not
colinear. If they were colinear, then 0 would be a point on the line through Pt1 and Pt2 which
is the same as the line through u and v by construction. But the origin can’t be on the line
between these points, or else we would be able to write 0 = (1 − t)u + tv for some real number
t, but then u and v would be linearly dependent, but this contradicts one being time like and
the other being space like. since all non-zero multiples of a space like vector are space like, and
similarly for time like vectors.
So, Πt1 and Πt2 are different planes. This implies their intersections with H2 are different,
since if not, they would have two points in common, but any two points will span a plane, unless
they are colinear. Two points on H2 can not be colinear, since for any timelike y, there is a
unique α with αy on H.
So, Lt are different for different t.
Hence there are infinitely many lines Lt which contain x but do not intersect L, as required.
MA243 December 8, 2023 42
https://www.geogebra.org/3d/kkhgqxbg
Hyperbolic isometries of H2
Recall that if A is in O+ (1, n), then A defines an Isometry of Hn . This means that AT JA = J and TA
maps H2 to H2 .
We have not yet proved that all isometies of Hn have this form, but this does turn out to be true.
Almost every Lorentz transformation of H2 is given by one of the following matrices, up to a Lorentz
orthonormal change of basis, i.e., from the standard basis to another Lorentz orthormal basis.
MA243 December 8, 2023 45
Lorentz x3
translation
(by β
on the x2
axis); ori- x2
cosh(β) sinh(β) 0
entation
sinh(β) cosh(β) 0 preserving none (in H2 ) 1, exp(±β)
0 0 1 (direct);
hyperbolic
x3
Lorentz
glide
x2
(in x2 direc-
cosh(β) sinh(β) 0
sinh(β) cosh(β) 0 tion); ori- none (in H2 ) −1, exp(±β)
entation re-
0 0 −1
versing (in-
direct / op-
posite)
x3
rotation
(about the
point
(1, 0, 0));
orientation x2
1 0 0 preserving
0 cos(θ) − sin(θ) one point 1, exp(±iθ)
(direct);
0 sin(θ) cos(θ) elliptic
x3
reflection
(in the line
x2 = 0);
orientation
x2
1 0 0 reversing
0 −1 0 a line 1, 1, −1
(indirect)
0 0 1
Note, each of the above matrices has an eigen value ±1 with an eigen vector which is space-like or
time-like. There are elements of O+ (1, 2) with light-like eigen vectors with eigen value 1, such as
MA243 December 8, 2023 46
3
− 12 −1
These correspond to “parabolic” transformations of H2 , which preserve the orien-
2
1 1
−1. tation, and don’t fix any points of H2 , but whereas a Lorentz translation fixes a
2 2
−1 1 1 space-like vector when extended to R3 , parabolic transformations fix a light-like
vector.
Proof: See [RS, 3.11(page 47) and 3.16(page 58) and B.3 page 189], and the RS erratum
You are expected to be able to
• Check all the above are elements of O+ (1, 2).
• given an element of O+ (1, 2), determine which kind of transformation it corresponds to, e.g., by
considering fixed points and eigen values
• sketch images of simple shapes e.g., lines, points, triangle, under the action of transformations
• compute the composition of hyperbolic isometries
• find the matrix for a hyperbolic isometry given a description
x1
x2
x2
x2 lies on another
hyperbola
MA243 December 8, 2023 47
Loose end: In our description of hyperbolic lines, we used that Lorentz planes are orthogonal to space
like vectors. We will now prove this.
Lemma 26. If w is Lorentz orthongonal to a time-like vector, then w is space like. In other words: If
x ∈ Rn with hx, xiL < 0, and w ∈ Rn \ {0} with hx, wiL = 0, then hw, wiL > 0.
Proof. Let x = (x1 , x2 , . . . , xn ) and w = (w1 , w2 , . . . , wn ). Let x0 = x − x1 e1 and w0 = w − w1 e1 .
Since hx0 , x0 iL ≥ 0 and hx, xiL = −x21 + hx0 , x0 iL , we must have x1 6= 0. If w1 = 0, then since w 6= 0, we
have hw, wiL = hw0 , w0 iL > 0, and we are done. So we may assume w1 6= 0. The vector x1Dw − w1 xE has
zero e1 component. This vector can not be zero, or x1 w = w1 x, but then 0 > hx, xiL = x, wx11 w =
L
x1
w1 hx, wiL = 0, a contradiction. Now
0 ≤ ||x1 w − w1 x||2L = hx1 w − w1 x, x1 w − w1 xiL = x21 hw, wiL + w12 hx, xiL
so
w12
hw, wiL ≥ − hx, xiL > 0.
x21
Examples. In H1 ,
if x = (x1 , x2 ) and w = (w1 , w2 ), then hx, w, iL = 0 means x1 w2 = x2 w2 . For fixed
x this gives an equation for a line through the origin on which w must lie.
x
time-like region
light-like vectors
vectors Lorentz orthogonal
to x lie on this line and are
space-like when x is time-
like. They are orthogonal
space-like region
to Jx.
Jx
MA243 December 8, 2023 49
So we can’t just measure hyperbolic angles by taking the dihedral angle between corresponding planes.
What do we do?
Recall
hP × R, P × Qi
For a spherical triangle: cos(a) = .
||P × R||||P × Q||
By analogy,
hP ×L R, P ×L QiL
(11) For a hyperbolic triangle: cos(a) = .
||P ×L R||L ||P ×L Q||L
It turns out the is invariant under Lorentz transformation. In this expression,
Definition 33. Let J = J3 For x, y ∈ R3 , the Lorentz cross-product of x, y is
−x2 y3 + x3 y2 −e1 e2 e3
x ×L y := J · (x × y) = x3 y1 − x1 y3
= (Jy) × (Jx) = x1 x2 x3
x1 y2 − x2 y1 y1 y2 y3
Note about invariance:
Lemma 27. (Binet–Cauchy identity.) For x, y, z ∈ R3 ,
hx × y, z × wi = hx, zi · hy, wi − hx, wi · hy, zi
The following is a version of this identity for the Lorentz inner product, where the difference with the
usual formula is highlighted in red.
Lemma 28. (Binet–Cauchy identity for Lorentz inner product.) For x, y, z ∈ R3 , we have
hx ×L y, z ×L wiL = − hx, ziL · hy, wiL + hx, wiL · hy, ziL
This result tells us that the expression on the right hand side of Equation 11 is invariant under Lorentz
transformations, since the Lorentz inner product is.
Suppose x = (1, 0, 0), then we have
−e1 e2 e3 −e1 e2 e3
e1 e2 e3
x ×L y = x1 x2 x3 = 1 0 0 = 1 0 0 =x×y
y1 y2 y3 y1 y2 y3 y1 y2 y3
So the angles are the same as in Euclidean space when x = 0.
So, we’re going to translate P to (1, 0, 0) by a Lorentz transformation so we can measure the triangle
angle at P.
MA243 December 8, 2023 50
Lemma 29. For points x, y, z in H2 , there is some Lorentz transformation T such that for some θ, β and
γ we have
Tx = ( 1, 0, 0)
T y = ( cosh(β), sinh(β), 0)
T z = ( cosh(γ), cos(θ) sinh(γ), sin(θ) sinh(γ))
Let
1 0 0 cosh(w) sinh(w) 0
Aφ = 0 cos(φ) − sin(φ) and Bw = sinh(w) cosh(w) 0
0 sin(φ) cos(φ) 0 0 1
These are hyprbolic rotation and translation matrices.
We have A−c x = (cosh(δ), sinh(δ), 0).
And B−δ A−c x = (cosh(0), sinh(0), 0) = (1, 0, 0).
Now we have that B−δ A−c y = (cosh(β), cos(b) sinh(β), sin(b) sinh(β)) for some β and b.
Now apply A−b , which fixes (1, 0, 0), and all the images of x, y, z under T = A−b B−β A−c have the required
form.
α = dHn (z, y)
β = dHn (x, z) x
γ = dHn (x, y)
a = the hyperbolic angle of ∆xyz at x. a
Then β γ
z
cosh α = cosh β · cosh γ − sinh β · sinh γ · cos a α
y
x1
sinh(γ)
cosh(γ),
z = cos(a) sinh(γ),
sin(a) sinh(γ)) sinh(β)
cosh(β),
γ y = sinh(β)
β 0
x = (1, 0, 0)
x2
cut out and fold along x1 axis; a is the angle between the two sides of the paper.
See how the distance between z and y varies as this angle varies.
MA243 December 8, 2023 51
Corollary 8. (The triangle inequality for the hyperbolic metric.) For x, y, z in Hn , we have
Projective geometry
We take 3 views of this subject: Algebraic; Classical perspectivities; Combinatorial/Axiomatic.
In the above picture, the red and white dots at the end of the semi circle correspond to the same line,
y = 0, so these points are identified. Topologically (in topology, you can bend and stretch but not tear
a geometric object), P1 is a circle, which you can see after identifying these points, i.e., stretching round
and gluing together as in the next picture. We can also think of the {x = 1} and {y = 1} projections of
P1 as real lines that together cover the whole of of P1 , as in the following figure:
Every point (a : b : c) in P2 is
represented by unique point
on either
the plane Z = 1, if c 6= 0
the line Z = 0, Y = 1 if c = 0, b 6= 0
the point (1, 0, 0) if b = c = 0
line at ∞
R2
R2 R point
z }| { z }| { z }| {
P2 ∼ {Z = 1} ∪ {Z = 0, Y = 1} ∪ {(1, 0, 0)}
= point at ∞
on line at ∞
You can think of Pn as Rn with a point added at ininfity for every radial direction in Rn .
If you take the hemisphere, and distort it to “glue together” points on opposite
side of the circular boundary on Z = 0, which lie on the same line in R3 , you
get a closed surface. This surface only can be viewed in R3 if it crosses itself.
One model is called “Boy’s surface”.
(Picture from Wikipedia, Ggleizer https://commons.wikimedia.org/wiki/
File:BoysSurfaceKusnerBryant.svg)
v 7→ kv
Definition 35. If V is a vector space V , with a k + 1 dimensional vector subspace W , then the
k-dimensional projective linear subspace P(W ) of P(V ) is the image under π of W in P(V ), that is
P(W ) := {x ∈ P(V ) : x ⊂ W } = π(W )
Warning: the dimension of P(W ) is one less than the dimension of W .
Definition 36. Let W be a subvector space of V .
point if dim(W ) = 1
P(W ) is a line if dim(W ) = 2
plane if dim(W ) = 3
MA243 December 8, 2023 55
(0, 0, 1) (1, 0, 1)
(0, 1, 0) (1, 1, 0)
(0, 0, 0) (1, 0, 0)
The points of P(V ) are given by the one dimensional subspaces of V , which have the form F2 v = {0, v}
for non zero v. So there are 7 of these.
Lines are given by the two dimensional subspaces. Each of these has the form {0, v, w, v + w} for some
v, w ∈ V . For example, the plane P = {(0, 0, 0), (0, 1, 0), (1, 0, 1), (1, 1, 1)}. So, there are 72 ways to
choose two points w and v, but any three non-zero points in P span P , so this would count the planes 3
1 7
times, so the number of planes is 3 2 = 7.
It’s not a coincidence that this is the same as the number of points, since each plane can also be defined
by the vector it is orthogonal to, e.g., P above is orthogonal to (1, 0, 1).
We can draw a diagram showing the points and lines as follows. Right shows labels for the points, with
a vector in V which generates each point in P(V ). This is called the Fano plane.
(0:1:1)
(1:0:1) (0:1:1)
(1:1:1)
23.2. Working in other finite fields. If we work in the field Fp = Z/pZ, which has p elements,
each line in Fnp has elements {0, v, 2v, 3v, . . . , (p − 1)v}, i.e., There are p − 1 non-zero points on any line.
Since Fnp \ {0} has pn − 1 points, this means it contains (pn − 1)/(p − 1) distinct lines, which are points
of Pn−1 (Fp ).
To determine the number of lines in Pn−1 (Fp ), we have to count the number of planes in Fnp . Each plane
is spanned by 2 a basis of non-zero vectors, u, v, which would be (pn − 1)(pn − p) sets of ordered basis,
because once the first, u is choosen, that rules out p choices for v, since v can not be a multiple of u.
but each plane would be counted multiple times. The number of times a plane is counted is equal to the
number of different choices of (ordered) basis. Once one non-zero basis vector is chosen, there are are
p2 − p choices for the remainder, so that’s a total of (p2 − 1)(p2 − p) possible basis. So this means there
n −1)(pn −p)
are (p
(p2 −1)(p2 −p)
lines.
Definition 37. For a vector space V and a subset Σ ⊂ P(V ), the projective cone of Σ is given by
[
Σ
e := L = {v ∈ V : v ∈ L ⊂ V for some line L ∈ Σ},
L∈Σ
i.e., elements of Σ may be considered to be lines, and we take their union.
The linear span or span of Σ is is the smallest projective linear subspace of P(V ) containing Σ,
hΣi := P(span(Σ)),
e
MA243 December 8, 2023 56
f (Q) R
f (R)
Q
P
L1 O
(Next week we will prove this is well defined, i.e., there is a unique intersection point.)
Big result
Perspectivities are the same thing as projective linear maps.
MA243 December 8, 2023 57
semi-circle of representatives of P1
[e2 ]
Standard frame of reference points for P1
[e1 + e2 ]
[e1 ]
Example: Any three distinct points P1 , P2 , P3 in P1 is a frame of reference for P1 , since being distinct
means that P f1 , P
f2 , P
f3 are pairwise linearly independent.
Motivation: Why do we need n + 2 points? This is because n + 2 points is enough to determine a
projecive linear map of Pn , but n + 1 is not. This might be suprising, since the images of n points is
enough to determine a linear map on Rn .
Example: There are infinitely many projective linear maps P1 → P1 with
(1 : 0) 7→ (1 : 0)
(0 : 1) 7→ (0 : 1)
namely, any diagonal map, of the form Example: The radial projec-
4 4
α 0
tion, with centre 0, from the
A= line x = 1 to the line x = 3
0 β 3 3 takes a point with y = 1 to
However, these maps are not all the same a point with y = 3. We can
map, since we have 2 2 paramaterise points on these
A : (1 : 0) 7→ (1 : 0) lines by their y-coordinates.
A : (0 : 1) 7→ (0 : 1) 1 1 If we complete these lines to
form copies of P1 , with point
A : (1 : 1) 7→ (α : β) with parameter y maping to
0 0
x=1
x=3
extended to a map on P1 by allowing the map to apply to (1 : 0). This map has the effect of switching 0
and ∞, thought of as the points (0 : 1) and (1 : 0).
4
0 α
Any map : P1 → P1 , for α, β 6= 0 also −1 0 1 2 3 4
β 0 3
switches (0 : 1) and (1 : 0), and corresponds to y=3
α
t 7→ βt . red line, → blue line,
2
By specifying the image of (1 : 1), the map is {x = 1} → {y = 3}
uniquely determined. 0 7→ ∞
1
The diagram on the right shows a projection from ∞ 7→ 0
{x = 1} to {y = 3}, which corresponds to the map 1 7→ 3
0
7→ 3t
0 3 t
x=1
: P1 → P1 sending (1 : 1) 7→ (3 : 1)
1 0
−1
4 Example: In the figure on the right, we
−1 project from the line {x = 1} to the line
y= {y = − 12 x + 3}.
−1 0 3
2x+ 1 We parameterise {x = 1} by the y coor-
red 3
→ blue 2 2 dinate, and {y = − 21 x + 3} by the x co-
line line ordinate, though we could choose different
0 7→ 6 3
∞ 7→ 0 parameterisations.
1 4
1 7→ 2 With respect to this parameterisation, as
5
a map from P1 to P1 , this map is given
− 12 7→ ∞ 6
6 0 0 6
x=1
The maps in these examples have been written as maps from P1 to P1 , but drawn as maps from R → R.
To extend from R to P1 , we should embed each copy of R in a copy of P1 , which can be acheived by
replacing R2 in these figures by P2 .
Example
In all the above examples, the coordinates could be translated, and we would still have a projection. That
is, you don’t have to project from zero, e.g.:
4 Example: In the figure on the right, we
−1 project from the point (1, 1) from the line
y=
−1 0 3
{x = 2} to the line {y = − 12 x + 3.5}.
x
2 + We parameterise {x = 1} by the y
red → blue 3.5 1
2 coordinate−1, and {y = − 12 x+3.5} by the
line line 2
0 7→ 6 3
x coordinate−1, though we could choose
∞ 7→ 0 different parameterisations.
1 4
1 7→ 2 With respect to this parameterisation, as
O = (1, 1) 5
a map from P1 to P1 , this map is given
− 12 7→ ∞ 6
6 0 0 6
x=1
An examples of a perspectivity
We will show that any three distinct points P1 , P2 , P3 in P1 can be projected onto any other three distinct
points Q1 , Q2 , Q3 . This is called three transitivity of the action of P GL(2) on P1 . This result will
follow from Theorem 13 which shows that there is some A maping the standard frame of reference to
P1 , P2 , P3 , and B maps the standard frame of reference to Q1 , Q2 , Q3 , then BA−1 maps P1 , P2 , P3 to
Q1 , Q2 , Q3 . −1 0 1 2 3 4 5
Example:
How do I project be-
tween these set of
points???
−1 0 1 2 3 4 5
Algebraic description of problem: Let’s just write the algebra first. I.e., suppose we just want a
projecive linear transformation given by a matrix A ∈ P GL(2), and with
TA (0 : 1) = (1 : 1), TA (1 : 1) = (4 : 1), TA (2 : 1) = (5 : 1)
This means we want A so that
0 1 1 4 2 5
A ∼ , A ∼ , A ∼
1 1 1 1 1 1
where ∼ means equal up to non-zero scalar multiplication. i.e., we want some A and some constants
λ1 , λ2 , λ3 with
0 1 1 4 2 5
A = λ1 , A = λ2 , A = λ3
1 1 1 1 1 1
You can either solve this directly, or by working via the standard frame of reference. It’s probably easier
to work via the standard frame of reference.
This means finding A as a composition of two maps, say B −1 and C, with
B −1 C
{0, 1, 2} {∞, 0, 1} {1, 4, 5}
Or, written as projective points, with the inclusion R → P1 given by t 7→ (t : 1).
B −1 C
{(0 : 1), (1 : 1), (2 : 1)} {(1 : 0), (0 : 1), (1 : 1)} {(1 : 1), (4 : 1), (5 : 1)}
(Note, we could also choose to include R1 in P1 as (1 : t), or many other ways; eventually this will lead
to the same formula for the map on R1 .)
Step 1: Find the matrix B:
Since B maps (1 : 0) to (0 : 1) and (0 : 1) to (1 : 1), it has the form:
0 β
B=
α β
Since B maps (1 : 1) to (2 : 1), we require
3
x=0
β : α + β = 2 : 1, i.e., 2(α + β) = β, so
red → blue
β = −2α, and the matrix is
2 line line
0 −2 ∞ 7→ 0
B=
1 −2 y=1 0 7→ 1
1 1 7→ 2
You don’t have to represent this geomet- −3 −2 −1 0 1 2 3
−2
rically, but one interpretation is as on the t 7→ t−2
right, which is a projection from the point 0
O (t : 1) 7→ (−2 : t − 2)
O = (2, 0) between the lines {y = 1} and (t : s) 7→ (−2s : t − 2s)
{x = 0}.
MA243 December 8, 2023 60
0 7→ 1
7 1 2 15 4 5 1 7 4
→
x
TA ((2 : 1)) = = = (5 : 1)
+
1 1 1 3 2 7→ 5
y
3 4
=
2 3
picture is not unique, because we could choose dif- t 7→ 1+7t
1+t
ferent parameterisations, or project from different 1 2
points, to different lines. One example projection
with this algberaic description is to the right. 0 1
In this examples, all we need to know is that a perspectivity is given by a projective linear map. Then
this map can be determined by knowing the images of three points.
You don’t have to draw the pictures. However, if you already know the lines and the point from which
you are projecting, then a diagram may help you find the images of ∞, 0 and 1 (projectively (1 : 0), (0 :
1), (1 : 1)), and so then you only need to compute one matrix, and get A without having to compute two
matrices and multiply.
MA243 December 8, 2023 61
Remarks: (Mostly for after lecture reading, but hopefully there is time in class to write the equations
for the above pictured example, which shows the lines X = Z and X = 2Z, which meet at the point
(0 : 1 : 0).)
Theorem 12 shows that lines always meet in P2 . This can also be seen as a conseqence of the theorem we
proved that spherical lines always intersect, since P2 can be considered to be the sphere S 2 with antipodal
points identified. We can also consider parallel lines in R2 considered as a subset of P2 to meet in the
“line at infinity”, which can be seen by projecting P2 to a different plane: (https://www.geogebra.org/
3d/gnkzhywe)
In this figure, the lines x = 1 and x = 2 are parallel, drawn on a copy of R2 which is the plane Z = 1 in
R3 in this figure. x, y are the coordinates on this plane. These lines are (radial) projections of the planes
X = Z and X = 2Z in R3 , where R3 has coordinates X, Y, Z. These planes project to x = z and x = 2z
on the plane Y = 1, where they meet at (x, y) = (0, 0).
Similarly, lines y = mx + c for fixed m, and varying c, are all parallel in the plane Z = 1. These lines are
projections of Y = mX + cZ in R3 . If we project to X = 1, we get lines y = m + cz, which all meet at
(y, z) = (m, 0). You may also wish to consider these lines as projections to the sphere.
Note: Lines in P3 can be skew; skew lines do not intersect. A corresponding result to Theorem 12 for
P3 would be e.g. that a plane and a line, not contained in that plane, in P3 always intersect in a point,
since their span must be 3 dimensional, so their intersecion has dimension 2 + 1 − 3 = 0, which means
we have a point.
MA243 December 8, 2023 63
26. Lecture 26: Projective frames of reference and projective linear maps
Theorem 13. There is a bijection between projective transformations of Pn and projective frames of
reference of Pn , defined as follows:
φ : P GL(n + 1) → {projective frames of reference}
T 7→ {T ([e1 ]), T ([e2 ]), . . . , T ([en+1 ]), T ([e1 + · · · + en+1 ])}
Proof. We need to show that this map is well defined, injective and surjective.
Well defined: The image of the standard projective frame of reference under T must also be a projective
frame of reference, because T is invertible, so maps any basis of Rn+1 to another basis.
Surjectivity: Suppose we are given a projective frame of reference, P0 , P1 , . . . , Pn+1 . By definition, any
choice of n + 1 of these these are linearly independent in Pn , which means that a choice of lifts, a0 =
P
f0 , a1 = P fn is linearly independent in Rn+1 , and so for any nonzero α0 , . . . , αn , the matrix
f1 , . . . an = P
A with columns αi ai , is invertible.
| | |
...
A = α0 a0 α1 a1 . . . αn an
| | ... |
We know that Aei is the ith column of A, and so for i = 0, . . . , n,
[TA (ei )] = [Aei ] = [αi ai ] = [ai ] = Pi
We want
n
" !#
X
TA ei = Pn+1 .
i=1
Pn Pn Pn
Let an+1P=P ]n+1 , so Pn+1 = [an+1 ]. We have [TA ( i=1 ei )] = [A( i=1 ei )] = [ i=1 αi ai ], so it’s sufficient
to solve ni=1 αi ai = an+1 , i.e., A(α0 , α1 , . . . , αn )T = an+1 . Since A is invertible, set
α0
α1
. = A−1 an+1 .
..
αn
Since a0 , . . . , an+1 is a projective frame of reference, all αi in this solution must be non-zero, since
otherwise there would be a set of n vectors from a0 , . . . , an which was not linearly independent. Hence
A ∈ P GL(n + 1). So φ(TA ) = {P0 , . . . , Pn+1 }. Thus φ is surjective.
Injectivity:
Suppose that φ(TA ) = φ(TB ) for matrices A, B ∈ P GL(n). Then for i = 0, . . . , n, we have
TA (ei ) = TB (ei ),
so the columns of B are multiples of the columns of A, so for some diagonal matrix Diag(β0 , . . . , βn ),
B = A · Diag(β0 , . . . , βn ).
P P
Since φ(TA ) = φ(TB ), we have [TA ( ei )] = [TB ( ei )] so
h X i h X i h X i
A ei = B ei = A βi ei .
ei = A−1 0 = 0,
P P
We know that A isPinvertible, so we can’t have A ei = 0, since then we would have
but we know that ei 6= 0. So for some scalar λ,
X X
λA ei = A βi ei
rearranging, A (λ − βi )ei = 0 and since A is invertible, (λ − βi )ei = 0 which is only possible if λ = βi
P P
for each i = 0, . . . , n, which implies B = λA, and so TA and TB are equal as elements of P GL(n).
MA243 December 8, 2023 64
R = (1 : λ), S = (1 : µ) P =(1:0) P0
Then the cross ratio is
λ in this example {P, Q; R, S} = 2,
{P, Q; R, S} = which is also the case for the pro-
µ jection to {P 0 , Q; R0 , S 0 }.
Warning: The cross ratio will change when the points are permuted, so it depends on the order P, Q, R, S
are given in.
Note: We could also map P, Q, R to the standard projective frame of reference for P1 , then the cross
ratio is the image of S.
It is convenient not to have to make a change of basis in order to compute the cross ratio, so the following
result is useful:
Proposition 14. The cross ratio is well defined. Moreover, if P, Q, R, S are points in P1 , then they can
be considered as lines in R2 . Let L be any line in R2 not through the origin. Let p, q, r, s be the vector
coordinates of the intersections of P, Q, R, S with L. Then
p−r q−s
{P, Q; R, S} = ,
p−s q−r
λv
where the ratios of vectors make sense, because they all lie in the direction of L, and we define v = λ.
P
p
−
r
R
q
−
p
−
r
s
q
− Q
s
L
MA243 December 8, 2023 65
Proof. In order to compute the cross ratio, we apply a change of basis transformation TA , so that
TA (P ) = (1 : 0), TA (Q) = (0 : 1), TA (R) = (1 : λ).
This means that
TA (p) = α(1, 0), TA (q) = β(0, 1), TA (r) = γ(1, λ), TA (s) = δ(1, µ),
and then by definition,
λ
{P, Q; R, S} =
.
µ
Note that any
other change of basis matrix B mapping P and Q to (1 : 0) and (0 : 1) must differ by
a 0
B= A for some a, b. So TB (r) = γ(a, bλ) = γa(1, b/aλ) and TB (s) = γ(a, bµ) = γa(1, b/aµ), so
0 b
the ratio of the second coordinates of r and s is still λ/µ, and so the cross ratio is well defined.
Since p, q, r, s are all chosen to be on a common line L, we must have that for some constants λ1 , λ2 , by
collinearity property of points in R2 , we have
r = λ1 p + (1 − λ1 )q
s = λ2 p + (1 − λ2 )q
Linear maps preserve the relationship between points on lines, so we also have
γ(1, λ) = λ1 α(1, 0) + (1 − λ1 )β(0, 1) = (αλ1 , β(1 − λ1 )) ⇒ λ = (1 − λ1 )/λ1
δ(1, µ) = λ2 α(1, 0) + (1 − λ2 )β(0, 1) = (αλ2 , β(1 − λ2 )) ⇒ µ = (1 − λ2 )/λ2
p−r q−s (1 − λ1 ) λ2 (1 − λ1 )/λ1 λ
= = =
p−s q−r (1 − λ2 ) λ1 (1 − λ2 )/λ2 µ
Example: Does there exist a projective linear map taking points P1 , Q1 , R1 , S1 = 0, 1, 2, 3 to points
P2 , Q2 , R2 , S2 = 0, 1, 7, 8, where the point t ∈ R is interpreted as a point (t : 1) in P1 ?
Solution: The cross ratios are
0−2 1−3 4 0−7 1−8 7×7
{P1 , Q1 ; R1 , S1 } = = 6= {P2 , Q2 ; R2 , S2 } = =
0−3 1−2 3 0−8 1−7 8×6
Since these are not equal, there is no such projective linear map.
Example: Does there exist a projective linear map taking points P1 , Q1 , R1 , S1 = 0, 1, 2, 5 to points
P2 , Q2 , R2 , S2 = 1, 4, 5, 6, where the point t ∈ R is interpreted as a point (t : 1) in P1 ?
Solution: The cross ratios are
0−2 1−5 8 1−5 4−6 8
{P1 , Q1 ; R1 , S1 } = = = {P2 , Q2 ; R2 , S2 } = =
0−5 1−2 5 1−6 4−5 5
So, there is such a map. Note that to compute the map, we only need to consider the images of the first
three points. Given that the cross ratios are equal, the fourth point of one set will automatically get
mapped to the fourth point of the other set.
Example: Determine whether or not there is a projective linear transformation (perspectivity) which
takes the points (1 : 0), (0 : 1), (1 : 1) and (1 : 2) to (1 : 1), (2 : 3), (4 : 5), (1 : 2), preserving the order of
the points. Either prove there is no such map, or find such a map by giving it’s matrix.
Solution: Since the first set of points includes a standard frame of reference, it may be easier just to
compute the matrix which maps (1 : 0), (0 : 1), (1 : 1) to (1 : 1), (2 : 3), (4: 5), and
see where (1 : 2) is
α 2β
mapped to. We can see that the required matrix must have the form A = , and for TA (1 : 1) =
α 3β
2 2
(4 : 5), we must have A = . Now we can check that TA (1 : 2) = (6 : 8) = (3 : 4) 6= (1 : 2), so
2 3
there is no projective linear transformation which takes the points (1 : 0), (0 : 1), (1 : 1) and (1 : 2) to
(1 : 1), (2 : 3), (4 : 5), (1 : 2).
MA243 December 8, 2023 66
We could also have shown this using the cross ratio. By definition, the cross ratio of the first set of
points is {(1 : 0), (0 : 1); (1 : 1), (1 : 2)} = 12 For the second set of points, either we can map the first
3 −2
−1 1
three to (1 : 0), (0 : 1); (1 : 1), which is acheived by A , and we have TA−1 (1 : 2) = =
−2 2 2
−1
= (1 : −2), so {(1 : 1), (2 : 3); (4 : 5), (1 : 2)} = − 21 .
2
We could also compute the cross ratio geometrically, using Proposition 14, as in the following diagram.
Q−S
Q−R
P −S
P −R
S Q R P
R = (4 : 5)
Q = (2 : 3)
S = (1 : 2)
P = (1 : 1)
(0, 0)
−1 23
!
p−r q−s 2 2 −5 1
{P, Q; R, S} = = = =−
p−s q−r 5 1 13 5 4 2
Note, in this computation, I used the line y = 10, but any line would give the same result. I scaled all
points to have the same y = 10 coordinate, e.g., Q = (2 : 3) = (6 23 : 10).
L0
P0 Q0 R0
Proof. Since P, Q, P 0 , Q0 are distinct and on two distinct lines, these points must be a projective
frame of reference, and so by Theorem 13 there is a projective transformation which takes these points
to the standard frame of reference for P2 .
Since a projective linear map preserves lines and intersection points, we can now assume
P = (1 : 0 : 0), Q = (0 : 1 : 0), P 0 = (0 : 0 : 1), Q0 = (1 : 1 : 1).
The picture, from https://www.geogebra.org/3d/zhwkackg shows these points on the projective plane
projected to a sphere. The line through P, Q, R is the “line at infinity”, where the sphere intersects the
z = 0 plane.
Since R ∈ hP, Qi, R, being a linear combination of
P and Q, has the form R = (1 : α : 0), where we
may assume the first coordinate is 1, since it can
not be zero, since R 6= Q. If the first coordinate is
non-zero, by scaling we can set it equal to 1. Since
R0 is on hP 0 , Q0 i, R0 has the form R0 = (1 : 1 : β),
where again, the first coordinates can not be zero,
since R0 6= P 0 .
Now compute the lines and intersection points:
hP, Q0 i = {(λ + µ : µ : µ)}
A = (0 : 1 : 1)
hP 0 , Qi = {(0 : λ2 : µ2 )}
hQ, R0 i = {(µ2 : µ2 + λ2 : µ2 β)}
B = (1 : α + β − αβ : β)
hR, Q0 i = {(µ + λ : µα + λ : λ)}
hP, R0 i = {(µ2 + λ2 : µ2 : µ2 β)}
C = (1 : α : αβ)
hR, P 0 i = {(µ : µα : λ)}
Now note that A, B, C all lie on the line α(1 − β)X −
Y + Z = 0. (Also, (β − αβ)Ae + Ce = B e for obvious
lifts.)
MA243 December 8, 2023 68
P = (1 : 0 : 0) Q = (0 : 1 : 0) R = (1 : α : 0) Z=0
A = (0 : 1 : 1) C = (1 : α + β − αβ : β)
B = (1 : α : αβ)
X=Y
0 0 0
P = (0 : 0 : 1) Q = (1 : 1 : 1) R = (1 : 1 : β)
Z=
βY
Y
=
Z
Quiz: Which of the following is an axiomatic projective plane (with usual concepts of points and lines,
and standard definitions of intersections etc):
P2 (R), P3 (R), R2 , R3 , S 2 , S 1 , R, H2 ?
28.1. Projective planes over finite fields. The simplest way to obtain a finite axiomatic pro-
jective plane is to take P2 (Fq ). Here, Fq is a finite field with q elements, which exists for all q which is
a power of a prime, q = pn , for a prime p. In the case q = p, then Fp = Z/pZ, integers mod p. For
n > 1, Fq = Fp [x]/(f (x)) where f (x) is an irreducible polynomial of degree n. I.e., the quotient of the
polynomial ring Fp [x] by a prime ideal generated by f (x). If you’ve not seen this in algebra, then just
work with the case Fp .
Proposition 15. The projective plane P2 (Fq ) for a field Fq with q elements
• has q 2 + q + 1 points.
• There are q 2 + q + 1 lines.
• Each line contains q + 1 points.
• Each point is on q + 1 lines.
• P2 (Fq ) satisfies the axioms of an axiomatic projective plane.
MA243 December 8, 2023 70
Proof. • There are a total of q 3 − 1 points in (F3q )∗ . Each line in (F3q )∗ contains q − 1 points
(all the points on the line in F3q except 0). Lines in F3q only intersect at 0, so there are
q3 − 1
= q2 + q + 1
q−1
lines in F3q , and so this is the number of points in P2 (Fq ).
• The number of lines is equal to the number of points because any line ` in P2 (Fq ) corresponds
to a plane V through the origin in F3q , that is, ` = π(V ), and V = `.
e
Any plane through the origin, V in F3q corresponds to the line which is orthogonal to the
plane. That is, for some w, we have V = (wFq )⊥ , so there is a correspondance, [w] ↔ π((wFq )⊥ ),
and so the number of lines in P2 (Fq ) equals the number of points. This is part of a more general
duality between points and lines in P2 .
• Each plane V through the origin in (Fq )3 contains q 2 − 1 non-zero points, since if v, u is a basis
for the plane, the points are
V = {au + bv : a, b ∈ Fq }.
Within this plane, any line wFq = {aw : a ∈ Fq } through the origin contains q − 1 non-zero
points. Any two lines in (Fq )3 only intersect at 0. So there are q + 1 = (q 2 − 1)/(q − 1) lines
through the origin in each plane V through the originin F3q , which after projectivising become
q + 1 points (of the form [w] for w ∈ V ) on each line ` = π(V ).
• Each point [w] is contained in q + 1 lines. This is because the plane V = (wFq )⊥ in F3q contains
q + 1 lines through the origin. For each of these lines, vFq , we get a plane V = Span(v, w). Note
that since by definition w and v are orthogonal, they must not lie on the same line. So V is a
plane. Since w ∈ V , we get [w] = π(w) ∈ ` := π(V ). So [w] lies on q + 1 points.
• Since q ≥ 1, we have that axioms (1) and (2) hold for P2 (Fq ). So we just need to check axioms
(3) and (4).
• Axiom (3): If [u] and [v] are two distinct points in P2 (Fq ), then the line containing them both
is given by π(V ) where
V = {au + bv : a, b ∈ Fq }.
V is a 2-dimensional subspace, since u and v are linearly independent, (otherwise [u] = [v]), so
π(V ) is a line. Any line must have the form π(V ) for some 2-dimensional subspace V , and any
such space V must contain u and v if π(V ) contains [u] and [v]. So we have Span(u, v) ⊂ V ,
but since u and v span a 2-dimensional space, and V is 2-dimensional, we know from linear
algebra that Span(u, v) = V . Hence the line containing u and v is unique.
• Axiom (4): If `1 and `2 are two distinct lines, then these must have the form `1 = π((v1 Fq )⊥ )
and `2 = π((v2 Fq )⊥ ) for some vectors v1 , v2 . Then the point given by [v1 × vv2 ] is contained
in both these lines. Any such point [w] in `1 and `2 must be determined by the equations
w · v1 = w · v2 = 0. Since `1 and `2 are distinct, v1 and v2 must be linearly independent,
so the two equations defined by w · v1 = w · v2 = 0 are linearly independent. Since F3q is
3 dimensional, by the rank nullity theorem, the set of solutions to w · v1 = w · v2 = 0 is 1
dimensional, spanned by some vector w, which defines the unique point [w] on `1 and `2 , unique
by the 1-dimensionality of this set of solutions.
Note, in the class we only proved the first point; we may skip the rest due to lack of time. However, you
are expected to know this material.
MA243 December 8, 2023 71
Dobble
The game Dobble was invented based on a finite projective plane. Junior Dobble is isomorphic to P2 (F5 ),
and corresponds to a finite projective plane of order 6. Each line contains 6 points, each point is on 6
lines. In the game as sold, one card is missing.
There are 31 different animal symbols, one for each line in the projective space P2 (F5 ).
I have made the following choice of animal to point of P2 (F5 ). A different choice would correspond to an
element of P GL(3, F5 ), which has order 372000.
animal orthogonal vector animal orthogonal vector
dog (0:0:1) duck (1:1:1)
elephant (1:0:0) parrot (1:1:2)
lion (4:0:1) crocodile (1:1:3)
rabbit (2:0:1) octopus (1:1:4)
tiger (3:0:1) shark (1:1:0)
whale (1:0:1) penguin (3:1:1)
kangaroo (0:1:1) zebra (3:1:2)
rooster (0:3:1) crab (3:1:3)
hippo (0:2:1) sheep (3:1:4)
tortoise (0:4:1) bear (3:1:0)
cow (0:0:1) horse (2:1:1)
dolphin (4:1:0) fish (2:1:2)
gorilla (4:1:1) cat (2:1:3)
snake (4:1:2) camel (2:1:4)
frog (4:1:3) ladybird (2:1:0)
owl (4:1:1)
E.g. the “cat” line, consists of points (x : y : z) with y = 2z − 2x, i.e., (x, y, z) · (2, 1, −2) = 0 meaning
“cat” is the line orthogonal to (2 : 1 : −2) ≡ (2 : 1 : 3) ≡ (4 : 2 : 1).
You can work out the point on P2 (F5 ) corresponding to your card by just considering two of the animals
on it. E.g., the card containing gorilla (4 : 1 : 1) and cat (2 : 1 : 3) must be a point (x : y : z) with
4x + y + z ≡ 2x + y + 3z ≡ 0 mod 5. From this we get x ≡ y + z (from first condition) and then
2y + 2z + y + 3z ≡ 3y ≡ 0 (sub in second) so y ≡ 0, and x ≡ z, so (up to scaling) the point is (1 : 0 : 1).
MA243 December 8, 2023 72
missing card:
dog,cat, camel, fish, ladybird, horse
kangaroo
rooster
elephant
rabbit
whale
tiger
lion
hippo
tortiose
cow
‘‘ d
o g ’’ ∞
li n e a t lines of the form {(αs : t : s) : (t : s) ∈ P1 } lines of the form {(t : αs : s) : (t : s) ∈ P1 }
u in
ng
b
pe
cra
dog, cat, camel, dog, cat, camel, dog, cat, camel,
fish, horse, fish, horse, fish, horse,
ladybird ladybird ladybird
ep
be she
ra
ar
go hin
zeb
s a
lp
og ke
ll
pa ro oc
du
do
ri
fr na
rr
ck
ot
l
c
ow
c od op
i le s
t
sh
u
ar
k
lines of the form {(t : t + αs : s) : (t : s) ∈ P1 } lines of the form {(t : αs − t : s) : (t : s) ∈ P1 } lines of the form {(t : 2t + αs : s) : (t : s) ∈ P1 }
(0 : 1 : 0)
(1 : −1 : 0)
(0,2) (1,2) (2,2) (3,2) (4,2) (1 : 0 : 0)
(1 : 1 : 0)
lines of the form {(t : αs − 2t : s) : (t : s) ∈ P1 } interpret (x, y) as (x : y : 1); all computations mod 5
This shows the 6 families of “parallel” lines. Note that “parallel” here means not meeting in the copy of
F25 ⊂ P2 (F5 ) given by (x, y) 7→ (x : y : 1).
MA243 December 8, 2023 73