Fix silly error in Coq proof.

This commit is contained in:
foreverbell 2018-01-21 20:45:05 +08:00
parent 5aee4f13c6
commit 7bf22a8151
No known key found for this signature in database
GPG Key ID: 92D5B279E66E4E51

View File

@ -142,7 +142,7 @@ Inductive StateMultiStep : State -> State -> Prop :=
StateMultiStep state state
| StateMultiStep1 :
forall state state1 state2,
StateMultiStep state1 state2 ->
StateStep state1 state2 ->
StateMultiStep state state1 ->
StateMultiStep state state2.
@ -275,7 +275,9 @@ Lemma Safety' :
Invariant state ->
Invariant state'.
Proof.
induction 1; crush.
induction 1; intros.
+ auto.
+ eapply StateStepKeepsInvariant; eauto.
Qed.
Theorem Safety :