Skip to content
Snippets Groups Projects
Verified Commit 673ad84e authored by Lennard Gäher's avatar Lennard Gäher
Browse files

remove sidecondition proof that now gets solved automatically

parent c9db3880
No related branches found
No related tags found
1 merge request!62Support trait attributes in more places + lifetime solver improvements
......@@ -30,22 +30,6 @@ Proof.
all: print_remaining_goal.
Unshelve. all: sidecond_solver.
Unshelve. all: sidecond_hammer.
{ (* TODO: currently not handled by the solver *)
apply Forall_forall.
intros κe Hlft.
eapply (lctx_lft_alive_incl ϝ); first sidecond_hook.
apply lctx_lft_incl_external.
apply elem_of_cons; right.
apply elem_of_cons; right.
apply elem_of_cons; right.
apply elem_of_app; right.
apply elem_of_app; right.
apply elem_of_app; right.
apply elem_of_app; left.
unfold_opaque @ty_outlives_E.
rewrite /lfts_outlives_E.
rewrite elem_of_list_fmap.
eexists. split; done. }
Unshelve. all: print_remaining_sidecond.
Qed.
End proof.
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