Skip to content

Commit

Permalink
switched to ssreflect 1.6
Browse files Browse the repository at this point in the history
  • Loading branch information
tebbi committed Jan 18, 2016
1 parent 3d7fcef commit 3214cec
Show file tree
Hide file tree
Showing 14 changed files with 33 additions and 17 deletions.
4 changes: 2 additions & 2 deletions README.md
Original file line number Diff line number Diff line change
Expand Up @@ -8,8 +8,8 @@ https://www.ps.uni-saarland.de/autosubst

## Requirements

- Coq 8.4 or Coq 8.5beta3
- ssreflect version 1.4 or 1.5 for some examples
- Coq 8.4 or Coq 8.5rc1
- ssreflect version 1.6 for some examples



Expand Down
2 changes: 1 addition & 1 deletion examples/plain/Context.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(** * Context *)
Require Import Omega List Program.Equality.
Require Import Autosubst.
Require Import Autosubst.Autosubst.

Fixpoint atn {X} l n (x : X) :=
match l with
Expand Down
8 changes: 6 additions & 2 deletions examples/plain/Demo.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
In this tutorial we will use Autosubst to formalize the simply typed lambda calculus and show substitutivity and type preservation of the reduction relation. *)

Require Import Autosubst.
Require Import Autosubst.Autosubst.

(** ** Syntax and the substitution operation
Expand Down Expand Up @@ -187,4 +187,8 @@ Proof.
inversion H_step; ainv; eauto using ty.
- eapply ty_subst; try eassumption.
intros [|]; simpl; eauto using ty.
Qed.
Qed.

(* Local Variables: *)
(* coq-load-path: (("." "Plain") ("../../theories" "Autosubst")) *)
(* End: *)
3 changes: 2 additions & 1 deletion examples/plain/POPLmark.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,8 @@
progress and preservation of System F with subtyping. *)

Require Import Program.Equality List Omega.
Require Import Autosubst Size Decidable Context.
Require Import Autosubst.Autosubst.
Require Import Size Decidable Context.

Inductive type : Type :=
| TyVar (x : var)
Expand Down
4 changes: 2 additions & 2 deletions examples/plain/Size.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
(** * Support for Size Induction *)
Require Import Omega List Program.Equality.
Require Import Autosubst_Basics.
Require Import Autosubst.Autosubst_Basics.

Class Size (A : Type) := size : A -> nat.

Expand Down Expand Up @@ -111,5 +111,5 @@ Instance size_fact_In (A : Type) (size_A : Size A) x l (x_in_l : In x l) :
Proof. now apply size_In. Qed.

(* Local Variables: *)
(* coq-load-path: (("." "Plain")) *)
(* coq-load-path: (("." "Plain") ("../../theories" "Autosubst")) *)
(* End: *)
3 changes: 2 additions & 1 deletion examples/ssr/ARS.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,8 @@
(** * Abstract Reduction Systems
Useful lemmas when working with small-step reduction relations. *)
Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down
3 changes: 2 additions & 1 deletion examples/ssr/AutosubstSsr.v
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,8 @@ Require Export Autosubst_Classes.
Require Export Autosubst_Tactics.
Require Export Autosubst_Lemmas.
Require Export Autosubst_Derive.
Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down
3 changes: 2 additions & 1 deletion examples/ssr/BetaSubstitution.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
(** * Correctness of Single Variable Substitutions *)
Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import Autosubst.

Set Implicit Arguments.
Expand Down
3 changes: 2 additions & 1 deletion examples/ssr/CR.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import AutosubstSsr ARS.

Set Implicit Arguments.
Expand Down
3 changes: 2 additions & 1 deletion examples/ssr/Context.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,8 @@
(** * Context
Support for dependent contexts with the right reduction behaviour. *)
Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import AutosubstSsr.

Definition get {T} `{Ids T} (Gamma : seq T) (n : var) : T :=
Expand Down
3 changes: 2 additions & 1 deletion examples/ssr/POPLmark.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,8 @@
and in particular does not contain well-formedness assumptions.
*)

Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import AutosubstSsr Context.

(** **** Syntax *)
Expand Down
3 changes: 2 additions & 1 deletion examples/ssr/SystemF_CBV.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,7 @@
(** * Normalization of Call-By-Value System F *)

Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import AutosubstSsr Context.

Set Implicit Arguments.
Expand Down
4 changes: 3 additions & 1 deletion examples/ssr/SystemF_SN.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,7 @@
(** * Strong Normalization of System F *)
Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.

Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import AutosubstSsr ARS Context.

Set Implicit Arguments.
Expand Down
4 changes: 3 additions & 1 deletion examples/ssr/pred_CC_omega.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,9 @@
(** * Predicative CC omega: Type Preservation and Confluence
*)

Require Import Ssreflect.ssreflect Ssreflect.ssrfun Ssreflect.ssrbool Ssreflect.eqtype Ssreflect.ssrnat Ssreflect.seq.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import mathcomp.ssreflect.ssreflect.
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
Require Import AutosubstSsr ARS Context.

Set Implicit Arguments.
Expand Down

0 comments on commit 3214cec

Please sign in to comment.