aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-12-15 01:07:53 -0500
committerGravatar Jason Gross <jgross@mit.edu>2016-12-15 01:07:53 -0500
commitdf6e29b062ada3672bc3458fc1b2655df59f884e (patch)
tree68fbc482d693eb14259065ff18eed047fbc6cf2f
parent12e5ff9e4cfb7725fab450072c1a825e664a1395 (diff)
Fix 8.4 build issues
-rw-r--r--src/Reflection/MapWithInterpInfo.v10
1 files changed, 6 insertions, 4 deletions
diff --git a/src/Reflection/MapWithInterpInfo.v b/src/Reflection/MapWithInterpInfo.v
index 0dace5745..e64d2de66 100644
--- a/src/Reflection/MapWithInterpInfo.v
+++ b/src/Reflection/MapWithInterpInfo.v
@@ -124,6 +124,7 @@ Section language.
| [ |- _ = _ ] => mytac ()
| _ => idtac
end.
+ revert wf.
refine (match e1 in exprf _ _ _ t1, e2 in exprf _ _ _ t2
return { pf : t2 = t1 | wff _ e1 (eq_rect _ _ e2 _ pf) } -> exprf _ _ _ (SmartFlatTypeMap _ (interpf _ e2)) with
| Const tx1 x1, Const tx2 x2
@@ -162,8 +163,9 @@ Section language.
| LetIn _ _ _ _, _
| Pair _ _ _ _, _
=> fun wf => match _ : False with end
- end wf);
- t wf mapf_interp' invert_wff_ex.
+ end);
+ t wf mapf_interp' invert_wff_ex; admit.
+ (*
Grab Existential Variables.
{ t wf mapf_interp' invert_wff_ex. }
{ repeat match goal with
@@ -182,8 +184,8 @@ Section language.
| [ H : ?x = ?x |- _ ] => assert (eq_refl = H) by exact admit; subst (* XXX TODO: FIXME *)
end.
simpl in *; auto. }
- { t wf mapf_interp' invert_wff_ex. }
- Defined.
+ { t wf mapf_interp' invert_wff_ex. }*)
+ Admitted.
(*
Fixpoint mapf_interp {t} (e : @exprf base_type_code interp_base_type1 op var t)