aboutsummaryrefslogtreecommitdiff
path: root/src
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-04-02 00:28:00 -0400
committerGravatar Jason Gross <jgross@mit.edu>2017-04-02 00:28:00 -0400
commit5961b8fa1f00c01c9c2b84ae048cc1531ed6aab4 (patch)
treeaaf3bc8eb8c19afcbb63effd937e5d27aaa6f731 /src
parent2882da783bf4a45cbdab2ff53d6acaea74c71f22 (diff)
Add Z instantiation of MapCastByDeBruijnInterp
Diffstat (limited to 'src')
-rw-r--r--src/Reflection/Z/MapCastByDeBruijnInterp.v50
1 files changed, 50 insertions, 0 deletions
diff --git a/src/Reflection/Z/MapCastByDeBruijnInterp.v b/src/Reflection/Z/MapCastByDeBruijnInterp.v
new file mode 100644
index 000000000..072563680
--- /dev/null
+++ b/src/Reflection/Z/MapCastByDeBruijnInterp.v
@@ -0,0 +1,50 @@
+Require Import Crypto.Reflection.Syntax.
+Require Import Crypto.Reflection.Wf.
+Require Import Crypto.Reflection.SmartMap.
+Require Import Crypto.Reflection.Relations.
+Require Import Crypto.Reflection.MapCastByDeBruijnInterp.
+Require Import Crypto.Reflection.Z.Syntax.
+Require Import Crypto.Reflection.Z.MapCastByDeBruijn.
+
+Section language.
+ Context {interp_base_type_bounds : base_type -> Type}
+ (interp_op_bounds : forall src dst, op src dst -> interp_flat_type interp_base_type_bounds src -> interp_flat_type interp_base_type_bounds dst)
+ (pick_typeb : forall t, interp_base_type_bounds t -> base_type).
+ Local Notation pick_type v := (SmartFlatTypeMap pick_typeb v).
+ Context (cast_op : forall t tR (opc : op t tR) args_bs,
+ op (pick_type args_bs) (pick_type (interp_op_bounds t tR opc args_bs)))
+ (cast_backb: forall t b, interp_base_type (pick_typeb t b) -> interp_base_type t).
+ Let cast_back : forall t b, interp_flat_type interp_base_type (pick_type b) -> interp_flat_type interp_base_type t
+ := fun t b => SmartFlatTypeMapUnInterp cast_backb.
+ Context (inboundsb : forall t, interp_base_type_bounds t -> interp_base_type t -> Prop).
+ Let inbounds : forall t, interp_flat_type interp_base_type_bounds t -> interp_flat_type interp_base_type t -> Prop
+ := fun t => interp_flat_type_rel_pointwise inboundsb (t:=t).
+ Context (interp_op_bounds_correct
+ : forall t tR opc bs
+ (v : interp_flat_type interp_base_type t)
+ (H : inbounds t bs v),
+ inbounds tR (interp_op_bounds t tR opc bs) (interp_op t tR opc v))
+ (pull_cast_back
+ : forall t tR opc bs
+ (v : interp_flat_type interp_base_type (pick_type bs))
+ (H : inbounds t bs (cast_back t bs v)),
+ interp_op t tR opc (cast_back t bs v)
+ =
+ cast_back _ _ (interp_op _ _ (cast_op _ _ opc bs) v)).
+
+ Local Notation MapCast
+ := (@MapCast interp_base_type_bounds interp_op_bounds pick_typeb cast_op).
+
+ Lemma MapCastCorrect
+ {t} (e : Expr base_type op t)
+ (Hwf : Wf e)
+ (input_bounds : interp_flat_type interp_base_type_bounds (domain t))
+ : forall {b} e' (He':MapCast e input_bounds = Some (existT _ b e'))
+ v v' (Hv : @inbounds _ input_bounds v /\ cast_back _ _ v' = v),
+ Interp interp_op_bounds e input_bounds = b
+ /\ @inbounds _ b (Interp interp_op e v)
+ /\ cast_back _ _ (Interp interp_op e' v') = (Interp interp_op e v).
+ Proof.
+ apply MapCastCorrect; auto using internal_base_type_dec_lb.
+ Qed.
+End language.