Algebra 1 Flashcards
What is a binary operation?
Let S be a set. A binary operation on S is a rule by which any two elements of S can be combined to give another element of S.
We are going to use the symbol * for binary operations. It’s use will mostly be
reserved for when we are talking about a general, non-specified, binary operation.
So given s1, s2 ∈ S we have a further element s1 * s2 ∈ S.
What does it mean for a binary operation to be associative and commutative?
Let S be a set and * a binary operation.
We say that the binary operation * is commutative on S if a * b = b * a for all
a, b ∈ S.
We say that the binary operation * is associative on S if (a * b) * c = a * (b * c)
for all a, b, c ∈ S.
What is a group?
A group is a pair (G, *) where G is a set and * is a binary operation on G, such that the following four properties hold:
(i) (closure) for all a, b ∈ G, a * b ∈ G;
(ii) (associativity) for all a, b, c ∈ G, a * (b * c) = (a * b) * c;
(iii) (existence of the identity element) there is an element e ∈ G such that for all a ∈ G, a * e = e * a = a;
(iv) (existence of inverses) for every a ∈ G, there is an element b ∈ G (called the inverse of a) such that a * b = b * a = e.
What is an Abelian group?
We say that a group (G, *) is abelian if , in addition to properties (i)->(iv) it also satisfes
(v) (commutativity) for all a, b ∈ G, a * b = b * a.
What is GL2(R)?
The group of 2x2 invertible matrices with real entries.
It is a group under matrix multiplication.
Is the identity element of a group Unique?
Let (G, *) be a group. Then (G, *) has a unique identity element.
Proof. Suppose that e and e’ are identity elements. Thus, for all a ∈ G we have
a * e = e * a = a (1)
and
a * e’ = e’ * a = a. (2)
Now let us try evaluating e * e’ . If we let a = e and use (2) we find
e * e’ = e.
But if we let a = e’ and use (1) we find
e * e’ = e’
Thus e = e’. In other words, the identity element is unique.
Is the inverse in a group Unique?
Let (G, *) be a group and let a be an element of G. Then a has a unique inverse.
Proof. Our proof follows the same pattern as the proof that the identity is unique, and you’ll see this pattern again and again during your undergraduate career. Almost all uniqueness proofs follow the same pattern: suppose that there are two of the thing that we want to prove unique; show that these two must be equal; therefore it is unique.
For our proof we suppose that b and c are both inverses of a. We want to show that b = c. By definition of inverse (property (iv) in the definition of a group) we know that
a * b = b * a = e, a * c = c * a = e,
where e is of course the identity element of the group. Thus
b = b * e by (iii) in the definition of a group
= b * (a * c) from the above a * c = e
= (b * a) * c by (ii) in the definition of a group
= e * c from the above b * a = e
= c by (iii) again.
Thus b = c. Since any two inverses of a must be equal, we see that the inverse of a is unique.
What is the inverse of an inverse element of a group?
Let G be a group and a ∈ G. Then (a^−1)^−1 = a.
Proof. We’re being asked to prove that a is the inverse of a^−1. Thinking carefully about what this would mean, we want to show that a^−1a = 1 = aa−1
But this is clearly true because a^−1 is the inverse of a.
What is the inverse of (ab)?
Let G be a group and a, b ∈ G. Then(ab)^−1 = b^−1a^−1.
Proof. We’re being asked to prove that b−1a−1is the inverse of ab. So we want to show that (b^−1^a−1)(ab) = 1 = (ab)(b^−1a^−1).
Now (b^−1a^−1)(ab) = b^−1(a^−1a)b by associativity
= b^−11b
= 1,
and similarly (ab)(b^−1a^−1) = 1.
What is the theorem for a^n (ie composition of a group element n times with itself)?
Let G be a group, and let a ∈ G. Then
1. a^n ∈ G for all n ∈ Z.
2. If n ∈ Z then (a^−1^)n = (a^n)^−1 = a^−n.
3. Moreover, if m, n are integers then (a^m)^n = a^mn, a^ma^n = a^(m+n).
4. Further, if the group G is abelian, a, b ∈ G and n an integer then (ab)^n = a^nb^n.
What is the order of a group element?
The order of an element a in a group G is the smallest positive integer n such that a^n = 1. If there is no such positive integer n, we say a has infinite order.
In a finite group (a group with a finite number of elements) every element must have finite order.
Does every element in a finite group have finite order?
Let G be a finite group and g be an element of G. The g has finite order.
Proof. Suppose g ∈ G has infinite order. Then g0, g1, g2, g3, . . . are elements of
G which are distinct from one another, since if gm = gn for some natural numbers m,n with m < n then e = g0 = g^(m−m) = g^(n−m) and g has finite order.
This cannot happen in a finite group and so g must have finite order
What are the rules for orders of an element?
Let G be a group and g be an element of G.
(i) g has order 1 if and only if g is the identity element.
(ii) Let m be a non-zero integer. Then g^m = 1 if and only if g has finite order d with d | m.
Proof. Let G be a group. Suppose g has order 1. By definition of order, g^1 = 1.
Thus g = 1 which is the identity element of G. Conversely, the identity element
clearly has order 1. This proves (i).
Part (ii) is an `if and only if’ statement. Suppose that g has order d and d | m.
Then g^d = 1 and m = qd where q is an integer. So g^m = (g^d)^q = 1. Let us prove
the converse. Suppose g^m = 1 where m is a non-zero integer. Then g^|m| = 1, and
|m| is a positive integer. Thus g has finite order, which we denote by d. By the
division algorithm which you met in Foundations we may write
m = qd + r, q, r ∈ Z and 0 ≤ r < d.
Now g^d = 1 by definition of order, so 1 = g^m = (g^d)^q · g^r = g^r. But 0 ≤ r < d.
As d is the order, it is the least positive integer such that g^d = 1. So g^r = 1 is
possible with 0 ≤ r < d if and only if r = 0. This happens if and only if m = qd
which is the same as d | m.
What is the order of a Group?
Let G be a group. The order of G is the number of elements that G has. We denote the order of G by |G| or #G.
When does an element have order 2?
Let G be a group and 1 /= g ∈ G. Then g has order 2 if and only if g = g^−1.
By definition, if g has order 2 then g^2 = 1. Multiplying both sides of this on the left by g^−1 gives g = g^−1g^2 = g^−1.
For the converse suppose that g = g^−1. Since g 6= 1, the order of g is not 1.
Multiplying both sides of g = g^−1 on the left by g gives g^2 = gg−1 = 1. Therefore
the order of g is 2.
What is a subgroup?
Let (G, *) be a group. Let H be a subset of G and suppose that (H, *) is also a group. Then we say that H is a subgroup of G (or more formally (H, *) is a subgroup of (G, *)).
For H to be a subgroup of G, we want H to a group with respect to the same binary operation that makes G a group.
What are the subgroup criterion?
Let G be a group. A subset H of G is a subgroup if and only if it satisfies the following three conditions:
(a) 1 ∈ H,
(b) if a, b ∈ H then ab ∈ H,
(c) if a ∈ H then a^−1 ∈ H.
What is Un?
Un = {1, ζ, ζ^2, . . . , ζ^(n−1)}.
That is, Un is the set of n-th roots of unity.
What are proper non-trivial subgroups?
{1} is the trivial subgroup
For a group G, any subgroup not equal to G is a proper subgroup.
What is a Cyclic Subgroup?
Theorem Let G be a group, and let g be an element of G. Write <g> for the set</g>
<g> = {g^n | n ∈ Z} = {. . . , g−2, g−1, 1, g, g2, g3, . . . }.
Then <g> is a subgroup of G.
For the proof just go through the subgroup criterion.
We call <g> the cyclic subgroup of G generated by g.
</g></g></g>
Are cyclic groups abelian?
Theorem Cyclic groups are abelian.
Proof. Let G be a cyclic group generated by g. Let a, b be elements of G. We want to show that ab = ba. Now, a = g^m and b = g^n for some integers m and n.
So, ab = g^mg^n = g^m+n and ba = g^ng^m = g^n+m.
But m + n = n + m (addition of integers is commutative). So ab = ba.
How does the order of a cyclic subgroup relate to the order of its generator?
Let G be a group and let g be an element of finite order n. Then
<g> = {1, g, g2, . . . , gn−1}.
In particular, the order of the subgroup <g> is equal to the order of g.
For the proof show that <g> and {1, g, g2, . . . , gn−1} are equal by showing both are subsets of one another.
=> is trivial
<= use division with remainder
</g></g></g>
Are congruence classes groups?
Let n be an integer satisfying n ≥ 1. Then (Z/nZ, +) is an abelian group.
What is Euclidean Distance?
Let a, b ∈ R^2 so that a = (a1, a2) and b = (b1, b2) where a1, a2, b1, b2 ∈ R. Then the (Euclidean) distance between a and b is given by
|a − b| = sqrt((a1 − b1)^2 + (a2 − b2)^2).
What is an Isometry?
Let f : R^2 → R^2 be a function such that for any a, b ∈ R^2,
|f(a) − f(b)| = |a − b|. Then f is called an isometry of R^2.
This just means that, in an isometry, the distance between any two given points
and the distance between their image points is the same. You may hear such maps
referred to as being distance preserving.
How do isometries commute?
Let f : R^2 → R^2 and g : R^2 → R^2 be isometries of R^2. Then
g ◦ f : R^2 → R^2 is an isometry of R^2
For proof just use definition of isometry with g(f(a)).
What is the special isometry case?
Let f : R^2 → R^2 be a function such that
1. f((0, 0)) = (0, 0) and f((1, 0)) = (1, 0)
2. f is an isometry of R^2
Then f is either the identity map (i.e. f((x, y)) = (x, y) for all x, y ∈ R or it is a reflection in the x-axis (i.e f((x, y)) = (x, −y) for all x, y ∈ R).
When is an isometry a reflection or rotation?
Let f : R^2 → R^2 be a function such that
1. f((0, 0)) = (0, 0)
2. f is an isometry of R^2
Then f is either a rotation about the origin or it is a reflection in the x-axis
followed by a rotation about the origin.
What is the orthogonal group?
The set of isometries of R^2, here identified with C, which fix the origin is a group under composition of functions. We call this group O2(R), the orthogonal group on R^2
What is the special orthogonal group?
The set of isometries, f : R^2 → R^2 of the form f(z) = e^iθz, where R^2 has been identified with C, is a subgroup of O2(R). This is the subgroup of all the rotations about the origin. It is called SO2(R), the special orthogonal group on R^2
.
What is the MAP of a set A?
The set of all functions from A to itself.
What is the SYM of a set A?
The set of all bijections from A to itself.