aboutsummaryrefslogtreecommitdiff
path: root/src/LegacyArithmetic/Double/Proofs/BitwiseOr.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/LegacyArithmetic/Double/Proofs/BitwiseOr.v
parent3ec21c64b3682465ca8e159a187689b207c71de4 (diff)
remove old pipeline
Diffstat (limited to 'src/LegacyArithmetic/Double/Proofs/BitwiseOr.v')
-rw-r--r--src/LegacyArithmetic/Double/Proofs/BitwiseOr.v32
1 files changed, 0 insertions, 32 deletions
diff --git a/src/LegacyArithmetic/Double/Proofs/BitwiseOr.v b/src/LegacyArithmetic/Double/Proofs/BitwiseOr.v
deleted file mode 100644
index 8588836ee..000000000
--- a/src/LegacyArithmetic/Double/Proofs/BitwiseOr.v
+++ /dev/null
@@ -1,32 +0,0 @@
-Require Import Coq.ZArith.ZArith.
-Require Import Crypto.LegacyArithmetic.Interface.
-Require Import Crypto.LegacyArithmetic.Double.Core.
-Require Import Crypto.LegacyArithmetic.Double.Proofs.Decode.
-Require Import Crypto.Util.ZUtil.Tactics.LtbToLt.
-Require Import Crypto.Util.ZUtil.LandLorShiftBounds.
-Require Import Crypto.Util.Tactics.BreakMatch.
-
-Local Open Scope Z_scope.
-
-Section bitwise_or.
- Context {n W}
- {decode : decoder n W}
- {is_decode : is_decode decode}
- {or : bitwise_or W}
- {is_or : is_bitwise_or or}.
-
- Global Instance is_bitwise_or_double
- : is_bitwise_or or_double.
- Proof using Type*.
- constructor; intros x y.
- destruct n as [|p|].
- { rewrite !(tuple_decoder_n_O (W:=W) 2); easy. }
- { assert (0 <= Z.lor (decode (fst x)) (decode (fst y)) < 2^Z.pos p) by auto with zarith.
- rewrite (tuple_decoder_2 x), (tuple_decoder_2 y), (tuple_decoder_2 (or_double x y))
- by apply Zle_0_pos.
- push_decode.
- apply Z.bits_inj'; intros; autorewrite with Ztestbit.
- break_match; Z.ltb_to_lt; autorewrite with Ztestbit; reflexivity. }
- { rewrite !(tuple_decoder_n_neg (W:=W) 2); easy. }
- Qed.
-End bitwise_or.