aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Coqlib.v
diff options
context:
space:
mode:
Diffstat (limited to 'lib/Coqlib.v')
-rw-r--r--lib/Coqlib.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/lib/Coqlib.v b/lib/Coqlib.v
index 75e158bd..4fc922b1 100644
--- a/lib/Coqlib.v
+++ b/lib/Coqlib.v
@@ -23,6 +23,8 @@ 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
@@ -36,7 +38,8 @@ Axiom extensionality:
Axiom proof_irrelevance:
forall (P: Prop) (p1 p2: P), p1 = p2.
-
+***)
+
(** * Useful tactics *)
Ltac inv H := inversion H; clear H; subst.