playground/coq/unfinished/water-jars.v

12 lines
359 B
Coq

Inductive jar (capacity:nat) : nat -> Set :=
| Jar : forall n:nat, n <= capacity -> jar capacity n.
(* Show me that n<=capacity then I'll give you a jar *)
(*
Inductive system (S B:nat) : Set :=
| System : forall s b:nat, s<=S /\ b<=B -> jar S s * jar B b -> system S B.
*)
Inductive moves (sys: system 9 5) : system 9 5 : Set :=
| S2B : System 9 5 _ (Jar