summaryrefslogtreecommitdiff
path: root/cfrontend/SimplExprspec.v
diff options
context:
space:
mode:
Diffstat (limited to 'cfrontend/SimplExprspec.v')
-rw-r--r--cfrontend/SimplExprspec.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/cfrontend/SimplExprspec.v b/cfrontend/SimplExprspec.v
index 5cb0f18..b31738b 100644
--- a/cfrontend/SimplExprspec.v
+++ b/cfrontend/SimplExprspec.v
@@ -591,7 +591,7 @@ Lemma within_widen:
Proof.
intros. destruct H. split.
eapply Ple_trans; eauto.
- unfold Plt, Ple in *. omega.
+ eapply Plt_Ple_trans; eauto.
Qed.
Definition contained (l: list ident) (g1 g2: generator) : Prop :=