summaryrefslogtreecommitdiff
path: root/arm/Op.v
diff options
context:
space:
mode:
Diffstat (limited to 'arm/Op.v')
-rw-r--r--arm/Op.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/arm/Op.v b/arm/Op.v
index 7a25511..5e85aae 100644
--- a/arm/Op.v
+++ b/arm/Op.v
@@ -24,6 +24,7 @@
syntax and dynamic semantics of the Cminor language.
*)
+Require Import Axioms.
Require Import Coqlib.
Require Import AST.
Require Import Integers.
@@ -132,7 +133,7 @@ Proof.
generalize Int.eq_dec; intro.
assert (forall (x y: shift_amount), {x=y}+{x<>y}).
destruct x as [x Px]. destruct y as [y Py]. destruct (H x y).
- subst x. rewrite (proof_irrelevance _ Px Py). left; auto.
+ subst x. rewrite (proof_irr Px Py). left; auto.
right. red; intro. elim n. inversion H0. auto.
decide equality.
Qed.