Skip to content

Commit

Permalink
Prepare the final ICFP'19 artefact.
Browse files Browse the repository at this point in the history
  • Loading branch information
geo2a committed Jun 28, 2019
1 parent c732d69 commit 3d41037
Show file tree
Hide file tree
Showing 15 changed files with 634 additions and 2,546 deletions.
21 changes: 11 additions & 10 deletions Makefile
Original file line number Diff line number Diff line change
@@ -1,15 +1,16 @@
COQFLAGS = ""
all: Makefile.coq
+$(MAKE) -f Makefile.coq all

VFILES = $(wildcard src/*.v)
VOFILES = $(patsubst %.v,%.vo,$(VFILES))
clean: Makefile.coq
+$(MAKE) -f Makefile.coq cleanall
rm -f Makefile.coq Makefile.coq.conf

all: $(VOFILES)
Makefile.coq: _CoqProject
$(COQBIN)coq_makefile -f _CoqProject -o Makefile.coq

%.vo: %.v Makefile.coq
$(MAKE) -f Makefile.coq OPT=$(COQFLAGS)
_CoqProject Makefile: ;

Makefile.coq: _CoqProject
coq_makefile -f _CoqProject -o $@
%: Makefile.coq
+$(MAKE) -f Makefile.coq $@

clean: Makefile.coq
$(MAKE) -f Makefile.coq clean
.PHONY: all clean
4 changes: 1 addition & 3 deletions _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -2,13 +2,11 @@
src/Prelude.v
src/Ltac.v
src/Data/Functor.v
src/Data/Functor/Contravariant.v
src/Data/Functor/Const.v
src/Control/Applicative.v
src/Data/Either.v
src/Data/Monoid.v
src/Control/Selective.v
src/Data/Over.v
src/Data/Under.v
src/Data/Validation.v
src/Control/Selective/FreerRigid.v
src/Control/Selective/Rigid.v
1 change: 0 additions & 1 deletion src/Control/Applicative.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,5 @@
Require Export Hask.Ltac.
Require Export Hask.Data.Functor.
Require Export Hask.Data.Functor.Const.
Require Import FunctionalExtensionality.

Generalizable All Variables.
Expand Down
219 changes: 0 additions & 219 deletions src/Control/Applicative/Free.v

This file was deleted.

6 changes: 2 additions & 4 deletions src/Control/Selective.v
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Require Import Hask.Prelude.
Require Import Data.Either.
Require Import Data.Monoid.
Require Import Hask.Data.Functor.
Require Import Hask.Data.Functor.Const.
Require Import Hask.Control.Applicative.

Generalizable All Variables.
Expand All @@ -31,11 +30,11 @@ Definition apS `{Selective f} {A B : Type}
(* selectA x y = (\e f -> either f id e) <$> x <*> y *)
Definition selectA `{Applicative f} {A B : Type}
(x : f (Either A B)) (y : f (A -> B)) : f B :=
(fun e f => either f id e) <$> x <*> y.
(fun e f => either f id e) <$> x <*> y.

Module SelectiveLaws.

Include ApplicativeLaws.
Include ApplicativeLaws.

Definition law3_f {A B C : Type}
(x : B + C) : B + (A + C) := Right <$> x.
Expand All @@ -62,4 +61,3 @@ Class SelectiveLaws (F : Type -> Type) `{Selective F} := {
}.

End SelectiveLaws.

Loading

0 comments on commit 3d41037

Please sign in to comment.