Skip to content

Commit

Permalink
compiles with Coq 8.8 and SSR dev from 23/05/2018
Browse files Browse the repository at this point in the history
  • Loading branch information
grianneau committed Jul 17, 2018
1 parent d441188 commit 59c4349
Show file tree
Hide file tree
Showing 7 changed files with 12 additions and 12 deletions.
2 changes: 1 addition & 1 deletion auxresults/auxresults.v
Original file line number Diff line number Diff line change
Expand Up @@ -508,7 +508,7 @@ End MorePath.

Section MoreFinmap.

Open Local Scope fset_scope.
Local Open Scope fset_scope.

Lemma finSet_notin_ind (T : choiceType) (P : {fset T} -> Prop) :
P fset0 -> (forall s x, P s -> x \notin s -> P (x |` s)) -> forall s, P s.
Expand Down
2 changes: 1 addition & 1 deletion coq-ssr-elliptic-curves/polyall.v
Original file line number Diff line number Diff line change
Expand Up @@ -13,7 +13,7 @@ From mathcomp Require Export polyorder.

Import GRing.Theory.

Open Local Scope ring_scope.
Local Open Scope ring_scope.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down
2 changes: 1 addition & 1 deletion coq-ssr-elliptic-curves/polydec.v
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ From mathcomp Require Import ssrfun choice tuple fintype bigop.

Import GRing.Theory.

Open Local Scope ring_scope.
Local Open Scope ring_scope.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down
2 changes: 1 addition & 1 deletion newtonsums/expansiblefracpoly.v
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ Unset Printing Implicit Defensive.

Import GRing.Theory.
Local Open Scope ring_scope.
Open Local Scope quotient_scope.
Local Open Scope quotient_scope.

Section ExpansibleFracpoly.

Expand Down
4 changes: 2 additions & 2 deletions newtonsums/fracrev.v
Original file line number Diff line number Diff line change
Expand Up @@ -14,8 +14,8 @@ Unset Strict Implicit.
Unset Printing Implicit Defensive.

Import GRing.Theory.
Open Local Scope ring_scope.
Open Local Scope quotient_scope.
Local Open Scope ring_scope.
Local Open Scope quotient_scope.

Reserved Notation "{ 'fracpoly' T }" (at level 0, format "{ 'fracpoly' T }").
Reserved Notation "x %:F" (at level 2, format "x %:F").
Expand Down
4 changes: 2 additions & 2 deletions newtonsums/fraction.v
Original file line number Diff line number Diff line change
Expand Up @@ -16,8 +16,8 @@ Unset Strict Implicit.
Unset Printing Implicit Defensive.

Import GRing.Theory.
Open Local Scope ring_scope.
Open Local Scope quotient_scope.
Local Open Scope ring_scope.
Local Open Scope quotient_scope.

Reserved Notation "{ 'ratio' T }" (at level 0, format "{ 'ratio' T }").
Reserved Notation "{ 'fraction' T }" (at level 0, format "{ 'fraction' T }").
Expand Down
8 changes: 4 additions & 4 deletions semialgebraic/semialgebraic.v
Original file line number Diff line number Diff line change
Expand Up @@ -1108,7 +1108,7 @@ Proof.
move : s; apply : quotP => f hf.
rewrite /SA_all_proj; unlock.
apply/eqP; rewrite eqmodE hf.
apply/rcf_satP/nforallP => u; rewrite cat0s.
apply/rcf_satP/nforallP => u; rewrite cat0s /=.
split=> h x.
+ by move/(_ x)/holds_repr_pi/(_ x) : h; rewrite set_set_nth eqxx.
+ apply/holds_repr_pi => y; rewrite set_set_nth eqxx.
Expand Down Expand Up @@ -3437,9 +3437,9 @@ Fail Fixpoint test (p : {poly F}) :=
else (test p^`())*(2%:R).

Check (fun (p : {poly F}) => if (size p <= 1)%N then [::] else (polyrcf.rootsR p)).
Fixpoint vroot (p : {poly F}) :=
if (size p <= 1)%N then [::]
else let s := vroot (p^`()) in (polyrcf.rootsR p).
(* Fixpoint vroot (p : {poly F}) := *)
(* if (size p <= 1)%N then [::] *)
(* else let s := vroot (p^`()) in (polyrcf.rootsR p). *)

(* Variables (A : choiceType) (x : {fset A}) (P : pred A) (a : A) (ha : P a) (i : nat). *)
(* Check (unpickle P i x). *)
Expand Down

0 comments on commit 59c4349

Please sign in to comment.