mirror of
https://github.com/achlipala/frap.git
synced 2024-11-10 00:07:51 +00:00
SharedMemory: model-checked a concrete program with partial-order reduction
This commit is contained in:
parent
34f586559f
commit
9de4dbdebe
1 changed files with 85 additions and 12 deletions
|
@ -635,18 +635,18 @@ Fixpoint pow2 (n : nat) : nat :=
|
||||||
end.
|
end.
|
||||||
|
|
||||||
Inductive boundRunningTime : cmd -> nat -> Prop :=
|
Inductive boundRunningTime : cmd -> nat -> Prop :=
|
||||||
| BrtReturn : forall r,
|
| BrtReturn : forall r n,
|
||||||
boundRunningTime (Return r) 0
|
boundRunningTime (Return r) n
|
||||||
| BrtFail :
|
| BrtFail : forall n,
|
||||||
boundRunningTime Fail 0
|
boundRunningTime Fail n
|
||||||
| BrtRead : forall a,
|
| BrtRead : forall a n,
|
||||||
boundRunningTime (Read a) 1
|
boundRunningTime (Read a) (S n)
|
||||||
| BrtWrite : forall a v,
|
| BrtWrite : forall a v n,
|
||||||
boundRunningTime (Write a v) 1
|
boundRunningTime (Write a v) (S n)
|
||||||
| BrtLock : forall a,
|
| BrtLock : forall a n,
|
||||||
boundRunningTime (Lock a) 1
|
boundRunningTime (Lock a) (S n)
|
||||||
| BrtUnlock : forall a,
|
| BrtUnlock : forall a n,
|
||||||
boundRunningTime (Unlock a) 1
|
boundRunningTime (Unlock a) (S n)
|
||||||
| BrtBind : forall c1 c2 n1 n2,
|
| BrtBind : forall c1 c2 n1 n2,
|
||||||
boundRunningTime c1 n1
|
boundRunningTime c1 n1
|
||||||
-> (forall r, boundRunningTime (c2 r) n2)
|
-> (forall r, boundRunningTime (c2 r) n2)
|
||||||
|
@ -1515,3 +1515,76 @@ Proof.
|
||||||
apply H9.
|
apply H9.
|
||||||
assumption.
|
assumption.
|
||||||
Qed.
|
Qed.
|
||||||
|
|
||||||
|
Ltac analyzer := repeat (match goal with
|
||||||
|
| [ |- context[if ?E then _ else _] ] => cases E
|
||||||
|
| _ => econstructor
|
||||||
|
end; simplify; try solve [ sets ]).
|
||||||
|
|
||||||
|
Ltac por_solve := simplify; repeat econstructor; sets; linear_arithmetic.
|
||||||
|
|
||||||
|
Ltac por_lister :=
|
||||||
|
repeat match goal with
|
||||||
|
| [ H : ?ls ++ _ = _ :: _ |- _ ] => cases ls; simplify; invert H
|
||||||
|
| [ H : @eq (list _) _ _ |- _ ] => apply (f_equal (@length _)) in H; simplify; linear_arithmetic
|
||||||
|
end.
|
||||||
|
|
||||||
|
Ltac por_invert1 :=
|
||||||
|
match goal with
|
||||||
|
| [ H : forall (c0 : cmd) (h'' : heap) (l'' : locks) (c'' : cmd), _ -> _ |- _ ] =>
|
||||||
|
(exfalso; eapply H; try por_solve; por_lister; por_solve) || (clear H; por_lister)
|
||||||
|
| _ => model_check_invert1
|
||||||
|
end.
|
||||||
|
|
||||||
|
Ltac por_invert := simplify; repeat por_invert1.
|
||||||
|
|
||||||
|
Ltac por_closure :=
|
||||||
|
repeat (apply oneStepClosure_empty
|
||||||
|
|| (apply oneStepClosure_split; [ por_invert; try equality; solve [ singletoner ] | ])).
|
||||||
|
|
||||||
|
Ltac por_step :=
|
||||||
|
eapply MscStep; [ por_closure | simplify ].
|
||||||
|
|
||||||
|
Ltac por_done :=
|
||||||
|
apply MscDone; eapply oneStepClosure_solve; [ por_closure | simplify; solve [ sets ] ].
|
||||||
|
|
||||||
|
Theorem independent_threads_ok_again :
|
||||||
|
invariantFor (trsys_of $0 {} independent_threads)
|
||||||
|
(fun p => let '(_, _, c) := p in
|
||||||
|
notAboutToFail c = true).
|
||||||
|
Proof.
|
||||||
|
eapply step_stepC with (cs := [(_, {| Reads := {0, 1};
|
||||||
|
Writes := {1};
|
||||||
|
Locks := {} |})]
|
||||||
|
++ [(_, {| Reads := {2};
|
||||||
|
Writes := {2};
|
||||||
|
Locks := {} |})]).
|
||||||
|
analyzer.
|
||||||
|
analyzer.
|
||||||
|
|
||||||
|
simplify.
|
||||||
|
eapply invariant_weaken.
|
||||||
|
apply multiStepClosure_ok; simplify.
|
||||||
|
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
por_step.
|
||||||
|
|
||||||
|
por_done.
|
||||||
|
|
||||||
|
sets.
|
||||||
|
|
||||||
|
Grab Existential Variables.
|
||||||
|
exact 0.
|
||||||
|
exact 0.
|
||||||
|
exact 0.
|
||||||
|
exact 0.
|
||||||
|
exact 0.
|
||||||
|
exact 0.
|
||||||
|
Qed.
|
||||||
|
|
Loading…
Reference in a new issue