aboutsummaryrefslogtreecommitdiff
path: root/coq/ex
diff options
context:
space:
mode:
authorPierre Courtieu2020-10-16 09:14:11 +0200
committerPierre Courtieu2020-10-16 17:31:52 +0200
commit0fdb1ae633baeb9afb07bbd8632bece5976f95f2 (patch)
tree1b65c8a70729ab6132a7cd8c9215a2ec4e40cab7 /coq/ex
parenteb6bba151b27f4d821088e10e1bda5cad0b70a28 (diff)
Fix #514 + support for named goal selector.
It was hard to separate this too fixes (same regexps).
Diffstat (limited to 'coq/ex')
-rw-r--r--coq/ex/indent.v25
1 files changed, 23 insertions, 2 deletions
diff --git a/coq/ex/indent.v b/coq/ex/indent.v
index e93616c8..72a3c201 100644
--- a/coq/ex/indent.v
+++ b/coq/ex/indent.v
@@ -4,8 +4,8 @@ Notation "[ ]" := nil : list_scope.
Notation "[ a ; .. ; b ]" := (a :: .. (b :: []) ..) : list_scope.
Require Import Arith.
-
-Definition arith1:
+Open Scope nat_scope.
+Definition arith1:=
1 + 3 *
4.
@@ -190,6 +190,27 @@ Module M1.
End M2.
End M1.
+Module GoalSelectors.
+ Theorem lt_n_S : (True \/ True \/ True \/ True \/ True ) -> True.
+ Proof.
+ refine (or_ind ?[aa] (or_ind ?[bb] (or_ind ?[cc] (or_ind ?[dd] ?[ee])))).
+ [aa]:{ auto. }
+ 2:{ auto. }
+ [ee]:auto.
+ { auto.}
+ Qed.
+ (* Same without space between "." and "}". *)
+ Theorem lt_n_S2 : (True \/ True \/ True \/ True \/ True ) -> True.
+ Proof.
+ refine (or_ind ?[aa] (or_ind ?[bb] (or_ind ?[cc] (or_ind ?[dd] ?[ee])))).
+ [aa]:{ auto.}
+ 2:{ auto.}
+ [ee]:auto.
+ { auto.}
+ Qed.
+
+
+End GoalSelectors.
Module M1'.
Module M2'.