aboutsummaryrefslogtreecommitdiff
path: root/src/Compilers/Z/OpInversion.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2019-01-08 04:21:38 -0500
committerGravatar Andres Erbsen <andreser@mit.edu>2019-01-09 22:49:02 -0500
commit3ca227f1137e6a3b65bc33f5689e1c230d591595 (patch)
treee1e5a2dd2a2f34f239d3276227ddbdc69eeeb667 /src/Compilers/Z/OpInversion.v
parent3ec21c64b3682465ca8e159a187689b207c71de4 (diff)
remove old pipeline
Diffstat (limited to 'src/Compilers/Z/OpInversion.v')
-rw-r--r--src/Compilers/Z/OpInversion.v29
1 files changed, 0 insertions, 29 deletions
diff --git a/src/Compilers/Z/OpInversion.v b/src/Compilers/Z/OpInversion.v
deleted file mode 100644
index c27f51aee..000000000
--- a/src/Compilers/Z/OpInversion.v
+++ /dev/null
@@ -1,29 +0,0 @@
-Require Import Crypto.Compilers.Syntax.
-Require Import Crypto.Compilers.TypeInversion.
-Require Import Crypto.Compilers.Z.TypeInversion.
-Require Import Crypto.Compilers.Z.Syntax.
-
-Ltac invert_one_op e :=
- preinvert_one_type e;
- intros ? e;
- destruct e;
- try exact I.
-
-Ltac invert_op_step :=
- match goal with
- | [ e : op _ (Tbase _) |- _ ] => invert_one_op e
- | [ e : op _ (Prod _ _) |- _ ] => invert_one_op e
- | [ e : op _ Unit |- _ ] => invert_one_op e
- end.
-
-Ltac invert_op := repeat invert_op_step.
-
-Ltac invert_match_op_step :=
- match goal with
- | [ |- context[match ?e with OpConst _ _ => _ | _ => _ end] ]
- => invert_one_op e
- | [ H : context[match ?e with OpConst _ _ => _ | _ => _ end] |- _ ]
- => invert_one_op e
- end.
-
-Ltac invert_match_op := repeat invert_match_op_step.