aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Coqlib.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-05-21 16:26:30 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-05-21 16:26:30 +0000
commit0053b1aa1d26da5d1f995a603b127daf799c2da9 (patch)
treefec49ad37e5edffa5be742bafcadff3c8b8ede7f /lib/Coqlib.v
parent219a2d178dcd5cc625f6b6261759f392cfca367b (diff)
downloadcompcert-kvx-0053b1aa1d26da5d1f995a603b127daf799c2da9.tar.gz
compcert-kvx-0053b1aa1d26da5d1f995a603b127daf799c2da9.zip
Merge of the newmem branch:
- Revised memory model with Max and Cur permissions, but without bounds - Constant propagation of 'const' globals - Function inlining at RTL level - (Unprovable) elimination of unreferenced static definitions git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1899 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'lib/Coqlib.v')
-rw-r--r--lib/Coqlib.v19
1 files changed, 1 insertions, 18 deletions
diff --git a/lib/Coqlib.v b/lib/Coqlib.v
index 87b19ca8..50535fb1 100644
--- a/lib/Coqlib.v
+++ b/lib/Coqlib.v
@@ -23,23 +23,6 @@ Require Export List.
Require Export Bool.
Require Import Wf_nat.
-(***
-
-(** * Logical axioms *)
-
-(** We use two logical axioms that are not provable in Coq but consistent
- with the logic: function extensionality and proof irrelevance.
- These are used in the memory model to show that two memory states
- that have identical contents are equal. *)
-
-Axiom extensionality:
- forall (A B: Type) (f g : A -> B),
- (forall x, f x = g x) -> f = g.
-
-Axiom proof_irrelevance:
- forall (P: Prop) (p1 p2: P), p1 = p2.
-***)
-
(** * Useful tactics *)
Ltac inv H := inversion H; clear H; subst.
@@ -51,7 +34,7 @@ Ltac caseEq name :=
generalize (refl_equal name); pattern name at -1 in |- *; case name.
Ltac destructEq name :=
- generalize (refl_equal name); pattern name at -1 in |- *; destruct name; intro.
+ destruct name as []_eqn.
Ltac decEq :=
match goal with