Skip to content

Commit

Permalink
Fix
Browse files Browse the repository at this point in the history
  • Loading branch information
alxest committed Jul 9, 2019
1 parent 9c556da commit b63ace0
Show file tree
Hide file tree
Showing 7 changed files with 10 additions and 390 deletions.
2 changes: 1 addition & 1 deletion demo/DemoTarget.v
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,7 @@ Definition code: list instruction :=
].

Definition func: function :=
mkfunction (Some (mksignature [Tlong] (Some Tfloat) cc_default)) code
mkfunction (mksignature [Tlong] (Some Tfloat) cc_default true) code
.

Definition prog: program := mkprogram [(func_id, (Gfun (Internal func)))] [func_id ; main_id] main_id.
Expand Down
2 changes: 1 addition & 1 deletion demo/mutrec/MutrecA.v
Original file line number Diff line number Diff line change
Expand Up @@ -57,7 +57,7 @@ Definition composites : list composite_definition := nil.
Definition global_definitions : list (ident * globdef fundef type) :=
((g_id,
Gfun(External (EF_external "g"
(mksignature (AST.Tint :: nil) (Some AST.Tint) cc_default))
(mksignature (AST.Tint :: nil) (Some AST.Tint) cc_default true))
(Tcons tint Tnil) tint cc_default)) :: (_memoized, Gvar v_memoized) ::
(f_id, Gfun(Internal func_f)) :: nil).

Expand Down
6 changes: 3 additions & 3 deletions demo/mutrec/MutrecB.v
Original file line number Diff line number Diff line change
Expand Up @@ -49,7 +49,7 @@ Definition code: list instruction :=
Pleal RDI (Addrmode (Some RBX) None (inl (- 1)));
(* leal -1(%ebx), %edi *)

Pcall_s f_id (mksignature [Tint] (Some Tint) cc_default);
Pcall_s f_id (mksignature [Tint] (Some Tint) cc_default true);
(* call f *)

Pleal RAX (Addrmode (Some RAX) (Some (RBX, 1)) (inl 0));
Expand Down Expand Up @@ -77,13 +77,13 @@ Definition code: list instruction :=
].

Definition func_g: function :=
mkfunction (Some (mksignature [Tint] (Some Tint) cc_default)) code
mkfunction (mksignature [Tint] (Some Tint) cc_default true) code
.

Definition global_definitions : list (ident * globdef fundef unit) :=
((f_id,
Gfun(External (EF_external "f"
(mksignature (AST.Tint :: nil) (Some AST.Tint) cc_default)))) :: (_memoized, Gvar v_memoized) ::
(mksignature (AST.Tint :: nil) (Some AST.Tint) cc_default true)))) :: (_memoized, Gvar v_memoized) ::
(g_id, Gfun(Internal func_g)) :: nil).

Definition public_idents : list ident :=
Expand Down
2 changes: 1 addition & 1 deletion demo/mutrec/MutrecHeader.v
Original file line number Diff line number Diff line change
Expand Up @@ -91,5 +91,5 @@ Qed.

Require AST.

Definition fg_sig: AST.signature := (AST.mksignature [AST.Tint] (Some AST.Tint) AST.cc_default).
Definition fg_sig: AST.signature := (AST.mksignature [AST.Tint] (Some AST.Tint) AST.cc_default true).

381 changes: 0 additions & 381 deletions demo/mutrec/a.v

This file was deleted.

1 change: 0 additions & 1 deletion demo/mutrec/b.v

This file was deleted.

6 changes: 4 additions & 2 deletions proof/Preservation.v
Original file line number Diff line number Diff line change
Expand Up @@ -673,9 +673,11 @@ Proof.
- inv INIT. rr. esplits; eauto.
+ refl.
- inv STEP. ss. inv SUST. des. exploit Sound.system_axiom; try apply EXTCALL; eauto.
{ instantiate (1:= Args.Cstyle _ _ _). ss. esplits; eauto. }
{ instantiate (1:= Args.Cstyle _ _ _). ss. }
{ rr. esplits; eauto. }
{ eapply Sound.system_skenv; eauto. eapply Sound.skenv_mle; eauto. }
i; des. r in RETV. des. ss. esplits; eauto.
{ eauto. }
i; des. r in RETV. ss. des. ss. esplits; eauto.
+ etrans; eauto.
+ eapply Sound.skenv_mle; eauto. etrans; eauto.
- inv FINAL. ss. des. esplits; eauto.
Expand Down

0 comments on commit b63ace0

Please sign in to comment.