Skip to content

Commit 04cc05c

Browse files
committed
Fix import in README.Data.Fin.Substitution.UntypedLambda (#2279)
Also import this module in doc/README.agda so that it is covered by CI. Closes #2278.
1 parent 07988c0 commit 04cc05c

File tree

2 files changed

+5
-1
lines changed

2 files changed

+5
-1
lines changed

doc/README.agda

+4
Original file line numberDiff line numberDiff line change
@@ -222,6 +222,10 @@ import Text.Printf
222222

223223
import README.Case
224224

225+
-- Showcasing the framework for well-scoped substitutions
226+
227+
import README.Data.Fin.Substitution.UntypedLambda
228+
225229
-- Some examples showing how combinators can be used to emulate
226230
-- "functional reasoning"
227231

doc/README/Data/Fin/Substitution/UntypedLambda.agda

+1-1
Original file line numberDiff line numberDiff line change
@@ -14,7 +14,7 @@ open import Data.Fin.Substitution.Lemmas
1414
open import Data.Nat.Base hiding (_/_)
1515
open import Data.Fin.Base using (Fin)
1616
open import Data.Vec.Base
17-
open import Relation.Binary.PropositionalEquality.Core
17+
open import Relation.Binary.PropositionalEquality
1818
using (_≡_; refl; sym; cong; cong₂; module ≡-Reasoning)
1919
open import Relation.Binary.Construct.Closure.ReflexiveTransitive
2020
using (Star; ε; _◅_)

0 commit comments

Comments
 (0)