diff options
Diffstat (limited to 'theories/Program/Syntax.v')
| -rw-r--r-- | theories/Program/Syntax.v | 2 |
1 files changed, 0 insertions, 2 deletions
diff --git a/theories/Program/Syntax.v b/theories/Program/Syntax.v index 2064977fef..916c33ee62 100644 --- a/theories/Program/Syntax.v +++ b/theories/Program/Syntax.v @@ -35,8 +35,6 @@ Implicit Arguments pair [[A] [B]]. Implicit Arguments fst [[A] [B]]. Implicit Arguments snd [[A] [B]]. -Require Import Coq.Lists.List. - Implicit Arguments nil [[A]]. Implicit Arguments cons [[A]]. |
