Skip to content

Commit

Permalink
Removed stdlib
Browse files Browse the repository at this point in the history
  • Loading branch information
patrick-nicodemus committed Aug 21, 2024
1 parent d47bbd7 commit 1359ed2
Show file tree
Hide file tree
Showing 13 changed files with 16 additions and 2 deletions.
4 changes: 3 additions & 1 deletion examples/dune
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,8 @@
(package coq-elpi)
(name elpi_examples)
(plugins coq-elpi.elpi)
(theories elpi))
(theories elpi Coq)
(stdlib no)
)

; (include_subdirs qualified)
1 change: 1 addition & 0 deletions examples/example_abs_evars.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Prelude.
From elpi Require Import elpi.

(** Closing a term with holes with binders *)
Expand Down
1 change: 1 addition & 0 deletions examples/example_curry_howard_tactics.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Prelude.
From elpi Require Import elpi.

(* Tactics
Expand Down
3 changes: 2 additions & 1 deletion examples/example_fuzzer.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Prelude.
From elpi Require Import elpi.

(** Intrinsically typed data type and semantics, from software foundations.
Expand Down Expand Up @@ -96,4 +97,4 @@ Elpi Typecheck.
Elpi fuzz eval eval1.

(* let's print our new, broken, semantics ;-) *)
Print eval1.
Print eval1.
1 change: 1 addition & 0 deletions examples/example_generalize.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Prelude.
From elpi Require Import elpi.

(** Abstract a term over something, like the generalize tactic *)
Expand Down
1 change: 1 addition & 0 deletions examples/example_import_projections.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Prelude.
From elpi Require Import elpi.

(* "import" a record instance by naming it's applied projections *)
Expand Down
1 change: 1 addition & 0 deletions examples/example_record_expansion.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Datatypes Logic.
From elpi Require Import elpi.

(**
Expand Down
1 change: 1 addition & 0 deletions examples/example_record_to_sigma.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,4 @@
From Coq Require Import Datatypes Logic Specif.
From elpi Require Import elpi.

(* Define a command to turn records into nested sigma types, suggested
Expand Down
1 change: 1 addition & 0 deletions examples/example_reduction_surgery.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@
from a given module.
*)

From Coq Require Import Prelude.
From elpi Require Import elpi.

Elpi Tactic reduce.
Expand Down
1 change: 1 addition & 0 deletions examples/example_reflexive_tactic.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,6 +9,7 @@
*)

From Coq Require Import Prelude.
From elpi Require elpi.
Require Arith ZArith Psatz List ssreflect.

Expand Down
1 change: 1 addition & 0 deletions examples/tutorial_coq_elpi_HOAS.v
Original file line number Diff line number Diff line change
Expand Up @@ -45,6 +45,7 @@ HOAS for Gallina
|*)

From Coq Require Import Prelude. (* .none *)
From elpi Require Import elpi. (* .none *)

Elpi Command tutorial_HOAS. (* .none *)
Expand Down
1 change: 1 addition & 0 deletions examples/tutorial_coq_elpi_command.v
Original file line number Diff line number Diff line change
Expand Up @@ -44,6 +44,7 @@ Let's create a simple command, called "hello", which prints :e:`"Hello"`
followed by the arguments we pass to it:
|*)
From Coq Require Import Prelude.
From elpi Require Import elpi.

Elpi Command hello.
Expand Down
1 change: 1 addition & 0 deletions examples/tutorial_coq_elpi_tactic.v
Original file line number Diff line number Diff line change
Expand Up @@ -55,6 +55,7 @@ Let's define a simple tactic that prints the current goal.
|*)

From Coq Require Import Prelude.
From elpi Require Import elpi.

Elpi Tactic show.
Expand Down

0 comments on commit 1359ed2

Please sign in to comment.