diff options
author | Adam Chlipala <adamc@hcoop.net> | 2009-02-21 13:17:06 -0500 |
---|---|---|
committer | Adam Chlipala <adamc@hcoop.net> | 2009-02-21 13:17:06 -0500 |
commit | e4b9964e2f79cac5eff8ef728560cc539d256cb3 (patch) | |
tree | 0c5d6549cc3f28a18b48f2a8a0cd2b4002e45428 /src/coq/Axioms.v | |
parent | 06c8fa2f35ba45081eca93d4ff6666eb83d16037 (diff) |
Most of expression semantics
Diffstat (limited to 'src/coq/Axioms.v')
-rw-r--r-- | src/coq/Axioms.v | 2 |
1 files changed, 0 insertions, 2 deletions
diff --git a/src/coq/Axioms.v b/src/coq/Axioms.v index f89bc1e8..0a0a84dc 100644 --- a/src/coq/Axioms.v +++ b/src/coq/Axioms.v @@ -25,8 +25,6 @@ * POSSIBILITY OF SUCH DAMAGE. *) -Require Import Syntax. - Set Implicit Arguments. |