Skip to content

Commit

Permalink
Fix import in README.Data.Fin.Substitution.UntypedLambda (#2279)
Browse files Browse the repository at this point in the history
Also import this module in doc/README.agda so that it is covered by CI.

Closes #2278.
  • Loading branch information
andreasabel authored Feb 7, 2024
1 parent 8567537 commit c8496d0
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 1 deletion.
4 changes: 4 additions & 0 deletions doc/README.agda
Original file line number Diff line number Diff line change
Expand Up @@ -222,6 +222,10 @@ import Text.Printf

import README.Case

-- Showcasing the framework for well-scoped substitutions

import README.Data.Fin.Substitution.UntypedLambda

-- Some examples showing how combinators can be used to emulate
-- "functional reasoning"

Expand Down
2 changes: 1 addition & 1 deletion doc/README/Data/Fin/Substitution/UntypedLambda.agda
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ open import Data.Fin.Substitution.Lemmas
open import Data.Nat.Base hiding (_/_)
open import Data.Fin.Base using (Fin)
open import Data.Vec.Base
open import Relation.Binary.PropositionalEquality.Core
open import Relation.Binary.PropositionalEquality
using (_≡_; refl; sym; cong; cong₂; module ≡-Reasoning)
open import Relation.Binary.Construct.Closure.ReflexiveTransitive
using (Star; ε; _◅_)
Expand Down

0 comments on commit c8496d0

Please sign in to comment.