Mercurial > cpdt > repo
diff src/Exercises.v @ 534:ed829eaa91b2
Builds with Coq 8.5beta2
author | Adam Chlipala <adam@chlipala.net> |
---|---|
date | Wed, 05 Aug 2015 14:46:55 -0400 |
parents | 5f25705a10ea |
children |
line wrap: on
line diff
--- a/src/Exercises.v Tue Apr 07 18:59:24 2015 -0400 +++ b/src/Exercises.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,7 +10,7 @@ (* begin hide *) Require Import List. -Require Import CpdtTactics. +Require Import Cpdt.CpdtTactics. (* end hide *) (** These exercises were originally included inline in the text, but my latest feeling is that I don't have the time to maintain the exercises at a sufficient quality level to match the level I'm targetting for the rest of the book. I'm including them in this file for now. *)