Skip to content

Commit f87cc31

Browse files
committed
fix L framework for 9.0
1 parent df94add commit f87cc31

File tree

20 files changed

+56
-517
lines changed

20 files changed

+56
-517
lines changed

theories/L/Computability/Synthetic.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -209,7 +209,7 @@ Qed.
209209
Definition F1 {X} (T : nat -> list X) := (fun n => let (n, m) := Cantor.of_nat n in nth_error (T n) m).
210210

211211
#[global]
212-
Instance term_F1 {X} {H : encodable X} : @computable ((nat -> list X) -> nat -> option X) ((! nat ~> ! list X) ~> ! nat ~> ! option X) (@F1 X).
212+
Instance term_F1 {X} {H : encodable X} : @computable ((nat -> list X) -> nat -> option X) ((! nat ~> ! (list X)) ~> ! nat ~> ! (option X)) (@F1 X).
213213
Proof.
214214
extract.
215215
Qed.

theories/L/Datatypes/LBool.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ From Undecidability.L.Tactics Require Import LTactics GenEncode.
66
(* Eval simpl in *)
77
(* if b then .\"t", "f"; "t" else .\"t", "f"; "f". *)
88

9-
MetaCoq Run (tmGenEncodeInj "bool_enc" bool).
9+
MetaRocq Run (tmGenEncodeInj "bool_enc" bool).
1010
(* For each encoding, Lrewrite must contain an lemma that solves goals like "encode b s t >* match ...end". The database Lrewrite also calls Lproc to discharge the other assumptions *)
1111
#[export] Hint Resolve bool_enc_correct : Lrewrite.
1212

theories/L/Datatypes/LNat.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ From Undecidability.L Require Import Datatypes.LBool Functions.EqBool Datatypes.
77
Import GenEncode. Import Nat.
88
(* ** Encoding of natural numbers *)
99

10-
MetaCoq Run (tmGenEncodeInj "nat_enc" nat).
10+
MetaRocq Run (tmGenEncodeInj "nat_enc" nat).
1111
#[export] Hint Resolve nat_enc_correct : Lrewrite.
1212

1313
#[global]
@@ -114,7 +114,7 @@ Proof.
114114
Qed.
115115

116116
Lemma unenc_correct2 t n : nat_unenc t = Some n -> nat_enc n = t.
117-
Proof with try solve [Coq.Init.Tactics.easy].
117+
Proof.
118118
revert n. eapply (size_induction (f := size) (p := (fun t => forall n, nat_unenc t = Some n -> nat_enc n = t))). clear t. intros t IHt n H.
119119
destruct t as [ | | t]. easy. easy.
120120
destruct t as [ | | t]. easy. easy.

theories/L/Datatypes/LOptions.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,7 @@ Section Fix_X.
88
Context {intX : encodable X}.
99

1010

11-
MetaCoq Run (tmGenEncode "option_enc" (option X)).
11+
MetaRocq Run (tmGenEncode "option_enc" (option X)).
1212
Hint Resolve option_enc_correct : Lrewrite.
1313

1414
Global Instance encInj_option_enc {H : encInj intX} : encInj (encodable_option_enc).

theories/L/Datatypes/LProd.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ Section Fix_XY.
1515
Context {intX : encodable X}.
1616
Context {intY : encodable Y}.
1717

18-
MetaCoq Run (tmGenEncode "prod_enc" (X * Y)).
18+
MetaRocq Run (tmGenEncode "prod_enc" (X * Y)).
1919
Hint Resolve prod_enc_correct : Lrewrite.
2020

2121
Global Instance encInj_prod_enc {H : encInj intX} {H' : encInj intY} : encInj (encodable_prod_enc).

theories/L/Datatypes/LSum.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -9,7 +9,7 @@ Section Fix_XY.
99
Variable intX : encodable X.
1010
Variable intY : encodable Y.
1111

12-
MetaCoq Run (tmGenEncode "sum_enc" (X + Y)).
12+
MetaRocq Run (tmGenEncode "sum_enc" (X + Y)).
1313
Hint Resolve sum_enc_correct : Lrewrite.
1414

1515
Global Instance encInj_sum_enc {H : encInj intX} {H' : encInj intY} : encInj (encodable_sum_enc).

theories/L/Datatypes/LTerm.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ From Undecidability.L Require Export Util.L_facts.
33
From Undecidability.L.Tactics Require Import LTactics GenEncode.
44

55
(* ** Encoding for L-terms *)
6-
MetaCoq Run (tmGenEncodeInj "term_enc" term).
6+
MetaRocq Run (tmGenEncodeInj "term_enc" term).
77
#[export] Hint Resolve term_enc_correct : Lrewrite.
88

99
(* register the non-constant constructors *)

theories/L/Datatypes/LUnit.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,5 +3,5 @@ From Undecidability.L.Tactics Require Import LTactics GenEncode.
33
(* * Encodings and extracted basic functions *)
44
(* ** Encoding of unit *)
55

6-
MetaCoq Run (tmGenEncodeInj "unit_enc" unit).
6+
MetaRocq Run (tmGenEncodeInj "unit_enc" unit).
77
#[export] Hint Resolve unit_enc_correct : Lrewrite.

theories/L/Datatypes/List/List_enc.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Section Fix_X.
66
Variable (X:Type).
77
Context {intX : encodable X}.
88

9-
MetaCoq Run (tmGenEncode "list_enc" (list X)).
9+
MetaRocq Run (tmGenEncode "list_enc" (list X)).
1010

1111
Global Instance encInj_list_enc {H : encInj intX} : encInj (encodable_list_enc).
1212
Proof. register_inj. Qed.

theories/L/Reductions/H10_to_L.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -27,7 +27,7 @@ Inductive poly : Set :=
2727
| poly_add : poly -> poly -> poly
2828
| poly_mul : poly -> poly -> poly.
2929

30-
MetaCoq Run (tmGenEncode "enc_poly" poly).
30+
MetaRocq Run (tmGenEncode "enc_poly" poly).
3131
#[export] Hint Resolve enc_poly_correct : Lrewrite.
3232

3333
#[export]

0 commit comments

Comments
 (0)