Skip to content

Commit

Permalink
consistently use #[local] instead of Local
Browse files Browse the repository at this point in the history
  • Loading branch information
palmskog committed Aug 3, 2023
1 parent 6d5f456 commit 652431a
Show file tree
Hide file tree
Showing 6 changed files with 10 additions and 10 deletions.
6 changes: 3 additions & 3 deletions theories/dfa.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,7 +11,7 @@ Unset Strict Implicit.

Section FA.
Variable char : finType.
Local Notation word := (word char).
#[local] Notation word := (word char).

(** * Deterministic Finite Automata *)

Expand Down Expand Up @@ -157,7 +157,7 @@ Qed.
Section CutOff.
Variables (aT rT : finType) (f : seq aT -> rT).
Hypothesis RC_f : forall x y a, f x = f y -> f (x++[::a]) = f (y++[::a]).
Local Set Default Proof Using "RC_f".
#[local] Set Default Proof Using "RC_f".

Lemma RC_seq x y z : f x = f y -> f (x++z) = f (y++z).
Proof.
Expand Down Expand Up @@ -436,7 +436,7 @@ Section NonRegular.
Qed.

Hypothesis (a b : char) (Hab : a != b).
Local Set Default Proof Using "Hab".
#[local] Set Default Proof Using "Hab".

Definition Lab w := exists n, w = nseq n a ++ nseq n b.

Expand Down
2 changes: 1 addition & 1 deletion theories/languages.v
Original file line number Diff line number Diff line change
Expand Up @@ -49,7 +49,7 @@ Section HomDef.

Definition homomorphism := forall w1 w2, h (w1 ++ w2) = h w1 ++ h w2.
Hypothesis h_hom : homomorphism.
Local Set Default Proof Using "h_hom".
#[local] Set Default Proof Using "h_hom".

Lemma h0 : h [::] = [::].
Proof.
Expand Down
6 changes: 3 additions & 3 deletions theories/minimization.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,14 +11,14 @@ Set Implicit Arguments.
Unset Printing Implicit Defensive.
Unset Strict Implicit.

Local Open Scope quotient_scope.
#[local] Open Scope quotient_scope.

(** * DFA Minimization *)

Section Minimization.
Variable (char : finType).
Local Notation word := (word char).
Local Notation dfa := (dfa char).
#[local] Notation word := (word char).
#[local] Notation dfa := (dfa char).

Definition coll (A : dfa) x y := forall w, (delta x w \in dfa_fin A) = (delta y w \in dfa_fin A).

Expand Down
2 changes: 1 addition & 1 deletion theories/misc.v
Original file line number Diff line number Diff line change
Expand Up @@ -121,7 +121,7 @@ Proof. rewrite -!cardsT -powersetT. exact: card_powerset. Qed.

(** Miscellaneous *)

Local Open Scope quotient_scope.
#[local] Open Scope quotient_scope.
Lemma epiK {T:choiceType} (e : equiv_rel T) x : e (repr (\pi_{eq_quot e} x)) x.
Proof. by rewrite -eqmodE reprK. Qed.

Expand Down
2 changes: 1 addition & 1 deletion theories/myhill_nerode.v
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,7 @@ exist most general classifiers corresponding to minimal automata. *)
Section Clasifiers.

Variable char: finType.
Local Notation word := (word char).
#[local] Notation word := (word char).

Record classifier := Classifier {
classifier_classes : finType;
Expand Down
2 changes: 1 addition & 1 deletion theories/nfa.v
Original file line number Diff line number Diff line change
Expand Up @@ -11,7 +11,7 @@ Unset Strict Implicit.

Section NFA.
Variable char : finType.
Local Notation word := (word char).
#[local] Notation word := (word char).

(** * Nondeterministic Finite Automata.
Expand Down

0 comments on commit 652431a

Please sign in to comment.