diff options
| author | Pierre Courtieu | 2020-02-07 23:17:11 +0100 |
|---|---|---|
| committer | Pierre Courtieu | 2020-03-12 18:24:21 +0100 |
| commit | db7149abd8e3355b9a195f5513075808fff8d197 (patch) | |
| tree | a033649fc4849dd17639b2c711e8e51604921190 /coq/ex | |
| parent | f737203ced2446ec54be7b31b21c47e731404e12 (diff) | |
Fix #465: Indentation of Equations (plugin).
Diffstat (limited to 'coq/ex')
| -rw-r--r-- | coq/ex/indent_plugins.v | 19 |
1 files changed, 6 insertions, 13 deletions
diff --git a/coq/ex/indent_plugins.v b/coq/ex/indent_plugins.v index b4f926a0..2c0c496f 100644 --- a/coq/ex/indent_plugins.v +++ b/coq/ex/indent_plugins.v @@ -55,14 +55,6 @@ Module Equations. neg true := false ; neg false := true. - Equations neg' (b : bool) : bool := - neg true => false ; - neg false => true. - - Check neg_graph. - Check neg_graph_equation_1. - Check neg_graph_equation_2. - Lemma neg_inv : forall b, neg (neg b) = b. Proof. intros b. @@ -76,17 +68,18 @@ Module Equations. Notation "x :: l" := (cons x l). Equations tail {A} (l : list A) : list A := - tail nil := + | nil := nil ; - tail (cons a v) - := v. + | (cons a v) + := v. (* The cases inside { } are recognized as record fields, which from an indentation perspective is OK *) Equations filter {A} (l : list A) (p : A -> bool) : list A := filter (cons a l) p with p a => - { filter (cons a l) p true := a :: filter l p ; - filter (cons a l) p false := filter l p + { + | true := a :: filter l p ; + | false := filter l p }; filter nil p := nil . |
