summaryrefslogtreecommitdiff
path: root/cfrontend
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-10 12:13:12 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2013-03-10 12:13:12 +0000
commit02779dbc71c0f6985427c47ec05dd25b44dd859c (patch)
treecdff116e8c7e5d82ae6943428018f39d1ce81d60 /cfrontend
parente29b0c71f446ea6267711c7cc19294fd93fb81ad (diff)
Glasnost: making transparent a number of definitions that were opaque
for no good reason. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2140 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend')
-rw-r--r--cfrontend/Cexec.v7
-rw-r--r--cfrontend/Cshmgen.v7
-rw-r--r--cfrontend/Initializersproof.v8
3 files changed, 8 insertions, 14 deletions
diff --git a/cfrontend/Cexec.v b/cfrontend/Cexec.v
index c638259..ebc27ad 100644
--- a/cfrontend/Cexec.v
+++ b/cfrontend/Cexec.v
@@ -92,7 +92,7 @@ Fixpoint is_val_list (al: exprlist) : option (list (val * type)) :=
Definition is_skip (s: statement) : {s = Sskip} + {s <> Sskip}.
Proof.
destruct s; (left; congruence) || (right; congruence).
-Qed.
+Defined.
(** * Events, volatile memory accesses, and external functions. *)
@@ -303,7 +303,7 @@ Proof with try (right; intuition omega).
destruct (zle (Int.unsigned ofs + sizeof ty) (Int.unsigned ofs')); auto.
right; intuition omega.
destruct Y... left; intuition omega.
-Qed.
+Defined.
Definition do_assign_loc (w: world) (ty: type) (m: mem) (b: block) (ofs: int) (v: val): option (world * trace * mem) :=
match access_mode ty with
@@ -464,7 +464,7 @@ Proof with try (right; intuition omega).
destruct (zle (odst + sz) osrc); auto.
right; intuition omega.
destruct Y... left; intuition omega.
-Qed.
+Defined.
Definition do_ef_memcpy (sz al: Z)
(w: world) (vargs: list val) (m: mem) : option (world * trace * val * mem) :=
@@ -2180,7 +2180,6 @@ Proof with (unfold ret; auto with coqlib).
rewrite H0...
rewrite H0...
rewrite pred_dec_false...
- rewrite pred_dec_true...
rewrite H0...
rewrite H0...
destruct H0; subst x...
diff --git a/cfrontend/Cshmgen.v b/cfrontend/Cshmgen.v
index 9d518cb..51f89da 100644
--- a/cfrontend/Cshmgen.v
+++ b/cfrontend/Cshmgen.v
@@ -486,11 +486,8 @@ Definition transl_function (f: Clight.function) : res function :=
(map fst (Clight.fn_temps f))
tbody).
-Definition list_typ_eq:
- forall (l1 l2: list typ), {l1=l2} + {l1<>l2}.
-Proof.
- generalize typ_eq; intro. decide equality.
-Qed.
+Definition list_typ_eq: forall (l1 l2: list typ), {l1=l2} + {l1<>l2}
+ := list_eq_dec typ_eq.
Definition transl_fundef (f: Clight.fundef) : res fundef :=
match f with
diff --git a/cfrontend/Initializersproof.v b/cfrontend/Initializersproof.v
index b64c309..b0884ac 100644
--- a/cfrontend/Initializersproof.v
+++ b/cfrontend/Initializersproof.v
@@ -397,13 +397,11 @@ Proof.
Opaque zeq.
intros. unfold sem_cmp in *.
destruct (classify_cmp ty1 ty2); try (destruct s); inv H1; inv H2; inv H; inv H0; auto with mval.
- destruct (Int.eq n Int.zero); try discriminate.
+- destruct (Int.eq n Int.zero); try discriminate.
unfold Val.cmp_different_blocks in *. destruct c; inv H3; inv H2; constructor.
- destruct (Int.eq n Int.zero); try discriminate.
+- destruct (Int.eq n Int.zero); try discriminate.
unfold Val.cmp_different_blocks in *. destruct c; inv H2; inv H1; constructor.
- rewrite (mem_empty_not_valid_pointer (Zpos id) (Int.unsigned ofs)) in H4.
- rewrite (mem_empty_not_weak_valid_pointer (Zpos id) (Int.unsigned ofs)) in H4. simpl in H4.
- destruct (zeq (Z.pos id) (Z.pos id0)); discriminate.
+- destruct (zeq (Z.pos id) (Z.pos id0)); discriminate.
Qed.
Lemma sem_binary_match: