You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
Copy file name to clipboardexpand all lines: theories/Algebra/AbGroups/TensorProduct.v
+4-4
Original file line number
Diff line number
Diff line change
@@ -222,7 +222,7 @@ Proof.
222
222
apply Hin.
223
223
Defined.
224
224
225
-
(** As a commonly occuring special case of the above induction principle, we have the case when the predicate in question is showing that two group homomorphisms out of the tensor product are homotopic. In order to do this, it suffices to show it only for simple tensors. The homotopy is closed under addition, so we don't need to hypothesise anything else. *)
225
+
(** As a commonly occurring special case of the above induction principle, we have the case when the predicate in question is showing that two group homomorphisms out of the tensor product are homotopic. In order to do this, it suffices to show it only for simple tensors. The homotopy is closed under addition, so we don't need to hypothesise anything else. *)
226
226
Definition ab_tensor_prod_ind_homotopy {A B G : AbGroup}
227
227
{f f' : ab_tensor_prod A B $-> G}
228
228
(H : forall a b, f (tensor a b) = f' (tensor a b))
@@ -361,7 +361,7 @@ Proof.
361
361
napply grp_homo_op.
362
362
Defined.
363
363
364
-
(** The universal property of the tensor product is that biadditive maps between abelian groups are in one-to-one corresondance with maps out of the tensor product. In this sense, the tensor product is the most perfect object describing biadditive maps between two abelian groups. *)
364
+
(** The universal property of the tensor product is that biadditive maps between abelian groups are in one-to-one correspondence with maps out of the tensor product. In this sense, the tensor product is the most perfect object describing biadditive maps between two abelian groups. *)
365
365
Definition equiv_ab_tensor_prod_rec `{Funext} (A B C : AbGroup)
366
366
: Biadditive A B C <~> (ab_tensor_prod A B $-> C).
367
367
Proof.
@@ -451,7 +451,7 @@ Defined.
451
451
452
452
(** ** Symmetry of the Tensor Product *)
453
453
454
-
(** The tensor product is symmetric in that the order in which we take the tensor shouldn't matter upto isomorphism. *)
454
+
(** The tensor product is symmetric in that the order in which we take the tensor shouldn't matter up to isomorphism. *)
455
455
456
456
(** We can define a swap map which swaps the order of simple tensors. *)
457
457
Definition ab_tensor_swap {A B} : ab_tensor_prod A B $-> ab_tensor_prod B A.
@@ -649,7 +649,7 @@ Proof.
649
649
exact (tensor_ab_mul z a b).
650
650
Defined.
651
651
652
-
(** The hexagon identity is also straighforward to prove. We simply have to reduce all the involved functions on the simple tensors using our custom triple tensor induction principle. *)
652
+
(** The hexagon identity is also straightforward to prove. We simply have to reduce all the involved functions on the simple tensors using our custom triple tensor induction principle. *)
Copy file name to clipboardexpand all lines: theories/Algebra/AbSES/Pullback.v
+1-1
Original file line number
Diff line number
Diff line change
@@ -221,7 +221,7 @@ Definition abses_pullback_pmap `{Univalence} {A B B' : AbGroup} (f : B' $-> B)
221
221
222
222
(** ** Functoriality of [abses_pullback] *)
223
223
224
-
(** [abses_pullback] is psuedo-functorial, and we can state this in terms of actual homotopies or "path data homotopies." We decorate the latter with the suffix ('). *)
224
+
(** [abses_pullback] is pseudo-functorial, and we can state this in terms of actual homotopies or "path data homotopies." We decorate the latter with the suffix ('). *)
225
225
226
226
(** For every [E : AbSES B A], the pullback of [E] along [id_B] is [E]. *)
227
227
Definition abses_pullback_id `{Univalence} {A B : AbGroup}
= abses_direct_sum (abses_pushout f E) (abses_pushout g F)
144
144
:= abses_pushout_component3_id (abses_directsum_pushout_morphism f g) (fun _ => idpath).
145
145
146
-
(** Given an AbSESMorphism whose third component is the identity, we know that it induces a path from the pushout of the domain along the first map to the codomain. Conversely, given a path from a pushout, we can deduce that the following square commutes: *)
146
+
(** Given an [AbSESMorphism] whose third component is the identity, we know that it induces a path from the pushout of the domain along the first map to the codomain. Conversely, given a path from a pushout, we can deduce that the following square commutes: *)
147
147
Definition abses_path_pushout_inclusion_commsq `{Univalence} {A A' B : AbGroup}
148
148
(alpha : A $-> A') (E : AbSES B A) (F : AbSES B A')
Copy file name to clipboardexpand all lines: theories/Algebra/Groups/Group.v
+3-3
Original file line number
Diff line number
Diff line change
@@ -79,7 +79,7 @@ Defined.
79
79
(** We create a database of hints for the group theory library *)
80
80
Create HintDb group_db.
81
81
82
-
(** Our group laws can be proven easily with tactics such as [rapply associativity]. However this requires a typeclass search on more general algebraic structures. Therefore we explicitly list many groups laws here so that coq can use them. We also create hints for each law in our groups database. *)
82
+
(** Our group laws can be proven easily with tactics such as [rapply associativity]. However this requires a typeclass search on more general algebraic structures. Therefore we explicitly list many groups laws here so that Coq can use them. We also create hints for each law in our groups database. *)
83
83
Section GroupLaws.
84
84
Context {G : Group} (x y z : G).
85
85
@@ -306,7 +306,7 @@ Defined.
306
306
307
307
(** ** Group Isomorphisms *)
308
308
309
-
(** Group isomorphsims are group homomorphisms whose underlying map happens to be an equivalence. They allow us to consider two groups to be the "same". They can be inverted and composed just like equivalences. *)
309
+
(** Group isomorphisms are group homomorphisms whose underlying map happens to be an equivalence. They allow us to consider two groups to be the "same". They can be inverted and composed just like equivalences. *)
310
310
311
311
(** An isomorphism of groups is defined as group homomorphism that is an equivalence. *)
312
312
Record GroupIsomorphism (G H : Group) := Build_GroupIsomorphism {
@@ -508,7 +508,7 @@ Section GroupEquations.
508
508
509
509
End GroupEquations.
510
510
511
-
(** ** Cancelation lemmas *)
511
+
(** ** Cancellation lemmas *)
512
512
513
513
(** Group elements can be cancelled both on the left and the right. *)
514
514
Definition grp_cancelL {G : Group} {x y : G} z : x = y <~> z * x = z * y
(** Pullbacks of groups are formalized by equipping the set-pullback with the desired group structure. The universal property in the category of groups is proved by saying that the corecursion principle (grp_pullback_corec) is an equivalence. *)
5
+
(** Pullbacks of groups are formalized by equipping the set-pullback with the desired group structure. The universal property in the category of groups is proved by saying that the corecursion principle [grp_pullback_corec] is an equivalence. *)
Copy file name to clipboardexpand all lines: theories/Algebra/Rings/CRing.v
+1-1
Original file line number
Diff line number
Diff line change
@@ -96,7 +96,7 @@ Defined.
96
96
Section IdealCRing.
97
97
Context {R : CRing}.
98
98
99
-
(** The section is meant to complement the IdealLemmas section in Algebra.Rings.Ideal. Since the results here only hold in commutative rings, they have to be kept here. *)
99
+
(** The section is meant to complement the [IdealLemmas] section in Algebra.Rings.Ideal. Since the results here only hold in commutative rings, they have to be kept here. *)
100
100
101
101
(** We import ideal notations as used in Algebra.Rings.Ideal but only for this section. Important to note is that [↔] corresponds to equality of ideals. *)
Copy file name to clipboardexpand all lines: theories/Algebra/Rings/Ideal.v
+5-5
Original file line number
Diff line number
Diff line change
@@ -14,7 +14,7 @@ Local Open Scope ideal_scope.
14
14
15
15
(** ** Definition of Ideals *)
16
16
17
-
(** An additive subgroup [I] of a ring [R] is a left ideal when it is closed under multiplciation on the left. *)
17
+
(** An additive subgroup [I] of a ring [R] is a left ideal when it is closed under multiplication on the left. *)
18
18
Class IsLeftIdeal {R : Ring} (I : Subgroup R) :=
19
19
isleftideal (r x : R) : I x -> I (r * x).
20
20
@@ -368,7 +368,7 @@ Definition ideal_kernel {R S : Ring} (f : RingHomomorphism R S) : Ideal R
368
368
369
369
(** *** Ideal generated by a subset *)
370
370
371
-
(** It seems tempting to define ideals generated by a subset in terms of subgroups generated by a subset but this does not work. Left ideals also have to be closed under left multiplciation by ring elements, and similarly for right and two sided ideals. Therefore we will do an analagous construction to the one done in Subgroup.v. *)
371
+
(** It seems tempting to define ideals generated by a subset in terms of subgroups generated by a subset but this does not work. Left ideals also have to be closed under left multiplication by ring elements, and similarly for right and two sided ideals. Therefore we will do an analagous construction to the one done in Subgroup.v. *)
372
372
373
373
(** Underlying type family of a left ideal generated by subset. *)
374
374
Inductive leftideal_generated_type (R : Ring) (X : R -> Type) : R -> Type :=
@@ -482,7 +482,7 @@ Proof.
482
482
rapply equiv_path_subgroup'.
483
483
Defined.
484
484
485
-
(** Under funext, ideal equiality is a proposition. *)
485
+
(** Under funext, ideal equality is a proposition. *)
(** The left annihilator of a left ideal also happens to be a right ideal. In fact, left ideal could be weakened to subset closed under multplication, however we don't need this generality currently. *)
654
+
(** The left annihilator of a left ideal also happens to be a right ideal. In fact, left ideal could be weakened to subset closed under multiplication, however we don't need this generality currently. *)
655
655
Instance isrightideal_ideal_left_annihilator {R : Ring} (I : Subgroup R)
(** We declare and import a module for various (unicode) ideal notations. These exist in their own special case, and can be imported and used in other files when needing to reason about ideals. *)
781
+
(** We declare and import a module for various (Unicode) ideal notations. These exist in their own special case, and can be imported and used in other files when needing to reason about ideals. *)
0 commit comments