Skip to content

Commit

Permalink
chore(computability/*FA): remove unnecessary type variables (#5613)
Browse files Browse the repository at this point in the history
  • Loading branch information
foxthomson committed Jan 4, 2021
1 parent 9535f91 commit 2300b47
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion src/computability/DFA.lean
Expand Up @@ -27,7 +27,7 @@ structure DFA (α : Type u) (σ : Type v) :=

namespace DFA

variables {α : Type u} {σ σ₁ σ₂ σ₃ : Type v} (M : DFA α σ)
variables {α : Type u} {σ : Type v} (M : DFA α σ)

instance [inhabited σ] : inhabited (DFA α σ) :=
⟨DFA.mk (λ _ _, default σ) (default σ) ∅⟩
Expand Down
4 changes: 2 additions & 2 deletions src/computability/NFA.lean
Expand Up @@ -29,11 +29,11 @@ structure NFA (α : Type u) (σ : Type v) :=
(start : set σ)
(accept : set σ)

variables {α : Type u} {σ σ' σ₁ σ₂ σ₃ : Type v} (M : NFA α σ)
variables {α : Type u} {σ σ' : Type v} (M : NFA α σ)

namespace NFA

instance : inhabited (NFA α σ') := ⟨ NFA.mk (λ _ _, ∅) ∅ ∅ ⟩
instance : inhabited (NFA α σ) := ⟨ NFA.mk (λ _ _, ∅) ∅ ∅ ⟩

/-- `M.step_set S a` is the union of `M.step s a` for all `s ∈ S`. -/
def step_set : set σ → α → set σ :=
Expand Down

0 comments on commit 2300b47

Please sign in to comment.