Skip to content

Commit ae84844

Browse files
authored
Merge pull request #2249 from patrick-nicodemus/aspell
Spelling and style changes
2 parents a470630 + 6741881 commit ae84844

File tree

172 files changed

+478
-476
lines changed

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

172 files changed

+478
-476
lines changed

theories/Algebra/AbGroups/AbPullback.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -25,6 +25,6 @@ Section AbPullback.
2525

2626
Definition ab_pullback : AbGroup := Build_AbGroup (grp_pullback f g) _.
2727

28-
(** The corecursion principle is inherited from Groups; use grp_pullback_corec and friends from Groups/GrpPullback.v. *)
28+
(** The corecursion principle is inherited from [Group]; use [grp_pullback_corec] and friends from Groups/GrpPullback.v. *)
2929

3030
End AbPullback.

theories/Algebra/AbGroups/AbelianGroup.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -154,7 +154,7 @@ Instance is0gpd_grouphomomorphism {A B : AbGroup} : Is0Gpd (A $-> B)
154154
Instance is2graph_abgroup : Is2Graph AbGroup
155155
:= is2graph_induced abgroup_group.
156156

157-
(** AbGroup forms a 1Cat *)
157+
(** [AbGroup] forms a 1Cat *)
158158
Instance is1cat_abgroup : Is1Cat AbGroup
159159
:= is1cat_induced _.
160160

@@ -164,15 +164,15 @@ Instance hasmorext_abgroup `{Funext} : HasMorExt AbGroup
164164
Instance hasequivs_abgroup : HasEquivs AbGroup
165165
:= hasequivs_induced _.
166166

167-
(** Zero object of AbGroup *)
167+
(** Zero object of [AbGroup] *)
168168

169169
Definition abgroup_trivial : AbGroup.
170170
Proof.
171171
rapply (Build_AbGroup grp_trivial).
172172
by intros [].
173173
Defined.
174174

175-
(** AbGroup is a pointed category *)
175+
(** [AbGroup] is a pointed category *)
176176
Instance ispointedcat_abgroup : IsPointedCat AbGroup.
177177
Proof.
178178
apply Build_IsPointedCat with abgroup_trivial.

theories/Algebra/AbGroups/Abelianization.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -123,7 +123,7 @@ Section Abel.
123123
rapply Coeq_ind_beta_cglue.
124124
Defined.
125125

126-
(** We also have a recursion princple. *)
126+
(** We also have a recursion principle. *)
127127
Definition Abel_rec (P : Type) `{IsHSet P} (a : G -> P)
128128
(c : forall x y z, a (x * (y * z)) = a (x * (z * y)))
129129
: Abel -> P.

theories/Algebra/AbGroups/Centralizer.v

+6-6
Original file line numberDiff line numberDiff line change
@@ -65,22 +65,22 @@ Proof.
6565
destruct h as [h H]; cbn in H.
6666
destruct k as [k K]; cbn in K.
6767
strip_truncations.
68-
(* It's enough to check equality after including into G: *)
68+
(* It's enough to check equality after including into [G]: *)
6969
apply (equiv_ap_isembedding (subgroup_incl _) _ _)^-1. cbn.
7070
induction H as [h [[] p]| |h1 h2 H1 H2 IHH1 IHH2].
71-
- (* The case when h = g: *)
71+
- (* The case when [h = g]: *)
7272
induction p.
7373
induction K as [k [[] q]| |k1 k2 K1 K2 IHK1 IHK2].
7474
+ (* The case when k = g: *)
7575
induction q.
7676
reflexivity.
77-
+ (* The case when k = mon_unit: *)
77+
+ (* The case when [k = mon_unit]: *)
7878
apply centralizer_unit.
79-
+ (* The case when k = k1 (-k2): *)
79+
+ (* The case when [k = k1 (-k2)]: *)
8080
srapply (issubgroup_in_op_inv (H:=centralizer (gen tt))); assumption.
81-
- (* The case when h = mon_unit: *)
81+
- (* The case when [h = mon_unit]: *)
8282
symmetry; apply centralizer_unit.
83-
- (* The case when h = h1 (-h2): *)
83+
- (* The case when [h = h1 (-h2)]: *)
8484
symmetry.
8585
srapply (issubgroup_in_op_inv (H:=centralizer k)); unfold centralizer; symmetry; assumption.
8686
Defined.

theories/Algebra/AbGroups/TensorProduct.v

+4-4
Original file line numberDiff line numberDiff line change
@@ -222,7 +222,7 @@ Proof.
222222
apply Hin.
223223
Defined.
224224

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. *)
226226
Definition ab_tensor_prod_ind_homotopy {A B G : AbGroup}
227227
{f f' : ab_tensor_prod A B $-> G}
228228
(H : forall a b, f (tensor a b) = f' (tensor a b))
@@ -361,7 +361,7 @@ Proof.
361361
napply grp_homo_op.
362362
Defined.
363363

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. *)
365365
Definition equiv_ab_tensor_prod_rec `{Funext} (A B C : AbGroup)
366366
: Biadditive A B C <~> (ab_tensor_prod A B $-> C).
367367
Proof.
@@ -451,7 +451,7 @@ Defined.
451451

452452
(** ** Symmetry of the Tensor Product *)
453453

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. *)
455455

456456
(** We can define a swap map which swaps the order of simple tensors. *)
457457
Definition ab_tensor_swap {A B} : ab_tensor_prod A B $-> ab_tensor_prod B A.
@@ -649,7 +649,7 @@ Proof.
649649
exact (tensor_ab_mul z a b).
650650
Defined.
651651

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. *)
653653
Instance hexagon_ab_tensor_prod : HexagonIdentity ab_tensor_prod.
654654
Proof.
655655
snapply hexagon_twist.

theories/Algebra/AbSES/Ext.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -166,7 +166,7 @@ Proof.
166166
symmetry; by apply abext_trivial_projective.
167167
Defined.
168168

169-
(* Converely, if all extensions ending in [P] are trivial, then [P] is projective. *)
169+
(* Conversely, if all extensions ending in [P] are trivial, then [P] is projective. *)
170170
Proposition abext_projective_trivial `{Univalence} (P : AbGroup)
171171
(ext_triv : forall A, forall E : AbSES P A, tr E = point (Ext P A))
172172
: IsAbProjective P.

theories/Algebra/AbSES/Pullback.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -221,7 +221,7 @@ Definition abses_pullback_pmap `{Univalence} {A B B' : AbGroup} (f : B' $-> B)
221221

222222
(** ** Functoriality of [abses_pullback] *)
223223

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 ('). *)
225225

226226
(** For every [E : AbSES B A], the pullback of [E] along [id_B] is [E]. *)
227227
Definition abses_pullback_id `{Univalence} {A B : AbGroup}

theories/Algebra/AbSES/Pushout.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -143,7 +143,7 @@ Definition abses_directsum_distributive_pushouts `{Univalence}
143143
= abses_direct_sum (abses_pushout f E) (abses_pushout g F)
144144
:= abses_pushout_component3_id (abses_directsum_pushout_morphism f g) (fun _ => idpath).
145145

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: *)
147147
Definition abses_path_pushout_inclusion_commsq `{Univalence} {A A' B : AbGroup}
148148
(alpha : A $-> A') (E : AbSES B A) (F : AbSES B A')
149149
(p : abses_pushout alpha E = F)

theories/Algebra/Categorical/MonoidObject.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -20,7 +20,7 @@ Section MonoidObject.
2020
Class IsMonoidObject (x : A) := {
2121
(** A multiplication map from the tensor product of [x] with itself to [x]. *)
2222
mo_mult : tensor x x $-> x;
23-
(** A unit of the multplication. *)
23+
(** A unit of the multiplication. *)
2424
mo_unit : unit $-> x;
2525
(** The multiplication map is associative. *)
2626
mo_assoc : mo_mult $o fmap10 tensor mo_mult x $o associator x x x
@@ -57,7 +57,7 @@ Section ComonoidObject.
5757

5858
(** We can build comonoid objects from the following data: *)
5959
Definition Build_IsComonoidObject (x : A)
60-
(** A comultplication map. *)
60+
(** A comultiplication map. *)
6161
(co_comult : x $-> tensor x x)
6262
(** A counit. *)
6363
(co_counit : x $-> unit)
@@ -184,7 +184,7 @@ Proof.
184184
exact (co_right_counit (A:=A^op) tensor unit (x:=x)).
185185
Defined.
186186

187-
(** A cocommutative cocomonoid object in [A^op] is a commutative monoid object in [A]. *)
187+
(** A cocommutative comonoid object in [A^op] is a commutative monoid object in [A]. *)
188188
Definition cmo_coco_op {A : Type} {tensor : A -> A -> A} {unit : A}
189189
`{HasEquivs A, !Is0Bifunctor tensor, !Is1Bifunctor tensor}
190190
`{!Associator tensor, !LeftUnitor tensor unit, !RightUnitor tensor unit,

theories/Algebra/Groups/FreeGroup.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -371,7 +371,7 @@ Section Reduction.
371371
exact (ap _ p).
372372
Defined.
373373

374-
(** Now we need to prove that the free group satisifes the unviersal property of the free group. *)
374+
(** Now we need to prove that the free group satisfies the universal property of the free group. *)
375375
(** TODO: remove funext from here and universal property of free group *)
376376
#[export] Instance isfreegroupon_freegroup `{Funext}
377377
: IsFreeGroupOn A FreeGroup freegroup_in.

theories/Algebra/Groups/FreeProduct.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -27,9 +27,9 @@ Local Open Scope mc_mult_scope.
2727
| omega_K : forall (x y : list (H + K)),
2828
amal_eta (x ++ [inr mon_unit] ++ y) = amal_eta (x ++ y).
2929
30-
We will build this HIT up sucessively out of coequalizers. *)
30+
We will build this HIT up successively out of coequalizers. *)
3131

32-
(** We will call M [amal_type] and prefix all the constructors with [amal_] (for amalgmated free product). *)
32+
(** We will call M [amal_type] and prefix all the constructors with [amal_] (for amalgamated free product). *)
3333

3434
Section FreeProduct.
3535

@@ -756,7 +756,7 @@ Proof.
756756
exact (grp_homo_unit _ @ (grp_homo_unit _)^).
757757
Defined.
758758

759-
(** The freeproduct is the coproduct in the category of groups. *)
759+
(** The free product is the coproduct in the category of groups. *)
760760
Instance hasbinarycoproducts : HasBinaryCoproducts Group.
761761
Proof.
762762
intros G H.

theories/Algebra/Groups/Group.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -79,7 +79,7 @@ Defined.
7979
(** We create a database of hints for the group theory library *)
8080
Create HintDb group_db.
8181

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. *)
8383
Section GroupLaws.
8484
Context {G : Group} (x y z : G).
8585

@@ -306,7 +306,7 @@ Defined.
306306

307307
(** ** Group Isomorphisms *)
308308

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. *)
310310

311311
(** An isomorphism of groups is defined as group homomorphism that is an equivalence. *)
312312
Record GroupIsomorphism (G H : Group) := Build_GroupIsomorphism {
@@ -508,7 +508,7 @@ Section GroupEquations.
508508

509509
End GroupEquations.
510510

511-
(** ** Cancelation lemmas *)
511+
(** ** Cancellation lemmas *)
512512

513513
(** Group elements can be cancelled both on the left and the right. *)
514514
Definition grp_cancelL {G : Group} {x y : G} z : x = y <~> z * x = z * y

theories/Algebra/Groups/GrpPullback.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -2,7 +2,7 @@ Require Import Basics Types Limits.Pullback Cubical.PathSquare.
22
Require Import Algebra.Groups.Group.
33
Require Import WildCat.Core.
44

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. *)
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. *)
66

77
Local Open Scope mc_scope.
88
Local Open Scope mc_mult_scope.

theories/Algebra/Groups/QuotientGroup.v

+5-5
Original file line numberDiff line numberDiff line change
@@ -111,7 +111,7 @@ End GroupCongruenceQuotient.
111111
Section Cosets.
112112

113113
Context (G : Group) (H : Subgroup G).
114-
114+
115115
Definition LeftCoset := G / in_cosetL H.
116116

117117
(** TODO: Way too many universes, needs fixing *)
@@ -130,7 +130,7 @@ Section Cosets.
130130
:= fcard LeftCoset.
131131

132132
Definition RightCoset := G / in_cosetR H.
133-
133+
134134
(** The set of left cosets is equivalent to the set of right coset. *)
135135
Definition equiv_leftcoset_rightcoset
136136
: LeftCoset <~> RightCoset.
@@ -226,7 +226,7 @@ Definition QuotientGroup' (G : Group) (N : Subgroup G) (H : IsNormalSubgroup N)
226226

227227
Local Open Scope group_scope.
228228

229-
(** Computation rule for grp_quotient_rec. *)
229+
(** Computation rule for [grp_quotient_rec]. *)
230230
Corollary grp_quotient_rec_beta `{F : Funext} {G : Group}
231231
(N : NormalSubgroup G) (H : Group)
232232
{A : Group} (f : G $-> A)
@@ -236,15 +236,15 @@ Proof.
236236
apply equiv_path_grouphomomorphism; reflexivity.
237237
Defined.
238238

239-
(** Computation rule for grp_quotient_rec. *)
239+
(** Computation rule for [grp_quotient_rec]. *)
240240
Definition grp_quotient_rec_beta' {G : Group}
241241
(N : NormalSubgroup G) (H : Group)
242242
{A : Group} (f : G $-> A)
243243
(h : forall n:G, N n -> f n = mon_unit)
244244
: (grp_quotient_rec G N f h) $o grp_quotient_map == f
245245
:= fun _ => idpath.
246246

247-
(** The proof of normality is irrelevent up to equivalence. This is unfortunate that it doesn't hold definitionally. *)
247+
(** The proof of normality is irrelevant up to equivalence. It is unfortunate that it doesn't hold definitionally. *)
248248
Definition grp_iso_quotient_normal (G : Group) (H : Subgroup G)
249249
{k k' : IsNormalSubgroup H}
250250
: QuotientGroup' G H k ≅ QuotientGroup' G H k'.

theories/Algebra/Groups/Subgroup.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -459,7 +459,7 @@ Proof.
459459
all: exact isnormal.
460460
Defined.
461461

462-
(** Our definiiton of normal subgroup implies the usual definition of invariance under conjugation. *)
462+
(** Our definition of normal subgroup implies the usual definition of invariance under conjugation. *)
463463
Definition isnormal_conj {G : Group} (N : Subgroup G)
464464
`{!IsNormalSubgroup N} {x y : G}
465465
: N x <~> N (y * x * y^).
@@ -1062,7 +1062,7 @@ Proof.
10621062
apply grp_image_in.
10631063
Defined.
10641064

1065-
(** ** Image of a subgroup under a group homomoprhism *)
1065+
(** ** Image of a subgroup under a group homomorphism *)
10661066

10671067
(** The image of a subgroup under group homomorphism. *)
10681068
Definition subgroup_image {G H : Group} (f : G $-> H)

theories/Algebra/Rings/CRing.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -96,7 +96,7 @@ Defined.
9696
Section IdealCRing.
9797
Context {R : CRing}.
9898

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. *)
100100

101101
(** 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. *)
102102
Import Ideal.Notation.

theories/Algebra/Rings/ChineseRemainder.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -140,7 +140,7 @@ Section ChineseRemainderTheorem.
140140

141141
End ChineseRemainderTheorem.
142142

143-
(** We also have the same for products of ideals when in a commuatative ring. *)
143+
(** We also have the same for products of ideals when in a commutative ring. *)
144144
Theorem chinese_remainder_prod `{Univalence}
145145
{R : CRing} (I J : Ideal R) (c : Coprime I J)
146146
: R / (I ⋅ J)%ideal ≅ (R / I) × (R / J).

theories/Algebra/Rings/Ideal.v

+5-5
Original file line numberDiff line numberDiff line change
@@ -14,7 +14,7 @@ Local Open Scope ideal_scope.
1414

1515
(** ** Definition of Ideals *)
1616

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. *)
1818
Class IsLeftIdeal {R : Ring} (I : Subgroup R) :=
1919
isleftideal (r x : R) : I x -> I (r * x).
2020

@@ -368,7 +368,7 @@ Definition ideal_kernel {R S : Ring} (f : RingHomomorphism R S) : Ideal R
368368

369369
(** *** Ideal generated by a subset *)
370370

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. *)
372372

373373
(** Underlying type family of a left ideal generated by subset. *)
374374
Inductive leftideal_generated_type (R : Ring) (X : R -> Type) : R -> Type :=
@@ -482,7 +482,7 @@ Proof.
482482
rapply equiv_path_subgroup'.
483483
Defined.
484484

485-
(** Under funext, ideal equiality is a proposition. *)
485+
(** Under funext, ideal equality is a proposition. *)
486486
Instance ishprop_ideal_eq `{Funext} {R : Ring} (I J : Ideal R)
487487
: IsHProp (ideal_eq I J) := _.
488488

@@ -651,7 +651,7 @@ Proof.
651651
apply rng_mult_zero_r.
652652
Defined.
653653

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 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. *)
655655
Instance isrightideal_ideal_left_annihilator {R : Ring} (I : Subgroup R)
656656
`{IsLeftIdeal R I}
657657
: IsRightIdeal (subgroup_ideal_left_annihilator I).
@@ -778,7 +778,7 @@ Defined.
778778

779779
(** *** Ideal notations *)
780780

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. *)
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. *)
782782

783783
Module Import Notation.
784784
Infix "⊆" := ideal_subset : ideal_scope.

0 commit comments

Comments
 (0)