MoreDep.v 64 KB
Newer Older
1
(* Copyright (c) 2008-2012, Adam Chlipala
Adam Chlipala's avatar
Adam Chlipala committed
2 3 4 5 6 7 8 9 10
 * 
 * This work is licensed under a
 * Creative Commons Attribution-Noncommercial-No Derivative Works 3.0
 * Unported License.
 * The license text is available at:
 *   http://creativecommons.org/licenses/by-nc-nd/3.0/
 *)

(* begin hide *)
11
Require Import Arith Bool List.
Adam Chlipala's avatar
Adam Chlipala committed
12

13
Require Import CpdtTactics MoreSpecif.
Adam Chlipala's avatar
Adam Chlipala committed
14 15 16 17 18 19 20

Set Implicit Arguments.
(* end hide *)


(** %\chapter{More Dependent Types}% *)

21
(** Subset types and their relatives help us integrate verification with programming.  Though they reorganize the certified programmer's workflow, they tend not to have deep effects on proofs.  We write largely the same proofs as we would for classical verification, with some of the structure moved into the programs themselves.  It turns out that, when we use dependent types to their full potential, we warp the development and proving process even more than that, picking up %``%#"#free theorems#"#%''% to the extent that often a certified program is hardly more complex than its uncertified counterpart in Haskell or ML.
Adam Chlipala's avatar
Adam Chlipala committed
22

Adam Chlipala's avatar
Adam Chlipala committed
23
   In particular, we have only scratched the tip of the iceberg that is Coq's inductive definition mechanism.  The inductive types we have seen so far have their counterparts in the other proof assistants that we surveyed in Chapter 1.  This chapter explores the strange new world of dependent inductive datatypes (that is, dependent inductive types outside [Prop]), a possibility that sets Coq apart from all of the competition not based on type theory. *)
Adam Chlipala's avatar
Adam Chlipala committed
24

25 26 27

(** * Length-Indexed Lists *)

Adam Chlipala's avatar
Adam Chlipala committed
28
(** Many introductions to dependent types start out by showing how to use them to eliminate array bounds checks%\index{array bounds checks}%.  When the type of an array tells you how many elements it has, your compiler can detect out-of-bounds dereferences statically.  Since we are working in a pure functional language, the next best thing is length-indexed lists%\index{length-indexed lists}%, which the following code defines. *)
29 30 31 32 33 34 35 36 37 38

Section ilist.
  Variable A : Set.

  Inductive ilist : nat -> Set :=
  | Nil : ilist O
  | Cons : forall n, A -> ilist n -> ilist (S n).

(** We see that, within its section, [ilist] is given type [nat -> Set].  Previously, every inductive type we have seen has either had plain [Set] as its type or has been a predicate with some type ending in [Prop].  The full generality of inductive definitions lets us integrate the expressivity of predicates directly into our normal programming.

39
   The [nat] argument to [ilist] tells us the length of the list.  The types of [ilist]'s constructors tell us that a [Nil] list has length [O] and that a [Cons] list has length one greater than the length of its tail.  We may apply [ilist] to any natural number, even natural numbers that are only known at runtime.  It is this breaking of the%\index{phase distinction}% _phase distinction_ that characterizes [ilist] as _dependently typed_.
40

41
   In expositions of list types, we usually see the length function defined first, but here that would not be a very productive function to code.  Instead, let us implement list concatenation. *)
42

43 44 45 46 47
  Fixpoint app n1 (ls1 : ilist n1) n2 (ls2 : ilist n2) : ilist (n1 + n2) :=
    match ls1 with
      | Nil => ls2
      | Cons _ x ls1' => Cons x (app ls1' ls2)
    end.
48

Adam Chlipala's avatar
Adam Chlipala committed
49
  (** Past Coq versions signalled an error for this definition.  The code is still invalid within Coq's core language, but current Coq versions automatically add annotations to the original program, producing a valid core program.  These are the annotations on [match] discriminees that we began to study in the previous chapter.  We can rewrite [app] to give the annotations explicitly. *)
Adam Chlipala's avatar
Adam Chlipala committed
50 51

(* begin thide *)
Adam Chlipala's avatar
Adam Chlipala committed
52 53 54 55 56
  Fixpoint app' n1 (ls1 : ilist n1) n2 (ls2 : ilist n2) : ilist (n1 + n2) :=
    match ls1 in (ilist n1) return (ilist (n1 + n2)) with
      | Nil => ls2
      | Cons _ x ls1' => Cons x (app' ls1' ls2)
    end.
Adam Chlipala's avatar
Adam Chlipala committed
57
(* end thide *)
58

59
(** Using [return] alone allowed us to express a dependency of the [match] result type on the _value_ of the discriminee.  What %\index{Gallina terms!in}%[in] adds to our arsenal is a way of expressing a dependency on the _type_ of the discriminee.  Specifically, the [n1] in the [in] clause above is a _binding occurrence_ whose scope is the [return] clause.
60

61
We may use [in] clauses only to bind names for the arguments of an inductive type family.  That is, each [in] clause must be an inductive type family name applied to a sequence of underscores and variable names of the proper length.  The positions for _parameters_ to the type family must all be underscores.  Parameters are those arguments declared with section variables or with entries to the left of the first colon in an inductive definition.  They cannot vary depending on which constructor was used to build the discriminee, so Coq prohibits pointless matches on them.  It is those arguments defined in the type to the right of the colon that we may name with [in] clauses.
62

63
Our [app] function could be typed in so-called%\index{stratified type systems}% _stratified_ type systems, which avoid true dependency.  That is, we could consider the length indices to lists to live in a separate, compile-time-only universe from the lists themselves.  This stratification between a compile-time universe and a run-time universe, with no references to the latter in the former, gives rise to the terminology %``%#"#stratified.#"#%''%  Our next example would be harder to implement in a stratified system.  We write an injection function from regular lists to length-indexed lists.  A stratified implementation would need to duplicate the definition of lists across compile-time and run-time versions, and the run-time versions would need to be indexed by the compile-time versions. *)
64

Adam Chlipala's avatar
Adam Chlipala committed
65 66 67
(* EX: Implement injection from normal lists *)

(* begin thide *)
68
Fixpoint inject (ls : list A) : ilist (length ls) :=
69
  match ls with
70 71 72 73 74 75
    | nil => Nil
    | h :: t => Cons h (inject t)
  end.

(** We can define an inverse conversion and prove that it really is an inverse. *)

76
Fixpoint unject n (ls : ilist n) : list A :=
77 78 79 80 81 82 83 84
  match ls with
    | Nil => nil
    | Cons _ h t => h :: unject t
  end.

Theorem inject_inverse : forall ls, unject (inject ls) = ls.
  induction ls; crush.
Qed.
Adam Chlipala's avatar
Adam Chlipala committed
85 86
(* end thide *)

Adam Chlipala's avatar
Adam Chlipala committed
87
(* EX: Implement statically checked "car"/"hd" *)
88

Adam Chlipala's avatar
Adam Chlipala committed
89
(** Now let us attempt a function that is surprisingly tricky to write.  In ML, the list head function raises an exception when passed an empty list.  With length-indexed lists, we can rule out such invalid calls statically, and here is a first attempt at doing so.  We write [???] as a placeholder for a term that we do not know how to write, not for any real Coq notation like those introduced in the previous chapter.
90 91 92 93 94 95 96

[[
Definition hd n (ls : ilist (S n)) : A :=
  match ls with
    | Nil => ???
    | Cons _ h _ => h
  end.
97 98
 
]]
99 100 101 102 103 104 105 106

It is not clear what to write for the [Nil] case, so we are stuck before we even turn our function over to the type checker.  We could try omitting the [Nil] case:

[[
Definition hd n (ls : ilist (S n)) : A :=
  match ls with
    | Cons _ h _ => h
  end.
Adam Chlipala's avatar
Adam Chlipala committed
107
]]
108

Adam Chlipala's avatar
Adam Chlipala committed
109
<<
110
Error: Non exhaustive pattern-matching: no clause found for pattern Nil
Adam Chlipala's avatar
Adam Chlipala committed
111
>>
112

113
Unlike in ML, we cannot use inexhaustive pattern matching, because there is no conception of a %\texttt{%#<tt>#Match#</tt>#%}% exception to be thrown.  In fact, recent versions of Coq _do_ allow this, by implicit translation to a [match] that considers all constructors.  It is educational to discover that encoding ourselves directly.  We might try using an [in] clause somehow.
114 115 116 117 118 119

[[
Definition hd n (ls : ilist (S n)) : A :=
  match ls in (ilist (S n)) with
    | Cons _ h _ => h
  end.
Adam Chlipala's avatar
Adam Chlipala committed
120
]]
121

Adam Chlipala's avatar
Adam Chlipala committed
122
<<
123
Error: The reference n was not found in the current environment
Adam Chlipala's avatar
Adam Chlipala committed
124
>>
125

126
In this and other cases, we feel like we want [in] clauses with type family arguments that are not variables.  Unfortunately, Coq only supports variables in those positions.  A completely general mechanism could only be supported with a solution to the problem of higher-order unification%~\cite{HOU}%, which is undecidable.  There _are_ useful heuristics for handling non-variable indices which are gradually making their way into Coq, but we will spend some time in this and the next few chapters on effective pattern matching on dependent types using only the primitive [match] annotations.
127 128 129

Our final, working attempt at [hd] uses an auxiliary function and a surprising [return] annotation. *)

Adam Chlipala's avatar
Adam Chlipala committed
130
(* begin thide *)
131 132 133 134 135 136
Definition hd' n (ls : ilist n) :=
  match ls in (ilist n) return (match n with O => unit | S _ => A end) with
    | Nil => tt
    | Cons _ h _ => h
  end.

Adam Chlipala's avatar
Adam Chlipala committed
137 138 139 140 141 142 143 144
Check hd'.
(** %\vspace{-.15in}% [[
hd'
     : forall n : nat, ilist n -> match n with
                                  | 0 => unit
                                  | S _ => A
                                  end
 
145 146
  ]]
  *)
Adam Chlipala's avatar
Adam Chlipala committed
147

148
Definition hd n (ls : ilist (S n)) : A := hd' ls.
Adam Chlipala's avatar
Adam Chlipala committed
149
(* end thide *)
150 151

End ilist.
152

Adam Chlipala's avatar
Adam Chlipala committed
153 154
(** We annotate our main [match] with a type that is itself a [match].  We write that the function [hd'] returns [unit] when the list is empty and returns the carried type [A] in all other cases.  In the definition of [hd], we just call [hd'].  Because the index of [ls] is known to be nonzero, the type checker reduces the [match] in the type of [hd'] to [A]. *)

155

156 157
(** * The One Rule of Dependent Pattern Matching in Coq *)

158
(** The rest of this chapter will demonstrate a few other elegant applications of dependent types in Coq.  Readers encountering such ideas for the first time often feel overwhelmed, concluding that there is some magic at work whereby Coq sometimes solves the halting problem for the programmer and sometimes does not, applying automated program understanding in a way far beyond what is found in conventional languages.  The point of this section is to cut off that sort of thinking right now!  Dependent type-checking in Coq follows just a few algorithmic rules.  Chapters 10 and 12 introduce many of those rules more formally, and the main additional rule is centered on%\index{dependent pattern matching}% _dependent pattern matching_ of the kind we met in the previous section.
159

160
A dependent pattern match is a [match] expression where the type of the overall [match] is a function of the value and/or the type of the%\index{discriminee}% _discriminee_, the value being matched on.  In other words, the [match] type _depends_ on the discriminee.
161

162
When exactly will Coq accept a dependent pattern match as well-typed?  Some other dependently typed languages employ fancy decision procedures to determine when programs satisfy their very expressive types.  The situation in Coq is just the opposite.  Only very straightforward symbolic rules are applied.  Such a design choice has its drawbacks, as it forces programmers to do more work to convince the type checker of program validity.  However, the great advantage of a simple type checking algorithm is that its action on _invalid_ programs is easier to understand!
163 164 165 166 167 168 169 170 171 172 173 174 175 176 177 178 179 180 181

We come now to the one rule of dependent pattern matching in Coq.  A general dependent pattern match assumes this form (with unnecessary parentheses included to make the syntax easier to parse):
[[
  match E in (T x1 ... xn) as y return U with
    | C z1 ... zm => B
    | ...
  end
]]

The discriminee is a term [E], a value in some inductive type family [T], which takes [n] arguments.  An %\index{in clause}%[in] clause binds an explicit name [xi] for the [i]th argument passed to [T] in the type of [E].  An %\index{as clause}%[as] clause binds the name [y] to refer to the discriminee [E].

We bind these new variables [xi] and [y] so that they may be referred to in [U], a type given in the %\index{return clause}%[return] clause.  The overall type of the [match] will be [U], with [E] substituted for [y], and with each [xi] substituted by the actual argument appearing in that position within [E]'s type.

In general, each case of a [match] may have a pattern built up in several layers from the constructors of various inductive type families.  To keep this exposition simple, we will focus on patterns that are just single applications of inductive type constructors to lists of variables.  Coq actually compiles the more general kind of pattern matching into this more restricted kind automatically, so understanding the typing of [match] requires understanding the typing of [match]es lowered to match one constructor at a time.

The last piece of the typing rule tells how to type-check a [match] case.  A generic constructor application [C z1 ... zm] has some type [T x1' ... xn'], an application of the type family used in [E]'s type, probably with occurrences of the [zi] variables.  From here, a simple recipe determines what type we will require for the case body [B].  The type of [B] should be [U] with the following two substitutions applied: we replace [y] (the [as] clause variable) with [C z1 ... zm], and we replace each [xi] (the [in] clause variables) with [xi'].  In other words, we specialize the result type based on what we learn based on which pattern has matched the discriminee.

This is an exhaustive description of the ways to specify how to take advantage of which pattern has matched!  No other mechanisms come into play.  For instance, there is no way to specify that the types of certain free variables should be refined based on which pattern has matched.  In the rest of the book, we will learn design patterns for achieving similar effects, where each technique leads to an encoding only in terms of [in], [as], and [return] clauses.

182
A few details have been omitted above.  In Chapter 3, we learned that inductive type families may have both%\index{parameters}% _parameters_ and regular arguments.  Within an [in] clause, a parameter position must have the wildcard [_] written, instead of a variable.  (In general, Coq uses wildcard [_]'s either to indicate pattern variables that will not be mentioned again or to indicate positions where we would like type inference to infer the appropriate terms.)  Furthermore, recent Coq versions are adding more and more heuristics to infer dependent [match] annotations in certain conditions.  The general annotation inference problem is undecidable, so there will always be serious limitations on how much work these heuristics can do.  When in doubt about why a particular dependent [match] is failing to type-check, add an explicit [return] annotation!  At that point, the mechanical rule sketched in this section will provide a complete account of %``%#"#what the type checker is thinking.#"#%''%  Be sure to avoid the common pitfall of writing a [return] annotation that does not mention any variables bound by [in] or [as]; such a [match] will never refine typing requirements based on which pattern has matched.  (One simple exception to this rule is that, when the discriminee is a variable, that same variable may be treated as if it were repeated as an [as] clause.) *)
183 184


185 186
(** * A Tagless Interpreter *)

187
(** A favorite example for motivating the power of functional programming is implementation of a simple expression language interpreter.  In ML and Haskell, such interpreters are often implemented using an algebraic datatype of values, where at many points it is checked that a value was built with the right constructor of the value type.  With dependent types, we can implement a%\index{tagless interpreters}% _tagless_ interpreter that both removes this source of runtime inefficiency and gives us more confidence that our implementation is correct. *)
188 189 190 191 192 193 194 195 196 197 198 199 200 201 202 203 204 205 206 207 208

Inductive type : Set :=
| Nat : type
| Bool : type
| Prod : type -> type -> type.

Inductive exp : type -> Set :=
| NConst : nat -> exp Nat
| Plus : exp Nat -> exp Nat -> exp Nat
| Eq : exp Nat -> exp Nat -> exp Bool

| BConst : bool -> exp Bool
| And : exp Bool -> exp Bool -> exp Bool
| If : forall t, exp Bool -> exp t -> exp t -> exp t

| Pair : forall t1 t2, exp t1 -> exp t2 -> exp (Prod t1 t2)
| Fst : forall t1 t2, exp (Prod t1 t2) -> exp t1
| Snd : forall t1 t2, exp (Prod t1 t2) -> exp t2.

(** We have a standard algebraic datatype [type], defining a type language of naturals, booleans, and product (pair) types.  Then we have the indexed inductive type [exp], where the argument to [exp] tells us the encoded type of an expression.  In effect, we are defining the typing rules for expressions simultaneously with the syntax.

209
   We can give types and expressions semantics in a new style, based critically on the chance for _type-level computation_. *)
210 211 212 213 214 215 216 217

Fixpoint typeDenote (t : type) : Set :=
  match t with
    | Nat => nat
    | Bool => bool
    | Prod t1 t2 => typeDenote t1 * typeDenote t2
  end%type.

218
(** The [typeDenote] function compiles types of our object language into %``%#"#native#"#%''% Coq types.  It is deceptively easy to implement.  The only new thing we see is the [%]%\coqdocvar{%#<tt>#type#</tt>#%}% annotation, which tells Coq to parse the [match] expression using the notations associated with types.  Without this annotation, the [*] would be interpreted as multiplication on naturals, rather than as the product type constructor.  The token %\coqdocvar{%#<tt>#type#</tt>#%}% is one example of an identifer bound to a%\index{notation scope delimiter}% _notation scope delimiter_.  In this book, we will not go into more detail on notation scopes, but the Coq manual can be consulted for more information.
219 220 221

   We can define a function [expDenote] that is typed in terms of [typeDenote]. *)

222 223
Fixpoint expDenote t (e : exp t) : typeDenote t :=
  match e with
224 225 226 227 228 229 230 231 232 233 234 235 236
    | NConst n => n
    | Plus e1 e2 => expDenote e1 + expDenote e2
    | Eq e1 e2 => if eq_nat_dec (expDenote e1) (expDenote e2) then true else false

    | BConst b => b
    | And e1 e2 => expDenote e1 && expDenote e2
    | If _ e' e1 e2 => if expDenote e' then expDenote e1 else expDenote e2

    | Pair _ _ e1 e2 => (expDenote e1, expDenote e2)
    | Fst _ _ e' => fst (expDenote e')
    | Snd _ _ e' => snd (expDenote e')
  end.

237
(** Despite the fancy type, the function definition is routine.  In fact, it is less complicated than what we would write in ML or Haskell 98, since we do not need to worry about pushing final values in and out of an algebraic datatype.  The only unusual thing is the use of an expression of the form [if E then true else false] in the [Eq] case.  Remember that [eq_nat_dec] has a rich dependent type, rather than a simple boolean type.  Coq's native [if] is overloaded to work on a test of any two-constructor type, so we can use [if] to build a simple boolean from the [sumbool] that [eq_nat_dec] returns.
238 239 240 241 242 243 244 245 246

   We can implement our old favorite, a constant folding function, and prove it correct.  It will be useful to write a function [pairOut] that checks if an [exp] of [Prod] type is a pair, returning its two components if so.  Unsurprisingly, a first attempt leads to a type error.

[[
Definition pairOut t1 t2 (e : exp (Prod t1 t2)) : option (exp t1 * exp t2) :=
  match e in (exp (Prod t1 t2)) return option (exp t1 * exp t2) with
    | Pair _ _ e1 e2 => Some (e1, e2)
    | _ => None
  end.
Adam Chlipala's avatar
Adam Chlipala committed
247
]]
248

Adam Chlipala's avatar
Adam Chlipala committed
249
<<
250
Error: The reference t2 was not found in the current environment
Adam Chlipala's avatar
Adam Chlipala committed
251
>>
252 253 254

We run again into the problem of not being able to specify non-variable arguments in [in] clauses.  The problem would just be hopeless without a use of an [in] clause, though, since the result type of the [match] depends on an argument to [exp].  Our solution will be to use a more general type, as we did for [hd].  First, we define a type-valued function to use in assigning a type to [pairOut]. *)

Adam Chlipala's avatar
Adam Chlipala committed
255 256 257
(* EX: Define a function [pairOut : forall t1 t2, exp (Prod t1 t2) -> option (exp t1 * exp t2)] *)

(* begin thide *)
258 259 260 261 262 263 264 265 266 267 268 269 270 271 272 273 274 275 276 277 278
Definition pairOutType (t : type) :=
  match t with
    | Prod t1 t2 => option (exp t1 * exp t2)
    | _ => unit
  end.

(** When passed a type that is a product, [pairOutType] returns our final desired type.  On any other input type, [pairOutType] returns [unit], since we do not care about extracting components of non-pairs.  Now we can write another helper function to provide the default behavior of [pairOut], which we will apply for inputs that are not literal pairs. *)

Definition pairOutDefault (t : type) :=
  match t return (pairOutType t) with
    | Prod _ _ => None
    | _ => tt
  end.

(** Now [pairOut] is deceptively easy to write. *)

Definition pairOut t (e : exp t) :=
  match e in (exp t) return (pairOutType t) with
    | Pair _ _ e1 e2 => Some (e1, e2)
    | _ => pairOutDefault _
  end.
Adam Chlipala's avatar
Adam Chlipala committed
279
(* end thide *)
280

Adam Chlipala's avatar
Adam Chlipala committed
281
(** There is one important subtlety in this definition.  Coq allows us to use convenient ML-style pattern matching notation, but, internally and in proofs, we see that patterns are expanded out completely, matching one level of inductive structure at a time.  Thus, the default case in the [match] above expands out to one case for each constructor of [exp] besides [Pair], and the underscore in [pairOutDefault _] is resolved differently in each case.  From an ML or Haskell programmer's perspective, what we have here is type inference determining which code is run (returning either [None] or [tt]), which goes beyond what is possible with type inference guiding parametric polymorphism in Hindley-Milner languages%\index{Hindley-Milner}%, but is similar to what goes on with Haskell type classes%\index{type classes}%.
282

283
With [pairOut] available, we can write [cfold] in a straightforward way.  There are really no surprises beyond that Coq verifies that this code has such an expressive type, given the small annotation burden.  In some places, we see that Coq's [match] annotation inference is too smart for its own good, and we have to turn that inference with explicit [return] clauses. *)
284

285 286
Fixpoint cfold t (e : exp t) : exp t :=
  match e with
287 288 289 290
    | NConst n => NConst n
    | Plus e1 e2 =>
      let e1' := cfold e1 in
      let e2' := cfold e2 in
291
      match e1', e2' return exp Nat with
292 293 294 295 296 297
        | NConst n1, NConst n2 => NConst (n1 + n2)
        | _, _ => Plus e1' e2'
      end
    | Eq e1 e2 =>
      let e1' := cfold e1 in
      let e2' := cfold e2 in
298
      match e1', e2' return exp Bool with
299 300 301 302 303 304 305 306
        | NConst n1, NConst n2 => BConst (if eq_nat_dec n1 n2 then true else false)
        | _, _ => Eq e1' e2'
      end

    | BConst b => BConst b
    | And e1 e2 =>
      let e1' := cfold e1 in
      let e2' := cfold e2 in
307
      match e1', e2' return exp Bool with
308 309 310 311 312 313 314 315 316 317 318 319 320 321 322 323 324 325 326 327 328 329 330 331 332 333 334 335 336
        | BConst b1, BConst b2 => BConst (b1 && b2)
        | _, _ => And e1' e2'
      end
    | If _ e e1 e2 =>
      let e' := cfold e in
      match e' with
        | BConst true => cfold e1
        | BConst false => cfold e2
        | _ => If e' (cfold e1) (cfold e2)
      end

    | Pair _ _ e1 e2 => Pair (cfold e1) (cfold e2)
    | Fst _ _ e =>
      let e' := cfold e in
      match pairOut e' with
        | Some p => fst p
        | None => Fst e'
      end
    | Snd _ _ e =>
      let e' := cfold e in
      match pairOut e' with
        | Some p => snd p
        | None => Snd e'
      end
  end.

(** The correctness theorem for [cfold] turns out to be easy to prove, once we get over one serious hurdle. *)

Theorem cfold_correct : forall t (e : exp t), expDenote e = expDenote (cfold e).
Adam Chlipala's avatar
Adam Chlipala committed
337
(* begin thide *)
338 339 340 341 342 343 344 345 346 347 348 349 350 351 352 353 354 355 356 357 358 359 360 361 362 363 364 365 366
  induction e; crush.

(** The first remaining subgoal is:

   [[
  expDenote (cfold e1) + expDenote (cfold e2) =
   expDenote
     match cfold e1 with
     | NConst n1 =>
         match cfold e2 with
         | NConst n2 => NConst (n1 + n2)
         | Plus _ _ => Plus (cfold e1) (cfold e2)
         | Eq _ _ => Plus (cfold e1) (cfold e2)
         | BConst _ => Plus (cfold e1) (cfold e2)
         | And _ _ => Plus (cfold e1) (cfold e2)
         | If _ _ _ _ => Plus (cfold e1) (cfold e2)
         | Pair _ _ _ _ => Plus (cfold e1) (cfold e2)
         | Fst _ _ _ => Plus (cfold e1) (cfold e2)
         | Snd _ _ _ => Plus (cfold e1) (cfold e2)
         end
     | Plus _ _ => Plus (cfold e1) (cfold e2)
     | Eq _ _ => Plus (cfold e1) (cfold e2)
     | BConst _ => Plus (cfold e1) (cfold e2)
     | And _ _ => Plus (cfold e1) (cfold e2)
     | If _ _ _ _ => Plus (cfold e1) (cfold e2)
     | Pair _ _ _ _ => Plus (cfold e1) (cfold e2)
     | Fst _ _ _ => Plus (cfold e1) (cfold e2)
     | Snd _ _ _ => Plus (cfold e1) (cfold e2)
     end
367
 
368 369 370 371 372 373
     ]]

     We would like to do a case analysis on [cfold e1], and we attempt that in the way that has worked so far.

     [[
  destruct (cfold e1).
Adam Chlipala's avatar
Adam Chlipala committed
374
]]
375

Adam Chlipala's avatar
Adam Chlipala committed
376
<<
377
User error: e1 is used in hypothesis e
Adam Chlipala's avatar
Adam Chlipala committed
378
>>
379 380 381

    Coq gives us another cryptic error message.  Like so many others, this one basically means that Coq is not able to build some proof about dependent types.  It is hard to generate helpful and specific error messages for problems like this, since that would require some kind of understanding of the dependency structure of a piece of code.  We will encounter many examples of case-specific tricks for recovering from errors like this one.

Adam Chlipala's avatar
Adam Chlipala committed
382
    For our current proof, we can use a tactic [dep_destruct]%\index{tactics!dep\_destruct}% defined in the book [CpdtTactics] module.  General elimination/inversion of dependently typed hypotheses is undecidable, since it must be implemented with [match] expressions that have the restriction on [in] clauses that we have already discussed.  The tactic [dep_destruct] makes a best effort to handle some common cases, relying upon the more primitive %\index{tactics!dependent destruction}%[dependent destruction] tactic that comes with Coq.  In a future chapter, we will learn about the explicit manipulation of equality proofs that is behind [dep_destruct]'s implementation in Ltac, but for now, we treat it as a useful black box.  (In Chapter 12, we will also see how [dependent destruction] forces us to make a larger philosophical commitment about our logic than we might like, and we will see some workarounds.) *)
383 384 385 386 387
  
  dep_destruct (cfold e1).

  (** This successfully breaks the subgoal into 5 new subgoals, one for each constructor of [exp] that could produce an [exp Nat].  Note that [dep_destruct] is successful in ruling out the other cases automatically, in effect automating some of the work that we have done manually in implementing functions like [hd] and [pairOut].

388
     This is the only new trick we need to learn to complete the proof.  We can back up and give a short, automated proof. *)
389 390 391 392 393

  Restart.

  induction e; crush;
    repeat (match goal with
394
              | [ |- context[match cfold ?E with NConst _ => _ | _ => _ end] ] =>
395 396 397 398
                dep_destruct (cfold E)
              | [ |- context[match pairOut (cfold ?E) with Some _ => _
                               | None => _ end] ] =>
                dep_destruct (cfold E)
399 400 401
              | [ |- (if ?E then _ else _) = _ ] => destruct E
            end; crush).
Qed.
Adam Chlipala's avatar
Adam Chlipala committed
402
(* end thide *)
403

404 405
(** With this example, we get a first taste of how to build automated proofs that adapt automatically to changes in function definitions. *)

406

Adam Chlipala's avatar
Adam Chlipala committed
407
(** * Dependently Typed Red-Black Trees *)
Adam Chlipala's avatar
Adam Chlipala committed
408

Adam Chlipala's avatar
Adam Chlipala committed
409
(** Red-black trees are a favorite purely functional data structure with an interesting invariant.  We can use dependent types to enforce that operations on red-black trees preserve the invariant.  For simplicity, we specialize our red-black trees to represent sets of [nat]s. *)
Adam Chlipala's avatar
Adam Chlipala committed
410

Adam Chlipala's avatar
Adam Chlipala committed
411 412 413 414
Inductive color : Set := Red | Black.

Inductive rbtree : color -> nat -> Set :=
| Leaf : rbtree Black 0
Adam Chlipala's avatar
Adam Chlipala committed
415
| RedNode : forall n, rbtree Black n -> nat -> rbtree Black n -> rbtree Red n
Adam Chlipala's avatar
Adam Chlipala committed
416 417
| BlackNode : forall c1 c2 n, rbtree c1 n -> nat -> rbtree c2 n -> rbtree Black (S n).

Adam Chlipala's avatar
Adam Chlipala committed
418 419 420 421
(** A value of type [rbtree c d] is a red-black tree node whose root has color [c] and that has black depth [d].  The latter property means that there are no more than [d] black-colored nodes on any path from the root to a leaf. *)

(** At first, it can be unclear that this choice of type indices tracks any useful property.  To convince ourselves, we will prove that every red-black tree is balanced.  We will phrase our theorem in terms of a depth calculating function that ignores the extra information in the types.  It will be useful to parameterize this function over a combining operation, so that we can re-use the same code to calculate the minimum or maximum height among all paths from root to leaf. *)

Adam Chlipala's avatar
Adam Chlipala committed
422 423 424
(* EX: Prove that every [rbtree] is balanced. *)

(* begin thide *)
Adam Chlipala's avatar
Adam Chlipala committed
425 426 427 428 429
Require Import Max Min.

Section depth.
  Variable f : nat -> nat -> nat.

Adam Chlipala's avatar
Adam Chlipala committed
430
  Fixpoint depth c n (t : rbtree c n) : nat :=
Adam Chlipala's avatar
Adam Chlipala committed
431 432 433 434 435 436 437
    match t with
      | Leaf => 0
      | RedNode _ t1 _ t2 => S (f (depth t1) (depth t2))
      | BlackNode _ _ _ t1 _ t2 => S (f (depth t1) (depth t2))
    end.
End depth.

Adam Chlipala's avatar
Adam Chlipala committed
438
(** Our proof of balanced-ness decomposes naturally into a lower bound and an upper bound.  We prove the lower bound first.  Unsurprisingly, a tree's black depth provides such a bound on the minimum path length.  We use the richly typed procedure [min_dec] to do case analysis on whether [min X Y] equals [X] or [Y]. *)
Adam Chlipala's avatar
Adam Chlipala committed
439

Adam Chlipala's avatar
Adam Chlipala committed
440 441 442 443
Check min_dec.
(** %\vspace{-.15in}% [[
min_dec
     : forall n m : nat, {min n m = n} + {min n m = m}
444 445
   ]]
   *)
Adam Chlipala's avatar
Adam Chlipala committed
446

Adam Chlipala's avatar
Adam Chlipala committed
447 448 449 450 451 452 453
Theorem depth_min : forall c n (t : rbtree c n), depth min t >= n.
  induction t; crush;
    match goal with
      | [ |- context[min ?X ?Y] ] => destruct (min_dec X Y)
    end; crush.
Qed.

Adam Chlipala's avatar
Adam Chlipala committed
454 455 456 457 458 459 460 461 462 463 464 465 466 467 468 469 470 471 472 473 474
(** There is an analogous upper-bound theorem based on black depth.  Unfortunately, a symmetric proof script does not suffice to establish it. *)

Theorem depth_max : forall c n (t : rbtree c n), depth max t <= 2 * n + 1.
  induction t; crush;
    match goal with
      | [ |- context[max ?X ?Y] ] => destruct (max_dec X Y)
    end; crush.

(** Two subgoals remain.  One of them is: [[
  n : nat
  t1 : rbtree Black n
  n0 : nat
  t2 : rbtree Black n
  IHt1 : depth max t1 <= n + (n + 0) + 1
  IHt2 : depth max t2 <= n + (n + 0) + 1
  e : max (depth max t1) (depth max t2) = depth max t1
  ============================
   S (depth max t1) <= n + (n + 0) + 1
 
   ]]

475
   We see that [IHt1] is _almost_ the fact we need, but it is not quite strong enough.  We will need to strengthen our induction hypothesis to get the proof to go through. *)
Adam Chlipala's avatar
Adam Chlipala committed
476 477 478 479 480

Abort.

(** In particular, we prove a lemma that provides a stronger upper bound for trees with black root nodes.  We got stuck above in a case about a red root node.  Since red nodes have only black children, our IH strengthening will enable us to finish the proof. *)

Adam Chlipala's avatar
Adam Chlipala committed
481 482 483 484 485 486 487
Lemma depth_max' : forall c n (t : rbtree c n), match c with
                                                  | Red => depth max t <= 2 * n + 1
                                                  | Black => depth max t <= 2 * n
                                                end.
  induction t; crush;
    match goal with
      | [ |- context[max ?X ?Y] ] => destruct (max_dec X Y)
Adam Chlipala's avatar
Adam Chlipala committed
488 489
    end; crush;
    repeat (match goal with
Adam Chlipala's avatar
Adam Chlipala committed
490 491
              | [ H : context[match ?C with Red => _ | Black => _ end] |- _ ] =>
                destruct C
Adam Chlipala's avatar
Adam Chlipala committed
492
            end; crush).
Adam Chlipala's avatar
Adam Chlipala committed
493 494
Qed.

Adam Chlipala's avatar
Adam Chlipala committed
495
(** The original theorem follows easily from the lemma.  We use the tactic %\index{tactics!generalize}%[generalize pf], which, when [pf] proves the proposition [P], changes the goal from [Q] to [P -> Q].  This transformation is useful because it makes the truth of [P] manifest syntactically, so that automation machinery can rely on [P], even if that machinery is not smart enough to establish [P] on its own. *)
Adam Chlipala's avatar
Adam Chlipala committed
496

Adam Chlipala's avatar
Adam Chlipala committed
497 498 499 500
Theorem depth_max : forall c n (t : rbtree c n), depth max t <= 2 * n + 1.
  intros; generalize (depth_max' t); destruct c; crush.
Qed.

Adam Chlipala's avatar
Adam Chlipala committed
501 502
(** The final balance theorem establishes that the minimum and maximum path lengths of any tree are within a factor of two of each other. *)

Adam Chlipala's avatar
Adam Chlipala committed
503 504 505
Theorem balanced : forall c n (t : rbtree c n), 2 * depth min t + 1 >= depth max t.
  intros; generalize (depth_min t); generalize (depth_max t); crush.
Qed.
Adam Chlipala's avatar
Adam Chlipala committed
506
(* end thide *)
Adam Chlipala's avatar
Adam Chlipala committed
507

Adam Chlipala's avatar
Adam Chlipala committed
508
(** Now we are ready to implement an example operation on our trees, insertion.  Insertion can be thought of as breaking the tree invariants locally but then rebalancing.  In particular, in intermediate states we find red nodes that may have red children.  The type [rtree] captures the idea of such a node, continuing to track black depth as a type index. *)
Adam Chlipala's avatar
Adam Chlipala committed
509

Adam Chlipala's avatar
Adam Chlipala committed
510 511 512
Inductive rtree : nat -> Set :=
| RedNode' : forall c1 c2 n, rbtree c1 n -> nat -> rbtree c2 n -> rtree n.

Adam Chlipala's avatar
Adam Chlipala committed
513
(** Before starting to define [insert], we define predicates capturing when a data value is in the set represented by a normal or possibly invalid tree. *)
Adam Chlipala's avatar
Adam Chlipala committed
514

515 516 517
Section present.
  Variable x : nat.

Adam Chlipala's avatar
Adam Chlipala committed
518
  Fixpoint present c n (t : rbtree c n) : Prop :=
519 520 521 522 523 524 525 526 527 528 529 530
    match t with
      | Leaf => False
      | RedNode _ a y b => present a \/ x = y \/ present b
      | BlackNode _ _ _ a y b => present a \/ x = y \/ present b
    end.

  Definition rpresent n (t : rtree n) : Prop :=
    match t with
      | RedNode' _ _ _ a y b => present a \/ x = y \/ present b
    end.
End present.

Adam Chlipala's avatar
Adam Chlipala committed
531
(** Insertion relies on two balancing operations.  It will be useful to give types to these operations using a relative of the subset types from last chapter.  While subset types let us pair a value with a proof about that value, here we want to pair a value with another non-proof dependently typed value.  The %\index{Gallina terms!sigT}%[sigT] type fills this role. *)
Adam Chlipala's avatar
Adam Chlipala committed
532

Adam Chlipala's avatar
Adam Chlipala committed
533
Locate "{ _ : _ & _ }".
Adam Chlipala's avatar
Adam Chlipala committed
534 535 536
(** [[
Notation            Scope     
"{ x : A  & P }" := sigT (fun x : A => P)
537 538
]]
*)
Adam Chlipala's avatar
Adam Chlipala committed
539

Adam Chlipala's avatar
Adam Chlipala committed
540
Print sigT.
Adam Chlipala's avatar
Adam Chlipala committed
541 542 543
(** [[
Inductive sigT (A : Type) (P : A -> Type) : Type :=
    existT : forall x : A, P x -> sigT P
544 545
]]
*)
Adam Chlipala's avatar
Adam Chlipala committed
546 547

(** It will be helpful to define a concise notation for the constructor of [sigT]. *)
Adam Chlipala's avatar
Adam Chlipala committed
548

Adam Chlipala's avatar
Adam Chlipala committed
549 550
Notation "{< x >}" := (existT _ _ x).

Adam Chlipala's avatar
Adam Chlipala committed
551 552
(** Each balance function is used to construct a new tree whose keys include the keys of two input trees, as well as a new key.  One of the two input trees may violate the red-black alternation invariant (that is, it has an [rtree] type), while the other tree is known to be valid.  Crucially, the two input trees have the same black depth.

Adam Chlipala's avatar
Adam Chlipala committed
553 554 555
   A balance operation may return a tree whose root is of either color.  Thus, we use a [sigT] type to package the result tree with the color of its root.  Here is the definition of the first balance operation, which applies when the possibly invalid [rtree] belongs to the left of the valid [rbtree].

   A quick word of encouragement: After writing this code, even I do not understand the precise details of how balancing works!  I consulted Chris Okasaki's paper %``%#"#Red-Black Trees in a Functional Setting#"#%''~\cite{Okasaki}% and transcribed the code to use dependent types.  Luckily, the details are not so important here; types alone will tell us that insertion preserves balanced-ness, and we will prove that insertion produces trees containing the right keys.*)
Adam Chlipala's avatar
Adam Chlipala committed
556

Adam Chlipala's avatar
Adam Chlipala committed
557
Definition balance1 n (a : rtree n) (data : nat) c2 :=
Adam Chlipala's avatar
Adam Chlipala committed
558 559
  match a in rtree n return rbtree c2 n
    -> { c : color & rbtree c (S n) } with
560 561
    | RedNode' _ c0 _ t1 y t2 =>
      match t1 in rbtree c n return rbtree c0 n -> rbtree c2 n
Adam Chlipala's avatar
Adam Chlipala committed
562 563 564
        -> { c : color & rbtree c (S n) } with
        | RedNode _ a x b => fun c d =>
          {<RedNode (BlackNode a x b) y (BlackNode c data d)>}
Adam Chlipala's avatar
Adam Chlipala committed
565
        | t1' => fun t2 =>
566
          match t2 in rbtree c n return rbtree Black n -> rbtree c2 n
Adam Chlipala's avatar
Adam Chlipala committed
567 568 569
            -> { c : color & rbtree c (S n) } with
            | RedNode _ b x c => fun a d =>
              {<RedNode (BlackNode a y b) x (BlackNode c data d)>}
Adam Chlipala's avatar
Adam Chlipala committed
570
            | b => fun a t => {<BlackNode (RedNode a y b) data t>}
Adam Chlipala's avatar
Adam Chlipala committed
571 572 573 574
          end t1'
      end t2
  end.

575
(** We apply a trick that I call the%\index{convoy pattern}% _convoy pattern_.  Recall that [match] annotations only make it possible to describe a dependence of a [match] _result type_ on the discriminee.  There is no automatic refinement of the types of free variables.  However, it is possible to effect such a refinement by finding a way to encode free variable type dependencies in the [match] result type, so that a [return] clause can express the connection.
Adam Chlipala's avatar
Adam Chlipala committed
576

577
   In particular, we can extend the [match] to return _functions over the free variables whose types we want to refine_.  In the case of [balance1], we only find ourselves wanting to refine the type of one tree variable at a time.  We match on one subtree of a node, and we want the type of the other subtree to be refined based on what we learn.  We indicate this with a [return] clause starting like [rbtree _ n -> ...], where [n] is bound in an [in] pattern.  Such a [match] expression is applied immediately to the %``%#"#old version#"#%''% of the variable to be refined, and the type checker is happy.
Adam Chlipala's avatar
Adam Chlipala committed
578

Adam Chlipala's avatar
Adam Chlipala committed
579
   Here is the symmetric function [balance2], for cases where the possibly invalid tree appears on the right rather than on the left. *)
Adam Chlipala's avatar
Adam Chlipala committed
580

Adam Chlipala's avatar
Adam Chlipala committed
581 582
Definition balance2 n (a : rtree n) (data : nat) c2 :=
  match a in rtree n return rbtree c2 n -> { c : color & rbtree c (S n) } with
583 584
    | RedNode' _ c0 _ t1 z t2 =>
      match t1 in rbtree c n return rbtree c0 n -> rbtree c2 n
Adam Chlipala's avatar
Adam Chlipala committed
585 586 587
        -> { c : color & rbtree c (S n) } with
        | RedNode _ b y c => fun d a =>
          {<RedNode (BlackNode a data b) y (BlackNode c z d)>}
Adam Chlipala's avatar
Adam Chlipala committed
588
        | t1' => fun t2 =>
589
          match t2 in rbtree c n return rbtree Black n -> rbtree c2 n
Adam Chlipala's avatar
Adam Chlipala committed
590 591 592
            -> { c : color & rbtree c (S n) } with
            | RedNode _ c z' d => fun b a =>
              {<RedNode (BlackNode a data b) z (BlackNode c z' d)>}
Adam Chlipala's avatar
Adam Chlipala committed
593
            | b => fun a t => {<BlackNode t data (RedNode a z b)>}
Adam Chlipala's avatar
Adam Chlipala committed
594 595 596 597
          end t1'
      end t2
  end.

Adam Chlipala's avatar
Adam Chlipala committed
598 599
(** Now we are almost ready to get down to the business of writing an [insert] function.  First, we enter a section that declares a variable [x], for the key we want to insert. *)

Adam Chlipala's avatar
Adam Chlipala committed
600 601 602
Section insert.
  Variable x : nat.

Adam Chlipala's avatar
Adam Chlipala committed
603 604
  (** Most of the work of insertion is done by a helper function [ins], whose return types are expressed using a type-level function [insResult]. *)

Adam Chlipala's avatar
Adam Chlipala committed
605 606 607 608 609 610
  Definition insResult c n :=
    match c with
      | Red => rtree n
      | Black => { c' : color & rbtree c' n }
    end.

Adam Chlipala's avatar
Adam Chlipala committed
611
  (** That is, inserting into a tree with root color [c] and black depth [n], the variety of tree we get out depends on [c].  If we started with a red root, then we get back a possibly invalid tree of depth [n].  If we started with a black root, we get back a valid tree of depth [n] with a root node of an arbitrary color.
Adam Chlipala's avatar
Adam Chlipala committed
612 613 614 615 616

     Here is the definition of [ins].  Again, we do not want to dwell on the functional details. *)

  Fixpoint ins c n (t : rbtree c n) : insResult c n :=
    match t with
Adam Chlipala's avatar
Adam Chlipala committed
617 618 619 620 621 622 623 624 625 626 627 628 629 630 631 632 633 634 635
      | Leaf => {< RedNode Leaf x Leaf >}
      | RedNode _ a y b =>
        if le_lt_dec x y
          then RedNode' (projT2 (ins a)) y b
          else RedNode' a y (projT2 (ins b))
      | BlackNode c1 c2 _ a y b =>
        if le_lt_dec x y
          then
            match c1 return insResult c1 _ -> _ with
              | Red => fun ins_a => balance1 ins_a y b
              | _ => fun ins_a => {< BlackNode (projT2 ins_a) y b >}
            end (ins a)
          else
            match c2 return insResult c2 _ -> _ with
              | Red => fun ins_b => balance2 ins_b y a
              | _ => fun ins_b => {< BlackNode a y (projT2 ins_b) >}
            end (ins b)
    end.

636
  (** The one new trick is a variation of the convoy pattern.  In each of the last two pattern matches, we want to take advantage of the typing connection between the trees [a] and [b].  We might naively apply the convoy pattern directly on [a] in the first [match] and on [b] in the second.  This satisfies the type checker per se, but it does not satisfy the termination checker.  Inside each [match], we would be calling [ins] recursively on a locally bound variable.  The termination checker is not smart enough to trace the dataflow into that variable, so the checker does not know that this recursive argument is smaller than the original argument.  We make this fact clearer by applying the convoy pattern on _the result of a recursive call_, rather than just on that call's argument.
Adam Chlipala's avatar
Adam Chlipala committed
637 638 639

     Finally, we are in the home stretch of our effort to define [insert].  We just need a few more definitions of non-recursive functions.  First, we need to give the final characterization of [insert]'s return type.  Inserting into a red-rooted tree gives a black-rooted tree where black depth has increased, and inserting into a black-rooted tree gives a tree where black depth has stayed the same and where the root is an arbitrary color. *)

Adam Chlipala's avatar
Adam Chlipala committed
640 641 642 643 644 645
  Definition insertResult c n :=
    match c with
      | Red => rbtree Black (S n)
      | Black => { c' : color & rbtree c' n }
    end.

Adam Chlipala's avatar
Adam Chlipala committed
646 647
  (** A simple clean-up procedure translates [insResult]s into [insertResult]s. *)

Adam Chlipala's avatar
Adam Chlipala committed
648
  Definition makeRbtree c n : insResult c n -> insertResult c n :=
Adam Chlipala's avatar
Adam Chlipala committed
649
    match c with
Adam Chlipala's avatar
Adam Chlipala committed
650
      | Red => fun r =>
Adam Chlipala's avatar
Adam Chlipala committed
651
        match r with
Adam Chlipala's avatar
Adam Chlipala committed
652 653 654 655 656
          | RedNode' _ _ _ a x b => BlackNode a x b
        end
      | Black => fun r => r
    end.

Adam Chlipala's avatar
Adam Chlipala committed
657 658
  (** We modify Coq's default choice of implicit arguments for [makeRbtree], so that we do not need to specify the [c] and [n] arguments explicitly in later calls. *)

Adam Chlipala's avatar
Adam Chlipala committed
659
  Implicit Arguments makeRbtree [c n].
Adam Chlipala's avatar
Adam Chlipala committed
660

Adam Chlipala's avatar
Adam Chlipala committed
661 662
  (** Finally, we define [insert] as a simple composition of [ins] and [makeRbtree]. *)

Adam Chlipala's avatar
Adam Chlipala committed
663
  Definition insert c n (t : rbtree c n) : insertResult c n :=
Adam Chlipala's avatar
Adam Chlipala committed
664
    makeRbtree (ins t).
Adam Chlipala's avatar
Adam Chlipala committed
665

Adam Chlipala's avatar
Adam Chlipala committed
666 667
  (** As we noted earlier, the type of [insert] guarantees that it outputs balanced trees whose depths have not increased too much.  We also want to know that [insert] operates correctly on trees interpreted as finite sets, so we finish this section with a proof of that fact. *)

Adam Chlipala's avatar
Adam Chlipala committed
668 669 670
  Section present.
    Variable z : nat.

Adam Chlipala's avatar
Adam Chlipala committed
671 672
    (** The variable [z] stands for an arbitrary key.  We will reason about [z]'s presence in particular trees.  As usual, outside the section the theorems we prove will quantify over all possible keys, giving us the facts we wanted.

673
       We start by proving the correctness of the balance operations.  It is useful to define a custom tactic [present_balance] that encapsulates the reasoning common to the two proofs.  We use the keyword %\index{Vernacular commands!Ltac}%[Ltac] to assign a name to a proof script.  This particular script just iterates between [crush] and identification of a tree that is being pattern-matched on and should be destructed. *)
Adam Chlipala's avatar
Adam Chlipala committed
674

675 676 677
    Ltac present_balance :=
      crush;
      repeat (match goal with
678 679
                | [ _ : context[match ?T with Leaf => _ | _ => _ end] |- _ ] => dep_destruct T
                | [ |- context[match ?T with Leaf => _ | _ => _ end] ] => dep_destruct T
680 681
              end; crush).

Adam Chlipala's avatar
Adam Chlipala committed
682 683
    (** The balance correctness theorems are simple first-order logic equivalences, where we use the function [projT2] to project the payload of a [sigT] value. *)

684
    Lemma present_balance1 : forall n (a : rtree n) (y : nat) c2 (b : rbtree c2 n),
685 686 687
      present z (projT2 (balance1 a y b))
      <-> rpresent z a \/ z = y \/ present z b.
      destruct a; present_balance.
Adam Chlipala's avatar
Adam Chlipala committed
688 689
    Qed.

690
    Lemma present_balance2 : forall n (a : rtree n) (y : nat) c2 (b : rbtree c2 n),
Adam Chlipala's avatar
Adam Chlipala committed
691 692
      present z (projT2 (balance2 a y b))
      <-> rpresent z a \/ z = y \/ present z b.
693
      destruct a; present_balance.
Adam Chlipala's avatar
Adam Chlipala committed
694 695
    Qed.

Adam Chlipala's avatar
Adam Chlipala committed
696 697
    (** To state the theorem for [ins], it is useful to define a new type-level function, since [ins] returns different result types based on the type indices passed to it.  Recall that [x] is the section variable standing for the key we are inserting. *)

Adam Chlipala's avatar
Adam Chlipala committed
698 699 700 701 702 703
    Definition present_insResult c n :=
      match c return (rbtree c n -> insResult c n -> Prop) with
        | Red => fun t r => rpresent z r <-> z = x \/ present z t
        | Black => fun t r => present z (projT2 r) <-> z = x \/ present z t
      end.

Adam Chlipala's avatar
Adam Chlipala committed
704 705
    (** Now the statement and proof of the [ins] correctness theorem are straightforward, if verbose.  We proceed by induction on the structure of a tree, followed by finding case analysis opportunities on expressions we see being analyzed in [if] or [match] expressions.  After that, we pattern-match to find opportunities to use the theorems we proved about balancing.  Finally, we identify two variables that are asserted by some hypothesis to be equal, and we use that hypothesis to replace one variable with the other everywhere. *)

Adam Chlipala's avatar
Adam Chlipala committed
706 707 708 709
    Theorem present_ins : forall c n (t : rbtree c n),
      present_insResult t (ins t).
      induction t; crush;
        repeat (match goal with
Adam Chlipala's avatar
Adam Chlipala committed
710
                  | [ _ : context[if ?E then _ else _] |- _ ] => destruct E
Adam Chlipala's avatar
Adam Chlipala committed
711
                  | [ |- context[if ?E then _ else _] ] => destruct E
Adam Chlipala's avatar
Adam Chlipala committed
712
                  | [ _ : context[match ?C with Red => _ | Black => _ end]
Adam Chlipala's avatar
Adam Chlipala committed
713
                      |- _ ] => destruct C
Adam Chlipala's avatar
Adam Chlipala committed
714 715
                end; crush);
        try match goal with
Adam Chlipala's avatar
Adam Chlipala committed
716
              | [ _ : context[balance1 ?A ?B ?C] |- _ ] =>
Adam Chlipala's avatar
Adam Chlipala committed
717 718 719
                generalize (present_balance1 A B C)
            end;
        try match goal with
Adam Chlipala's avatar
Adam Chlipala committed
720
              | [ _ : context[balance2 ?A ?B ?C] |- _ ] =>
Adam Chlipala's avatar
Adam Chlipala committed
721 722 723 724 725 726 727 728 729 730
                generalize (present_balance2 A B C)
            end;
        try match goal with
              | [ |- context[balance1 ?A ?B ?C] ] =>
                generalize (present_balance1 A B C)
            end;
        try match goal with
              | [ |- context[balance2 ?A ?B ?C] ] =>
                generalize (present_balance2 A B C)
            end;
Adam Chlipala's avatar
Adam Chlipala committed
731
        crush;
Adam Chlipala's avatar
Adam Chlipala committed
732 733 734 735 736 737 738 739 740
          match goal with
            | [ z : nat, x : nat |- _ ] =>
              match goal with
                | [ H : z = x |- _ ] => rewrite H in *; clear H
              end
          end;
          tauto.
    Qed.

Adam Chlipala's avatar
Adam Chlipala committed
741 742
    (** The hard work is done.  The most readable way to state correctness of [insert] involves splitting the property into two color-specific theorems.  We write a tactic to encapsulate the reasoning steps that work to establish both facts. *)

743 744
    Ltac present_insert :=
      unfold insert; intros n t; inversion t;
Adam Chlipala's avatar
Adam Chlipala committed
745 746
        generalize (present_ins t); simpl;
          dep_destruct (ins t); tauto.
Adam Chlipala's avatar
Adam Chlipala committed
747 748 749 750

    Theorem present_insert_Red : forall n (t : rbtree Red n),
      present z (insert t)
      <-> (z = x \/ present z t).
751
      present_insert.
Adam Chlipala's avatar
Adam Chlipala committed
752 753 754 755 756
    Qed.

    Theorem present_insert_Black : forall n (t : rbtree Black n),
      present z (projT2 (insert t))
      <-> (z = x \/ present z t).
757
      present_insert.
Adam Chlipala's avatar
Adam Chlipala committed
758 759
    Qed.
  End present.
Adam Chlipala's avatar
Adam Chlipala committed
760 761
End insert.

762
(** We can generate executable OCaml code with the command %\index{Vernacular commands!Recursive Extraction}%[Recursive Extraction insert], which also automatically outputs the OCaml versions of all of [insert]'s dependencies.  In our previous extractions, we wound up with clean OCaml code.  Here, we find uses of %\index{Obj.magic}\texttt{%#<tt>#Obj.magic#</tt>#%}%, OCaml's unsafe cast operator for tweaking the apparent type of an expression in an arbitrary way.  Casts appear for this example because the return type of [insert] depends on the _value_ of the function's argument, a pattern which OCaml cannot handle.  Since Coq's type system is much more expressive than OCaml's, such casts are unavoidable in general.  Since the OCaml type-checker is no longer checking full safety of programs, we must rely on Coq's extractor to use casts only in provably safe ways. *)
Adam Chlipala's avatar
Adam Chlipala committed
763 764 765 766

(* begin hide *)
Recursive Extraction insert.
(* end hide *)
Adam Chlipala's avatar
Adam Chlipala committed
767

Adam Chlipala's avatar
Adam Chlipala committed
768

769 770
(** * A Certified Regular Expression Matcher *)

Adam Chlipala's avatar
Adam Chlipala committed
771 772
(** Another interesting example is regular expressions with dependent types that express which predicates over strings particular regexps implement.  We can then assign a dependent type to a regular expression matching function, guaranteeing that it always decides the string property that we expect it to decide.

Adam Chlipala's avatar
Adam Chlipala committed
773
   Before defining the syntax of expressions, it is helpful to define an inductive type capturing the meaning of the Kleene star.  That is, a string [s] matches regular expression [star e] if and only if [s] can be decomposed into a sequence of substrings that all match [e].  We use Coq's string support, which comes through a combination of the [Strings] library and some parsing notations built into Coq.  Operators like [++] and functions like [length] that we know from lists are defined again for strings.  Notation scopes help us control which versions we want to use in particular contexts.%\index{Vernacular commands!Open Scope}% *)
Adam Chlipala's avatar
Adam Chlipala committed
774

775 776 777
Require Import Ascii String.
Open Scope string_scope.

778 779 780 781 782 783 784 785 786 787 788
Section star.
  Variable P : string -> Prop.

  Inductive star : string -> Prop :=
  | Empty : star ""
  | Iter : forall s1 s2,
    P s1
    -> star s2
    -> star (s1 ++ s2).
End star.

Adam Chlipala's avatar
Adam Chlipala committed
789
(** Now we can make our first attempt at defining a [regexp] type that is indexed by predicates on strings.  Here is a reasonable-looking definition that is restricted to constant characters and concatenation.  We use the constructor [String], which is the analogue of list cons for the type [string], where [""] is like list nil.
Adam Chlipala's avatar
Adam Chlipala committed
790 791 792 793 794 795
[[
Inductive regexp : (string -> Prop) -> Set :=
| Char : forall ch : ascii,
  regexp (fun s => s = String ch "")
| Concat : forall (P1 P2 : string -> Prop) (r1 : regexp P1) (r2 : regexp P2),
  regexp (fun s => exists s1, exists s2, s = s1 ++ s2 /\ P1 s1 /\ P2 s2).
Adam Chlipala's avatar
Adam Chlipala committed
796
]]
Adam Chlipala's avatar
Adam Chlipala committed
797

Adam Chlipala's avatar
Adam Chlipala committed
798
<<
Adam Chlipala's avatar
Adam Chlipala committed
799
User error: Large non-propositional inductive types must be in Type
Adam Chlipala's avatar
Adam Chlipala committed
800
>>
Adam Chlipala's avatar
Adam Chlipala committed
801

Adam Chlipala's avatar
Adam Chlipala committed
802
What is a %\index{large inductive types}%large inductive type?  In Coq, it is an inductive type that has a constructor which quantifies over some type of type [Type].  We have not worked with [Type] very much to this point.  Every term of CIC has a type, including [Set] and [Prop], which are assigned type [Type].  The type [string -> Prop] from the failed definition also has type [Type].
Adam Chlipala's avatar
Adam Chlipala committed
803 804 805

It turns out that allowing large inductive types in [Set] leads to contradictions when combined with certain kinds of classical logic reasoning.  Thus, by default, such types are ruled out.  There is a simple fix for our [regexp] definition, which is to place our new type in [Type].  While fixing the problem, we also expand the list of constructors to cover the remaining regular expression operators. *)

806
Inductive regexp : (string -> Prop) -> Type :=
807 808 809
| Char : forall ch : ascii,
  regexp (fun s => s = String ch "")
| Concat : forall P1 P2 (r1 : regexp P1) (r2 : regexp P2),
810 811
  regexp (fun s => exists s1, exists s2, s = s1 ++ s2 /\ P1 s1 /\ P2 s2)
| Or : forall P1 P2 (r1 : regexp P1) (r2 : regexp P2),
812 813 814
  regexp (fun s => P1 s \/ P2 s)
| Star : forall P (r : regexp P),
  regexp (star P).
815

816
(** Many theorems about strings are useful for implementing a certified regexp matcher, and few of them are in the [Strings] library.  The book source includes statements, proofs, and hint commands for a handful of such omitted theorems.  Since they are orthogonal to our use of dependent types, we hide them in the rendered versions of this book. *)
Adam Chlipala's avatar
Adam Chlipala committed
817 818

(* begin hide *)
819 820 821 822 823 824 825 826 827 828 829 830 831 832 833 834 835 836 837 838 839 840 841 842 843 844 845
Open Scope specif_scope.

Lemma length_emp : length "" <= 0.
  crush.
Qed.

Lemma append_emp : forall s, s = "" ++ s.
  crush.
Qed.

Ltac substring :=
  crush;
  repeat match goal with
           | [ |- context[match ?N with O => _ | S _ => _ end] ] => destruct N; crush
         end.

Lemma substring_le : forall s n m,
  length (substring n m s) <= m.
  induction s; substring.
Qed.

Lemma substring_all : forall s,
  substring 0 (length s) s = s.
  induction s; substring.
Qed.

Lemma substring_none : forall s n,
Adam Chlipala's avatar
Adam Chlipala committed
846
  substring n 0 s = "".
847 848 849
  induction s; substring.
Qed.

850
Hint Rewrite substring_all substring_none.
851 852 853 854 855 856 857 858 859 860 861 862 863 864 865 866 867 868 869 870 871 872

Lemma substring_split : forall s m,
  substring 0 m s ++ substring m (length s - m) s = s.
  induction s; substring.
Qed.

Lemma length_app1 : forall s1 s2,
  length s1 <= length (s1 ++ s2).
  induction s1; crush.
Qed.

Hint Resolve length_emp append_emp substring_le substring_split length_app1.

Lemma substring_app_fst : forall s2 s1 n,
  length s1 = n
  -> substring 0 n (s1 ++ s2) = s1.
  induction s1; crush.
Qed.

Lemma substring_app_snd : forall s2 s1 n,
  length s1 = n
  -> substring n (length (s1 ++ s2) - n) (s1 ++ s2) = s2.
873
  Hint Rewrite <- minus_n_O.
874 875 876 877

  induction s1; crush.
Qed.

878
Hint Rewrite substring_app_fst substring_app_snd using solve [trivial].
Adam Chlipala's avatar
Adam Chlipala committed
879 880 881
(* end hide *)

(** A few auxiliary functions help us in our final matcher definition.  The function [split] will be used to implement the regexp concatenation case. *)
882 883 884

Section split.
  Variables P1 P2 : string -> Prop.
Adam Chlipala's avatar
Adam Chlipala committed
885 886
  Variable P1_dec : forall s, {P1 s} + {~ P1 s}.
  Variable P2_dec : forall s, {P2 s} + {~ P2 s}.
Adam Chlipala's avatar
Adam Chlipala committed
887
  (** We require a choice of two arbitrary string predicates and functions for deciding them. *)
888 889

  Variable s : string.
Adam Chlipala's avatar
Adam Chlipala committed
890 891
  (** Our computation will take place relative to a single fixed string, so it is easiest to make it a [Variable], rather than an explicit argument to our functions. *)

Adam Chlipala's avatar
Adam Chlipala committed
892
  (** The function [split'] is the workhorse behind [split].  It searches through the possible ways of splitting [s] into two pieces, checking the two predicates against each such pair.  The execution of [split'] progresses right-to-left, from splitting all of [s] into the first piece to splitting all of [s] into the second piece.  It takes an extra argument, [n], which specifies how far along we are in this search process. *)
893

894
  Definition split' : forall n : nat, n <= length s
895
    -> {exists s1, exists s2, length s1 <= n /\ s1 ++ s2 = s /\ P1 s1 /\ P2 s2}
Adam Chlipala's avatar
Adam Chlipala committed
896
    + {forall s1 s2, length s1 <= n -> s1 ++ s2 = s -> ~ P1 s1 \/ ~ P2 s2}.
897 898
    refine (fix F (n : nat) : n <= length s
      -> {exists s1, exists s2, length s1 <= n /\ s1 ++ s2 = s /\ P1 s1 /\ P2 s2}
Adam Chlipala's avatar
Adam Chlipala committed
899 900
      + {forall s1 s2, length s1 <= n -> s1 ++ s2 = s -> ~ P1 s1 \/ ~ P2 s2} :=
      match n with
901
        | O => fun _ => Reduce (P1_dec "" && P2_dec s)
Adam Chlipala's avatar
Adam Chlipala committed
902 903
        | S n' => fun _ => (P1_dec (substring 0 (S n') s)
            && P2_dec (substring (S n') (length s - S n') s))
904 905 906 907
          || F n' _
      end); clear F; crush; eauto 7;
    match goal with
      | [ _ : length ?S <= 0 |- _ ] => destruct S
Adam Chlipala's avatar
Adam Chlipala committed
908
      | [ _ : length ?S' <= S ?N |- _ ] => destruct (eq_nat_dec (length S') (S N))
909 910 911
    end; crush.
  Defined.

Adam Chlipala's avatar
Adam Chlipala committed
912
  (** There is one subtle point in the [split'] code that is worth mentioning.  The main body of the function is a [match] on [n].  In the case where [n] is known to be [S n'], we write [S n'] in several places where we might be tempted to write [n].  However, without further work to craft proper [match] annotations, the type-checker does not use the equality between [n] and [S n'].  Thus, it is common to see patterns repeated in [match] case bodies in dependently typed Coq code.  We can at least use a [let] expression to avoid copying the pattern more than once, replacing the first case body with:
Adam Chlipala's avatar
Adam Chlipala committed
913 914 915 916 917
     [[
        | S n' => fun _ => let n := S n' in
          (P1_dec (substring 0 n s)
            && P2_dec (substring n (length s - n) s))
          || F n' _
Adam Chlipala's avatar
Adam Chlipala committed
918
 
Adam Chlipala's avatar
Adam Chlipala committed
919 920
     ]]

Adam Chlipala's avatar
Adam Chlipala committed
921
     The [split] function itself is trivial to implement in terms of [split'].  We just ask [split'] to begin its search with [n = length s]. *)
Adam Chlipala's avatar
Adam Chlipala committed
922

923
  Definition split : {exists s1, exists s2, s = s1 ++ s2 /\ P1 s1 /\ P2 s2}
Adam Chlipala's avatar
Adam Chlipala committed
924
    + {forall s1 s2, s = s1 ++ s2 -> ~ P1 s1 \/ ~ P2 s2}.
925 926 927 928 929 930
    refine (Reduce (split' (n := length s) _)); crush; eauto.
  Defined.
End split.

Implicit Arguments split [P1 P2].

Adam Chlipala's avatar
Adam Chlipala committed
931
(* begin hide *)
932 933 934 935
Lemma app_empty_end : forall s, s ++ "" = s.
  induction s; crush.
Qed.

936
Hint Rewrite app_empty_end.
937 938 939 940 941 942 943 944 945 946 947 948 949

Lemma substring_self : forall s n,
  n <= 0
  -> substring n (length s - n) s = s.
  induction s; substring.
Qed.

Lemma substring_empty : forall s n m,
  m <= 0
  -> substring n m s = "".
  induction s; substring.
Qed.

950
Hint Rewrite substring_self substring_empty using omega.
951 952 953 954

Lemma substring_split' : forall s n m,
  substring n m s ++ substring (n + m) (length s - (n + m)) s
  = substring n (length s - n) s.
955
  Hint Rewrite substring_split.
956 957 958 959 960 961 962 963 964 965 966 967 968 969 970 971 972 973 974 975 976 977 978 979 980 981 982 983 984 985 986 987 988 989 990 991 992 993 994 995 996 997 998 999 1000 1001 1002

  induction s; substring.
Qed.

Lemma substring_stack : forall s n2 m1 m2,
  m1 <= m2
  -> substring 0 m1 (substring n2 m2 s)
  = substring n2 m1 s.
  induction s; substring.
Qed.

Ltac substring' :=
  crush;
  repeat match goal with
           | [ |- context[match ?N with O => _ | S _ => _ end] ] => case_eq N; crush
         end.

Lemma substring_stack' : forall s n1 n2 m1 m2,
  n1 + m1 <= m2
  -> substring n1 m1 (substring n2 m2 s)
  = substring (n1 + n2) m1 s.
  induction s; substring';
    match goal with
      | [ |- substring ?N1 _ _ = substring ?N2 _ _ ] =>
        replace N1 with N2; crush
    end.
Qed.

Lemma substring_suffix : forall s n,
  n <= length s
  -> length (substring n (length s - n) s) = length s - n.
  induction s; substring.
Qed.

Lemma substring_suffix_emp' : forall s n m,
  substring n (S m) s = ""
  -> n >= length s.
  induction s; crush;
    match goal with
      | [ |- ?N >= _ ] => destruct N; crush
    end;
    match goal with
      [ |- S ?N >= S ?E ] => assert (N >= E); [ eauto | omega ]
    end.
Qed.

Lemma substring_suffix_emp : forall s n m,
Adam Chlipala's avatar
Adam Chlipala committed
1003 1004
  substring n m s = ""
  -> m > 0
1005
  -> n >= length s.
Adam Chlipala's avatar
Adam Chlipala committed
1006
  destruct m as [ | m]; [crush | intros; apply substring_suffix_emp' with m; assumption].
1007 1008 1009
Qed.

Hint Rewrite substring_stack substring_stack' substring_suffix
1010
  using omega.
1011 1012 1013 1014 1015 1016 1017 1018 1019 1020 1021

Lemma minus_minus : forall n m1 m2,
  m1 + m2 <= n
  -> n - m1 - m2 = n - (m1 + m2).
  intros; omega.
Qed.

Lemma plus_n_Sm' : forall n m : nat, S (n + m) = m + S n.
  intros; omega.
Qed.

1022
Hint Rewrite minus_minus using omega.
Adam Chlipala's avatar
Adam Chlipala committed
1023 1024 1025
(* end hide *)

(** One more helper function will come in handy: [dec_star], for implementing another linear search through ways of splitting a string, this time for implementing the Kleene star. *)
1026 1027 1028

Section dec_star.
  Variable P : string -> Prop.
Adam Chlipala's avatar
Adam Chlipala committed
1029
  Variable P_dec : forall s, {P s} + {~ P s}.
1030

Adam Chlipala's avatar
Adam Chlipala committed
1031
  (** Some new lemmas and hints about the [star] type family are useful.  We omit them here; they are included in the book source at this point. *)
Adam Chlipala's avatar
Adam Chlipala committed
1032 1033

  (* begin hide *)
1034 1035 1036 1037 1038 1039 1040 1041 1042 1043 1044 1045 1046 1047 1048 1049 1050 1051 1052 1053 1054 1055 1056 1057 1058 1059 1060 1061 1062 1063 1064 1065 1066 1067 1068 1069 1070 1071 1072 1073 1074 1075 1076 1077 1078 1079 1080 1081 1082 1083 1084 1085 1086 1087
  Hint Constructors star.

  Lemma star_empty : forall s,
    length s = 0
    -> star P s.
    destruct s; crush.
  Qed.

  Lemma star_singleton : forall s, P s -> star P s.
    intros; rewrite <- (app_empty_end s); auto.
  Qed.

  Lemma star_app : forall s n m,
    P (substring n m s)
    -> star P (substring (n + m) (length s - (n + m)) s)
    -> star P (substring n (length s - n) s).
    induction n; substring;
      match goal with
        | [ H : P (substring ?N ?M ?S) |- _ ] =>
          solve [ rewrite <- (substring_split S M); auto
            | rewrite <- (substring_split' S N M); auto ]
      end.
  Qed.

  Hint Resolve star_empty star_singleton star_app.

  Variable s : string.

  Lemma star_inv : forall s,
    star P s
    -> s = ""
    \/ exists i, i < length s
      /\ P (substring 0 (S i) s)
      /\ star P (substring (S i) (length s - S i) s).
    Hint Extern 1 (exists i : nat, _) =>
      match goal with
        | [ H : P (String _ ?S) |- _ ] => exists (length S); crush
      end.

    induction 1; [
      crush
      | match goal with
          | [ _ : P ?S |- _ ] => destruct S; crush
        end
    ].
  Qed.    

  Lemma star_substring_inv : forall n,
    n <= length s
    -> star P (substring n (length s - n) s)
    -> substring n (length s - n) s = ""
    \/ exists l, l < length s - n
      /\ P (substring n (S l) s)
      /\ star P (substring (n + S l) (length s - (n + S l)) s).
1088
    Hint Rewrite plus_n_Sm'.
1089 1090 1091 1092 1093 1094

    intros;
      match goal with
        | [ H : star _ _ |- _ ] => generalize (star_inv H); do 3 crush; eauto
      end.
  Qed.
Adam Chlipala's avatar
Adam Chlipala committed
1095 1096 1097
  (* end hide *)

  (** The function [dec_star''] implements a single iteration of the star.  That is, it tries to find a string prefix matching [P], and it calls a parameter function on the remainder of the string. *)
1098 1099 1100

  Section dec_star''.
    Variable n : nat.
Adam Chlipala's avatar
Adam Chlipala committed
1101
    (** [n] is the length of the prefix of [s] that we have already processed. *)
1102 1103 1104 1105

    Variable P' : string -> Prop.
    Variable P'_dec : forall n' : nat, n' > n
      -> {P' (substring n' (length s - n') s)}
Adam Chlipala's avatar
Adam Chlipala committed
1106
      + {~ P' (substring n' (length s - n') s)}.
Adam Chlipala's avatar
Adam Chlipala committed
1107 1108 1109
    (** When we use [dec_star''], we will instantiate [P'_dec] with a function for continuing the search for more instances of [P] in [s]. *)

    (** Now we come to [dec_star''] itself.  It takes as an input a natural [l] that records how much of the string has been searched so far, as we did for [split'].  The return type expresses that [dec_star''] is looking for an index into [s] that splits [s] into a nonempty prefix and a suffix, such that the prefix satisfies [P] and the suffix satisfies [P']. *)
1110

1111 1112
    Definition dec_star'' : forall l : nat,
      {exists l', S l' <= l
1113 1114
        /\ P (substring n (S l') s) /\ P' (substring (n + S l') (length s - (n + S l')) s)}
      + {forall l', S l' <= l
Adam Chlipala's avatar
Adam Chlipala committed
1115 1116
        -> ~ P (substring n (S l') s)
        \/ ~ P' (substring (n + S l') (length s - (n + S l')) s)}.
1117 1118 1119
      refine (fix F (l : nat) : {exists l', S l' <= l
        /\ P (substring n (S l') s) /\ P' (substring (n + S l') (length s - (n + S l')) s)}
      + {forall l', S l' <= l
Adam Chlipala's avatar
Adam Chlipala committed
1120 1121
        -> ~ P (substring n (S l') s)
        \/ ~ P' (substring (n + S l') (length s - (n + S l')) s)} :=
1122 1123 1124 1125 1126
      match l return {exists l', S l' <= l
        /\ P (substring n (S l') s) /\ P' (substring (n + S l') (length s - (n + S l')) s)}
      + {forall l', S l' <= l
        -> ~ P (substring n (S l') s)
        \/ ~ P' (substring (n + S l') (length s - (n + S l')) s)} with
1127 1128 1129 1130 1131 1132 1133 1134 1135 1136 1137
        | O => _
        | S l' =>
          (P_dec (substring n (S l') s) && P'_dec (n' := n + S l') _)
          || F l'
      end); clear F; crush; eauto 7;
      match goal with
        | [ H : ?X <= S ?Y |- _ ] => destruct (eq_nat_dec X (S Y)); crush
      end.
    Defined.
  End dec_star''.

Adam Chlipala's avatar
Adam Chlipala committed
1138
  (* begin hide *)
Adam Chlipala's avatar
Adam Chlipala committed
1139 1140 1141 1142 1143 1144 1145 1146 1147 1148 1149 1150 1151 1152 1153
  Lemma star_length_contra : forall n,
    length s > n
    -> n >= length s
    -> False.
    crush.
  Qed.

  Lemma star_length_flip : forall n n',
    length s - n <= S n'
    -> length s > n
    -> length s - n > 0.
    crush.
  Qed.

  Hint Resolve star_length_contra star_length_flip substring_suffix_emp.
Adam Chlipala's avatar
Adam Chlipala committed
1154
  (* end hide *)
Adam Chlipala's avatar
Adam Chlipala committed
1155

Adam Chlipala's avatar
Adam Chlipala committed
1156 1157
  (** The work of [dec_star''] is nested inside another linear search by [dec_star'], which provides the final functionality we need, but for arbitrary suffixes of [s], rather than just for [s] overall. *)
  
1158
  Definition dec_star' : forall n n' : nat, length s - n' <= n
1159
    -> {star P (substring n' (length s - n') s)}
Adam Chlipala's avatar
Adam Chlipala committed
1160 1161
    + {~ star P (substring n' (length s - n') s)}.
    refine (fix F (n n' : nat) : length s - n' <= n
1162
      -> {star P (substring n' (length s - n') s)}
Adam Chlipala's avatar
Adam Chlipala committed
1163 1164
      + {~ star P (substring n' (length s - n') s)} :=
      match n with
1165 1166 1167
        | O => fun _ => Yes
        | S n'' => fun _ =>
          le_gt_dec (length s) n'
Adam Chlipala's avatar
Adam Chlipala committed
1168 1169
          || dec_star'' (n := n') (star P)
            (fun n0 _ => Reduce (F n'' n0 _)) (length s - n')
Adam Chlipala's avatar
Adam Chlipala committed
1170 1171 1172 1173 1174 1175 1176 1177
      end); clear F; crush; eauto;
    match goal with
      | [ H : star _ _ |- _ ] => apply star_substring_inv in H; crush; eauto
    end;
    match goal with
      | [ H1 : _ < _ - _, H2 : forall l' : nat, _ <= _ - _ -> _ |- _ ] =>
        generalize (H2 _ (lt_le_S _ _ H1)); tauto
    end.
1178 1179
  Defined.

1180
  (** Finally, we have [dec_star], defined by straightforward reduction from [dec_star']. *)
Adam Chlipala's avatar
Adam Chlipala committed
1181

Adam Chlipala's avatar
Adam Chlipala committed
1182
  Definition dec_star : {star P s} + {~ star P s}.
1183
    refine (Reduce (dec_star' (n := length s) 0 _)); crush.
1184 1185 1186
  Defined.
End dec_star.

Adam Chlipala's avatar
Adam Chlipala committed
1187
(* begin hide *)
1188 1189 1190 1191 1192 1193 1194 1195
Lemma app_cong : forall x1 y1 x2 y2,
  x1 = x2
  -> y1 = y2
  -> x1 ++ y1 = x2 ++ y2.
  congruence.
Qed.

Hint Resolve app_cong.
Adam Chlipala's avatar
Adam Chlipala committed
1196 1197 1198
(* end hide *)

(** With these helper functions completed, the implementation of our [matches] function is refreshingly straightforward.  We only need one small piece of specific tactic work beyond what [crush] does for us. *)
1199

1200
Definition matches : forall P (r : regexp P) s, {P s} + {~ P s}.
Adam Chlipala's avatar
Adam Chlipala committed
1201
  refine (fix F P (r : regexp P) s : {P s} + {~ P s} :=
1202 1203 1204
    match r with
      | Char ch => string_dec s (String ch "")
      | Concat _ _ r1 r2 => Reduce (split (F _ r1) (F _ r2) s)
1205
      | Or _ _ r1 r2 => F _ r1 s || F _ r2 s
1206
      | Star _ r => dec_star _ _ _
1207 1208 1209
    end); crush;
  match goal with
    | [ H : _ |- _ ] => generalize (H _ _ (refl_equal _))
Adam Chlipala's avatar
Adam Chlipala committed
1210
  end; tauto.
1211 1212
Defined.

Adam Chlipala's avatar
Adam Chlipala committed
1213 1214
(** It is interesting to pause briefly to consider alternate implementations of [matches].  Dependent types give us much latitude in how specific correctness properties may be encoded with types.  For instance, we could have made [regexp] a non-indexed inductive type, along the lines of what is possible in traditional ML and Haskell.  We could then have implemented a recursive function to map [regexp]s to their intended meanings, much as we have done with types and programs in other examples.  That style is compatible with the [refine]-based approach that we have used here, and it might be an interesting exercise to redo the code from this subsection in that alternate style or some further encoding of the reader's choice.  The main advantage of indexed inductive types is that they generally lead to the smallest amount of code. *)

Adam Chlipala's avatar
Adam Chlipala committed
1215
(* begin hide *)
1216
Example hi := Concat (Char "h"%char) (Char "i"%char).
1217 1218
Eval hnf in matches hi "hi".
Eval hnf in matches hi "bye".
1219 1220

Example a_b := Or (Char "a"%char) (Char "b"%char).
1221 1222 1223 1224
Eval hnf in matches a_b "".
Eval hnf in matches a_b "a".
Eval hnf in matches a_b "aa".
Eval hnf in matches a_b "b".
Adam Chlipala's avatar
Adam Chlipala committed
1225 1226
(* end hide *)

1227
(** Many regular expression matching problems are easy to test.  The reader may run each of the following queries to verify that it gives the correct answer.  We use evaluation strategy %\index{tactics!hnf}%[hnf] to reduce each term to%\index{head-normal form}% _head-normal form_, where the datatype constructor used to build its value is known. *)
1228 1229

Example a_star := Star (Char "a"%char).
1230 1231 1232 1233
Eval hnf in matches a_star "".
Eval hnf in matches a_star "a".
Eval hnf in matches a_star "b".
Eval hnf in matches a_star "aa".
Adam Chlipala's avatar
Adam Chlipala committed
1234 1235

(** Evaluation inside Coq does not scale very well, so it is easy to build other tests that run for hours or more.  Such cases are better suited to execution with the extracted OCaml code. *)