Mercurial > cpdt > repo
diff src/DataStruct.v @ 534:ed829eaa91b2
Builds with Coq 8.5beta2
author | Adam Chlipala <adam@chlipala.net> |
---|---|
date | Wed, 05 Aug 2015 14:46:55 -0400 |
parents | 28c2fa8af4eb |
children | 81d63d9c1cc5 |
line wrap: on
line diff
--- a/src/DataStruct.v Tue Apr 07 18:59:24 2015 -0400 +++ b/src/DataStruct.v Wed Aug 05 14:46:55 2015 -0400 @@ -1,4 +1,4 @@ -(* Copyright (c) 2008-2012, Adam Chlipala +(* Copyright (c) 2008-2012, 2015, Adam Chlipala * * This work is licensed under a * Creative Commons Attribution-Noncommercial-No Derivative Works 3.0 @@ -10,9 +10,10 @@ (* begin hide *) Require Import Arith List. -Require Import CpdtTactics. +Require Import Cpdt.CpdtTactics. Set Implicit Arguments. +Set Asymmetric Patterns. (* end hide *) @@ -489,6 +490,11 @@ (** %\index{index function}%Indexed lists can be useful in defining other inductive types with constructors that take variable numbers of arguments. In this section, we consider parameterized trees with arbitrary branching factor. *) +(* begin hide *) +Definition red_herring := O. +(* working around a bug in Coq 8.5! *) +(* end hide *) + Section tree. Variable A : Set. @@ -553,6 +559,10 @@ Abort. Reset tree. +(* begin hide *) +Reset red_herring. +(* working around a bug in Coq 8.5! *) +(* end hide *) (** First, let us try using our recursive definition of [ilist]s instead of the inductive version. *)