aboutsummaryrefslogtreecommitdiff
path: root/src/Reflection/Reify.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-11-06 13:42:42 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-11-06 13:57:32 -0500
commit7ec5494a230388ad0715c5dba87b57d19a0eb838 (patch)
treeaf1252428a2a34b65f623170fa07f0555881a1b4 /src/Reflection/Reify.v
parent1d871e22bbdf011b6711d1488d975d019367b00e (diff)
Add support for dependent reification
Diffstat (limited to 'src/Reflection/Reify.v')
-rw-r--r--src/Reflection/Reify.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/src/Reflection/Reify.v b/src/Reflection/Reify.v
index ed9646eb4..1a2f22eca 100644
--- a/src/Reflection/Reify.v
+++ b/src/Reflection/Reify.v
@@ -68,11 +68,11 @@ Inductive reify_result_helper :=
| reification_unsuccessful.
(** Override this to get a faster [reify_op] *)
-Ltac base_reify_op op op_head :=
+Ltac base_reify_op op op_head expr :=
let r := constr:(_ : reify_op op op_head _ _) in
type of r.
-Ltac reify_op op op_head :=
- let t := base_reify_op op op_head in
+Ltac reify_op op op_head expr :=
+ let t := base_reify_op op op_head expr in
constr:(op_info t).
(** Change this with [Ltac reify_debug_level ::= constr:(1).] to get
@@ -152,7 +152,7 @@ Ltac reifyf base_type_code interp_base_type op var e :=
let retv := match constr:(Set) with
| _ => let retv := reifyf_var x mkVar in constr:(finished_value retv)
| _ => let op_head := head x in
- reify_op op op_head
+ reify_op op op_head x
| _ => let c := mkConst t x in
constr:(finished_value c)
| _ => constr:(reification_unsuccessful)