Skip to content

Commit f109980

Browse files
committed
Globally delete all trailing whitespace
1 parent fc32bf6 commit f109980

File tree

18 files changed

+43
-43
lines changed

18 files changed

+43
-43
lines changed

Tealeaves/Backends/LN/AssocList.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -438,7 +438,7 @@ Section range_lemmas.
438438
range (envmap f Γ) = fmap list f (range Γ).
439439
Proof.
440440
intros. unfold range, envmap. compose near Γ.
441-
unfold_ops @Fmap_compose.
441+
unfold_ops @Fmap_compose.
442442
rewrite (fun_fmap_fmap list _ _ _ (fmap (prod atom) f) (extract (prod atom))).
443443
rewrite (fun_fmap_fmap list _ _ _ (extract (prod atom)) f).
444444
fequal. now ext [? ?].

Tealeaves/Backends/LN/LN.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -149,7 +149,7 @@ Section locally_nameless_operations.
149149

150150
Definition subst x (u : T LN) : T LN -> T LN :=
151151
bind T (subst_loc x u).
152-
152+
153153
Definition free : T LN -> list atom :=
154154
fun t => bind list free_loc (tolist T t).
155155

@@ -210,7 +210,7 @@ Tactic Notation "unfold_lia" :=
210210
Section locally_nameless_basic_principles.
211211

212212
Import Notations.
213-
213+
214214
Context
215215
`{DT.Monad.Monad nat T
216216
(unit := Monoid_unit_zero)

Tealeaves/Classes/DT/Monad.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -67,12 +67,12 @@ From Tealeaves Require
6767
Module ToKleisli.
6868

6969
Import Classes.Kleisli.DT.Monad.
70-
70+
7171
Import Classes.Kleisli.DT.Monad.Notations.
7272
Import Classes.Monad.Notations.
7373
Import Classes.Traversable.Functor.Notations.
7474
Import Data.Strength.Notations.
75-
75+
7676
Section operation.
7777

7878
Context
@@ -145,7 +145,7 @@ Module ToKleisli.
145145

146146
Import Decorated.Monad.ToKleisli.
147147
Import Kleisli.Decorated.Monad.
148-
148+
149149
Theorem kdtm_binddt1_T {A} : binddt T (fun A => A) (ret T ∘ extract (prod W)) = @id (T A).
150150
Proof.
151151
introv. unfold_ops @Binddt_ddj.

Tealeaves/Classes/Decorated/Functor.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -312,7 +312,7 @@ Module ToKleisli.
312312

313313
Import Classes.Kleisli.Decorated.Functor.
314314
Import Comonad.Notations.
315-
315+
316316
Section operation.
317317

318318
Context

Tealeaves/Classes/Equivalences/Decorated/Functor.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -77,7 +77,7 @@ End properties.
7777
Import Kleisli.Decorated.Functor.ToFunctor.
7878

7979
Module Roundtrip1.
80-
80+
8181
Context
8282
`{fmapT : Fmap T}
8383
`{decT : Decorate E T}

Tealeaves/Classes/Equivalences/Decorated/Monad.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -256,7 +256,7 @@ End Instances.
256256
#[local] Generalizable Variables T W.
257257

258258
Module CategoricalToKleisli.
259-
259+
260260
Context
261261
`{fmapT : Fmap T}
262262
`{decT : Decorate W T}

Tealeaves/Classes/Equivalences/Traversable/Functor.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -101,7 +101,7 @@ Module AlgebraicToKleisli.
101101
`{! Traversable.Functor.TraversableFunctor T}.
102102

103103
#[local] Instance traverse' : Traverse T := ToKleisli.Traverse_dist T.
104-
104+
105105
Definition fmap' : Fmap T := ToFunctor.Fmap_Traverse T.
106106
Definition dist' : Dist T := Dist_Traverse T.
107107

Tealeaves/Classes/Kleisli/Decorated/Functor.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -42,7 +42,7 @@ End class.
4242
(** * To functor *)
4343
(******************************************************************************)
4444
Module ToFunctor.
45-
45+
4646
Section operation.
4747

4848
Context

Tealeaves/Classes/Kleisli/Decorated/Monad.v

+6-6
Original file line numberDiff line numberDiff line change
@@ -176,15 +176,15 @@ End kleisli_composition.
176176
From Tealeaves Require Import
177177
Classes.Kleisli.Monad
178178
Classes.Kleisli.Decorated.Functor.
179-
179+
180180
(** * Derived instances *)
181181
(******************************************************************************)
182182
Module Derived.
183183

184184
Import
185185
Kleisli.Monad.Notations
186186
Comonad.Notations.
187-
187+
188188
Section operations.
189189

190190
Context
@@ -197,7 +197,7 @@ Module Derived.
197197
#[export] Instance Fmapd_Bindd: Fmapd W T := fun A B f => bindd T (ret T ∘ f).
198198

199199
End operations.
200-
200+
201201
(** ** Lesser Kleisli composition laws *)
202202
(******************************************************************************)
203203
Section Kleisli_composition.
@@ -304,9 +304,9 @@ Module Derived.
304304
Qed.
305305

306306
End with_monad.
307-
307+
308308
Section laws.
309-
309+
310310
Context
311311
(T : Type -> Type)
312312
`{Decorated.Monad.Monad W T}.
@@ -383,5 +383,5 @@ Module Derived.
383383
(******************************************************************************)
384384

385385
End laws.
386-
386+
387387
End Derived.

Tealeaves/Classes/Kleisli/Monad.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -16,7 +16,7 @@ Section kleisli_operations.
1616
(F T : Type -> Type).
1717

1818
Class Return := ret : (fun A => A) ⇒ T.
19-
19+
2020
Class Bind :=
2121
bind : forall (A B : Type), (A -> T B) -> F A -> F B.
2222

Tealeaves/Classes/Kleisli/Traversable/Functor.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -53,7 +53,7 @@ End class.
5353
(** ** <<Functor>> instance *)
5454
(******************************************************************************)
5555
Module ToFunctor.
56-
56+
5757
Section operation.
5858

5959
Context
@@ -64,7 +64,7 @@ Module ToFunctor.
6464
fun (A B : Type) (f : A -> B) => traverse T (fun A => A) f.
6565

6666
End operation.
67-
67+
6868
Section properties.
6969

7070
Context
@@ -149,7 +149,7 @@ Module ToFunctor.
149149
Qed.
150150

151151
End properties.
152-
152+
153153
End ToFunctor.
154154

155155
Import Batch.Notations.

Tealeaves/Classes/Kleisli/Traversable/Monad.v

+7-7
Original file line numberDiff line numberDiff line change
@@ -121,7 +121,7 @@ Module Derived.
121121
fun G _ _ _ A B f => bindt T G (fmap G (ret T) ∘ f).
122122

123123
End operations.
124-
124+
125125
Section special_cases.
126126

127127
Context
@@ -207,7 +207,7 @@ Module Derived.
207207
{| fun_fmap_id := fmap_id;
208208
fun_fmap_fmap := fmap_fmap;
209209
|}.
210-
210+
211211
(** *** Monad instance *)
212212
(******************************************************************************)
213213
#[export] Instance: Kleisli.Monad.Monad T.
@@ -236,7 +236,7 @@ Module Derived.
236236
Qed.
237237

238238
End with_kleisli.
239-
239+
240240
(** ** Special cases for Kleisli composition *)
241241
(******************************************************************************)
242242
Section Kleisli_composition.
@@ -347,7 +347,7 @@ Module Derived.
347347
rewrite (fun_fmap_id T).
348348
now rewrite (fun_fmap_id G1).
349349
Qed.
350-
350+
351351
End Kleisli_composition.
352352

353353
(** ** Composition with lesser Kleisli operations *)
@@ -361,7 +361,7 @@ Module Derived.
361361
(G2 : Type -> Type)
362362
`{Applicative G2}
363363
`{Applicative G1}.
364-
364+
365365
(** *** Composition with <<fmap>> *)
366366
(******************************************************************************)
367367
Lemma fmap_bindt : forall `(g : B -> C) `(f : A -> G1 (T B)),
@@ -382,7 +382,7 @@ Module Derived.
382382
fequal. now rewrite Mult_compose_identity2.
383383
rewrite kcompose_tm30; auto.
384384
Qed.
385-
385+
386386
(** *** Composition with <<traverse>> *)
387387
(******************************************************************************)
388388
Lemma traverse_bindt : forall `(g : B -> G2 C) `(f : A -> G1 (T B)),
@@ -492,7 +492,7 @@ Module Derived.
492492
change (@Fmap_Bindt T H0 H) with (@ToFunctor.Fmap_Bind T _ _).
493493
now rewrite (ToFunctor.fmap_bind T).
494494
Qed.
495-
495+
496496
End Kleisli_composition.
497497

498498
End Derived.

Tealeaves/Classes/Listable/Monad.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -44,7 +44,7 @@ End Listable_list.
4444
Section listable_monad_compatibility_conditions.
4545

4646
Generalizable All Variables.
47-
47+
4848
Context
4949
`{Monad T}
5050
`{Tolist T}
@@ -110,7 +110,7 @@ End listable_monad_compatibility_conditions.
110110
(** * Properties of listable monads *)
111111
(******************************************************************************)
112112
Section ListableMonad_theory.
113-
113+
114114
Context
115115
`{ListableMonad T}.
116116

Tealeaves/Classes/Monad.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -85,16 +85,16 @@ Module ToKleisli.
8585
Generalizable All Variables.
8686

8787
Section operation.
88-
88+
8989
Context
9090
(T : Type -> Type)
9191
`{Fmap T} `{Join T}.
9292

9393
#[export] Instance Bind_join : Bind T T :=
9494
fun {A B} (f : A -> T B) => join T ∘ fmap T f.
95-
95+
9696
End operation.
97-
97+
9898
Section with_monad.
9999

100100
Context

Tealeaves/Classes/Monad/ToApplicative.v

+4-4
Original file line numberDiff line numberDiff line change
@@ -1,18 +1,18 @@
11
From Tealeaves.Classes Require Import
22
Monad
33
Applicative.
4-
4+
55
(** * Monadic applicative functors *)
66
(******************************************************************************)
77
Section Applicative_Monad.
88

99
#[local] Generalizable Variable T.
10-
10+
1111
Import Applicative.Notations.
12-
12+
1313
Context
1414
`{Classes.Monad.Monad T}.
15-
15+
1616
Import Monad.ToKleisli.Operation.
1717
Import Monad.ToKleisli.Instance.
1818

Tealeaves/Classes/RightModule.v

+4-4
Original file line numberDiff line numberDiff line change
@@ -64,7 +64,7 @@ End RightModule_Monad.
6464
Section functor_module_composition.
6565

6666
#[local] Generalizable Variables F G.
67-
67+
6868
Context
6969
`{Functor F}
7070
`{RightModule G T}.
@@ -103,14 +103,14 @@ From Tealeaves Require Import Classes.Kleisli.Monad.
103103
(** * Kleisli laws for <<bind>> *)
104104
(******************************************************************************)
105105
Module ToKleisli.
106-
106+
107107
Import Kleisli.Monad.Notations.
108108
Import Classes.Monad.ToKleisli.
109-
109+
110110
Section Monad_kleisli_laws.
111111

112112
Generalizable All Variables.
113-
113+
114114
Context
115115
(T : Type -> Type)
116116
`{Classes.RightModule.RightModule F T}.

Tealeaves/Classes/Traversable/Listable.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -40,7 +40,7 @@ Section TraversableFunctor_fold_spec.
4040
Context
4141
(T : Type -> Type)
4242
`{TraversableFunctor T}.
43-
43+
4444
Import Classes.Kleisli.Traversable.Functor.
4545
Import Traversable.Functor.ToKleisli.
4646

Tealeaves/Functors/Sets.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -159,7 +159,7 @@ Qed.
159159
TODO: This isn't really necessary because it is inferred from the monad instance.
160160
*)
161161
Section set_applicative.
162-
162+
163163
Instance Pure_set : Pure set := @eq.
164164

165165
#[export] Instance Mult_set : Mult set :=

0 commit comments

Comments
 (0)