Skip to content
Snippets Groups Projects
Commit 5cca350d authored by Ralf Jung's avatar Ralf Jung
Browse files

add a helpful comment

parent f4ecf1f2
No related branches found
No related tags found
No related merge requests found
......@@ -114,6 +114,8 @@ Module Type IRIS_HT_RULES (RL : VIRA_T) (C : CORE_LANG) (R: IRIS_RES RL C) (WP:
Proof.
intros w n He. destruct HFill as (HFval & HFstep & HFfstep).
revert e w He; induction n using wf_nat_ind; intros; rename H into IH.
(* We need to actually decide whether e is a value, to establish safety in the case that
it is not. *)
destruct (is_value_dec e) as [HVal | HNVal]; [clear IH |].
- eapply (wpValue _ HVal) in He. exact:He.
- rewrite ->unfold_wp in He; rewrite unfold_wp. split; intros.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment