aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssrtest/gen_pattern.v
diff options
context:
space:
mode:
Diffstat (limited to 'mathcomp/ssrtest/gen_pattern.v')
-rw-r--r--mathcomp/ssrtest/gen_pattern.v20
1 files changed, 20 insertions, 0 deletions
diff --git a/mathcomp/ssrtest/gen_pattern.v b/mathcomp/ssrtest/gen_pattern.v
new file mode 100644
index 0000000..de57e8d
--- /dev/null
+++ b/mathcomp/ssrtest/gen_pattern.v
@@ -0,0 +1,20 @@
+Require Import ssreflect ssrbool ssrnat.
+
+Notation "( a 'in' c )" := (a + c) (only parsing) : myscope.
+Delimit Scope myscope with myscope.
+
+Notation "( a 'in' c )" := (a + c) (only parsing).
+
+Lemma foo x y : x + x.+1 = x.+1 + y.
+move: {x} (x.+1) {1}x y (x.+1 in RHS).
+ match goal with |- forall a b c d, b + a = d + c => idtac end.
+Admitted.
+
+Lemma bar x y : x + x.+1 = x.+1 + y.
+move E: ((x.+1 in y)) => w.
+ match goal with |- x + x.+1 = w => rewrite -{w}E end.
+move E: (x.+1 in y)%myscope => w.
+ match goal with |- x + x.+1 = w => rewrite -{w}E end.
+move E: ((x + y).+1 as RHS) => w.
+ match goal with |- x + x.+1 = w => rewrite -{}E -addSn end.
+Admitted. \ No newline at end of file