Skip to content

Commit

Permalink
Add locality to Hint commands
Browse files Browse the repository at this point in the history
  • Loading branch information
Casteran committed Sep 11, 2023
1 parent b38f24b commit 175a5b5
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 5 deletions.
4 changes: 2 additions & 2 deletions theories/ordinals/Epsilon0/Canon.v
Original file line number Diff line number Diff line change
Expand Up @@ -1039,7 +1039,7 @@ Proof.
destruct k; apply E0_eq_intro; reflexivity.
Qed.

Hint Rewrite Canon_Omega : E0_rw.
#[export] Hint Rewrite Canon_Omega : E0_rw.

Lemma CanonSSn (i:nat) :
forall alpha n , alpha <> E0zero ->
Expand Down Expand Up @@ -1095,7 +1095,7 @@ Proof.
simpl; apply T1limit_canonS_not_zero; auto.
Qed.

#[global]
#[export]
Hint Resolve CanonS_lt Canon_lt Canon_of_limit_not_null : E0.

Lemma CanonS_phi0_Succ alpha i : CanonS (E0phi0 (E0succ alpha)) i =
Expand Down
2 changes: 1 addition & 1 deletion theories/ordinals/Epsilon0/Hprime.v
Original file line number Diff line number Diff line change
Expand Up @@ -94,7 +94,7 @@ Proof.
- apply Succ_Succb.
Qed.

Hint Rewrite H'_eq1 H'_eq2 : H'_rw.
#[export] Hint Rewrite H'_eq1 H'_eq2 : H'_rw.

Ltac lim_rw alpha := (assert (E0limit alpha) by auto with E0);
rewrite (H'_eq3 alpha); auto with E0.
Expand Down
4 changes: 2 additions & 2 deletions theories/ordinals/Epsilon0/L_alpha.v
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ From Equations Require Import Equations.
Import RelationClasses Relations.

#[global] Instance Olt : WellFounded E0lt := E0lt_wf.
#[global] Hint Resolve Olt : E0.
#[export] Hint Resolve Olt : E0.

(** Using Coq-Equations for building a function which satisfies
[Large_sets.L_spec] *)
Expand Down Expand Up @@ -68,7 +68,7 @@ Proof.
Qed.


Hint Rewrite L_zero_eqn L_succ_eqn : L_rw.
#[export] Hint Rewrite L_zero_eqn L_succ_eqn : L_rw.

(* begin snippet Paraphrasesc:: no-out *)
Lemma L_lim_eqn alpha i :
Expand Down

0 comments on commit 175a5b5

Please sign in to comment.