Skip to content

Commit

Permalink
proof simplification
Browse files Browse the repository at this point in the history
  • Loading branch information
adelaett committed Apr 8, 2024
1 parent 128d650 commit e77bc88
Showing 1 changed file with 4 additions and 23 deletions.
27 changes: 4 additions & 23 deletions theories/trans.v
Original file line number Diff line number Diff line change
Expand Up @@ -415,41 +415,22 @@ Theorem correction_continuations:
(trans_state s2) target.
Proof.

Local Ltac step' := (
Local Ltac step' := ( idtac
(* This tatic try to advance the computation on the right or on the left of the diagram. *)
try (eapply step_left; [solve
(* generic case *)
[ econstructor; simpl; eauto using List.map_nth_error
(* for contextual error cases *)
| econstructor; repeat intro; tryfalse
]|])
; try (eapply step_right; [solve
[ econstructor; simpl; eauto using List.map_nth_error
| econstructor; repeat intro; tryfalse
]|])
; try (eapply step_left; [solve [ econstructor; simpl; eauto using List.map_nth_error, trans_value_op_correct]|])
; try (eapply step_right; [solve [ econstructor; simpl; eauto using List.map_nth_error, trans_value_op_correct]|])
).

intros s1 s2 Hsred.
induction Hsred;
try induction phi;
try induction o;
intros; unpack.
intros; unpack; tryfalse.

all:
try solve [
repeat step';
try eapply diagram_finish;
eauto
].

(* Only two cases are left. *)
{ tryfalse. }
{ (* requires operator translation correction *)
eexists; split; asimpl; [|eapply star_refl].
eapply star_step.
{ econstructor.
eapply trans_value_op_correct; eauto.
}
eapply star_refl.
}
Qed.

0 comments on commit e77bc88

Please sign in to comment.