Skip to content

Commit b04c199

Browse files
committed
documentation cleanup
- use a style that only shows the "Proof." command on mouseover - limit the depth of the ToC to 2 - clean up headers to yield a cleaner ToC
1 parent e971cb1 commit b04c199

16 files changed

+42
-49
lines changed

Makefile.coq.local

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ DOCDIR = docs
1212
COQDOCDIR = $(DOCDIR)/coqdoc
1313

1414
COQDOCHTMLFLAGS = --toc -s --external 'http://math-comp.github.io/htmldoc/' mathcomp --html \
15-
--with-header $(HEADER) --with-footer $(FOOTER) --index indexpage --parse-comments
15+
--with-header $(HEADER) --with-footer $(FOOTER) --index indexpage --parse-comments --toc-depth 2
1616

1717
coqdoc: $(GLOBFILES) $(VFILES) $(HEADER) $(FOOTER) $(RESOURCES)
1818
$(SHOW)'COQDOC -d $(COQDOCDIR)'

theories/arc.v

Lines changed: 2 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,7 @@ Qed.
1717
Lemma leq_subl n m o : n <= m -> n - o <= m.
1818
Proof. move => A. rewrite -[m]subn0. exact: leq_sub. Qed.
1919

20-
(** ** Lemmas on [index], [mask], and [subseq] *)
20+
(** *** Lemmas on [index] and [subseq] *)
2121
(** could go to seq.v *)
2222

2323
Lemma mem2_index (T : eqType) (x y : T) (s : seq T) :
@@ -41,9 +41,6 @@ rewrite -!mem2_index ?mem2E // => [?|]; last exact: (mem_subseq sub_s1_s2).
4141
exact: subseq_trans sub_s1_s2.
4242
Qed.
4343

44-
(** ** Lemmas on [next] and [rot] *)
45-
(** could go to path.v *)
46-
4744
Section Path.
4845

4946
Lemma eq_traject (T : Type) (f g : T -> T) : f =1 g -> traject f =2 traject g.
@@ -115,7 +112,7 @@ move=> inj_f; case: s => //= a s.
115112
by elim: s a {2 4}a => /= [|y s IHs] a b; rewrite inj_eq // ?IHs -fun_if.
116113
Qed.
117114

118-
(** ** Lemmas on [index] *)
115+
(** *** Lemmas on [index] *)
119116
(** could go to [fingraph.v] *)
120117

121118
Lemma eq_findex (T : finType) (f g : T -> T) :

theories/completeness.v

Lines changed: 3 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,7 @@ Unset Strict Implicit.
88
Unset Printing Implicit Defensive.
99
Set Bullet Behavior "Strict Subproofs".
1010

11-
(** * Completeness *)
11+
(** * Completeness of the 2pdom axioms *)
1212

1313
Section s.
1414
Variable A: Type.
@@ -153,10 +153,8 @@ Proof.
153153
apply relabel2_iso=>//.
154154
case=>//=??/=->//.
155155
Qed.
156-
157-
(** ** Main Result *)
158156

159-
(* main completeness theorem *)
157+
(** main completeness theorem *)
160158
Theorem completeness (u v: term): graph_of_term u ≃2p graph_of_term v -> u ≡ v.
161159
Proof.
162160
move=>/tgraph_graph_iso h.
@@ -168,7 +166,7 @@ Proof.
168166
apply normal_iso. by rewrite HF'.
169167
Qed.
170168

171-
(* actually an iff since graphs from a 2pdom algebra *)
169+
(** actually an iff since graphs from a 2pdom algebra *)
172170
Theorem soundness_and_completeness (u v: term): graph_of_term u ≃2p graph_of_term v <-> u ≡ v.
173171
Proof.
174172
split => [|uv]; first exact: completeness.

theories/connectivity.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1189,7 +1189,7 @@ Proof.
11891189
Qed.
11901190

11911191

1192-
(** * k-connectivity *)
1192+
(** ** k-connectivity *)
11931193

11941194
Definition kconnected (k : nat) (G : sgraph) :=
11951195
k < #|G| /\ forall S : {set G}, vseparator S -> k <= #|S|.

theories/dom.v

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -7,9 +7,8 @@ Unset Printing Implicit Defensive.
77

88
Set Bullet Behavior "Strict Subproofs".
99

10-
(**********************************************************************************)
11-
(** * Domination Theory *)
12-
(**********************************************************************************)
10+
(** * Domination Theory *)
11+
1312
(** ** Hereditary and superhereditary properties *)
1413
Section Hereditary.
1514
Variable (T : finType).

theories/embedding.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,7 @@ Lemma plain_face (D : hypermap) (x : D) :
1717
plain D -> face x = finv node (edge x).
1818
Proof. by move=> plainD; rewrite -plain_eq' // finv_f. Qed.
1919

20-
(** * Hypermaps as embeddings of (planar) grahs *)
20+
(** * Hypermaps as Embeddings of (planar) Grahps *)
2121

2222
(** This is mainly usedful when takling about embeddings, as hypermaps
2323
cannot represent isolated vertices. *)

theories/extraction_def.v

Lines changed: 7 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -25,9 +25,11 @@ Local Notation link_rel := checkpoint.link_rel.
2525
(the latter start from a 2pdom term rather than a 2p term) *)
2626
Definition graph_of_term: term sym -> graph2 := eval (fun a : flat sym => @g2_var _ _ a).
2727

28-
(** * Term Extraction Function *)
28+
(** * Term Extraction for 2p-graphs in TW2 *)
2929

30-
(** ** Termination Metric *)
30+
(** ** Extraction function for connected graphs *)
31+
32+
(** *** Termination Metric *)
3133

3234
Definition term_of_measure (G : graph2) :=
3335
(input == output :> G) + 2*#|edge G|.
@@ -79,7 +81,7 @@ Proof.
7981
move: He. by rewrite !inE => /orP[/andP[/eqP<- _]|/andP[_ /eqP<-]].
8082
Qed.
8183

82-
(** ** Subroutines *)
84+
(** *** Subroutines *)
8385

8486
Definition lens (G : graph2) :=
8587
[&& edge_set G (@bag G IO input) == set0 ,
@@ -216,7 +218,7 @@ Definition tm_ (G : graph2) (e : edge G): term sym :=
216218

217219
Definition tmEs (G : graph2) : seq (term sym) := [seq tm_ e | e in edge_set G IO].
218220

219-
(** ** The Extraction Functional *)
221+
(** *** The Extraction Functional *)
220222

221223
(** Here we define the extraction function. The case distinctions are chosen
222224
such that we can make use of induced subgraphs (rather than the more generic
@@ -256,7 +258,7 @@ Definition term_of_rec (term_of : graph2 -> term sym) (G : graph2) :=
256258

257259
Definition term_of := Fix top term_of_measure term_of_rec.
258260

259-
(** ** Termination Argument *)
261+
(** *** Termination Argument *)
260262

261263

262264
Notation sigraph := cp_minor.igraph.

theories/extraction_iso.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ Notation graph2 := (graph2 unit (flat sym)).
2121
Notation g2_top := (g2_top : graph2).
2222
Notation g2_one := (g2_one : graph2).
2323

24-
(** * Isomorphim Theorem *)
24+
(** ** Correctness of the Extraction Function *)
2525

2626
(** In this file we prove correctness of the extraction function. This
2727
mainly amounts to establishing a variety of isomorphisms corresponding

theories/extraction_top.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ Notation graph2 := (graph2 unit (flat sym)).
2121
Open Scope ptt_ops.
2222

2323

24-
(** * Extraction from Disconnected Graphs *)
24+
(** ** Extraction from Disconnected Graphs *)
2525

2626
Arguments iso_id {Lv Le G}.
2727
Arguments merge_union_K_l [Lv Le F K i o h] k.

0 commit comments

Comments
 (0)