Skip to content

Commit adb1852

Browse files
committed
[ fix ] We can't turn non-fatal error warnings anymore
1 parent 037ba15 commit adb1852

File tree

2 files changed

+6
-2
lines changed

2 files changed

+6
-2
lines changed

README/Data/List/Relation/Binary/Equality.agda

+3-1
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
-- Documentation for pointwise equality over `List`s
55
------------------------------------------------------------------------
66

7-
{-# OPTIONS --warning noMissingDefinitions #-}
7+
{-# OPTIONS --allow-unsolved-metas #-}
88

99
module README.Data.List.Relation.Binary.Equality where
1010

@@ -37,6 +37,7 @@ lem₁ = refl
3737
-- equality of two lists of the type `List (ℕ → ℕ)`:
3838

3939
lem₂ : (λ x 2 * x + 2) ∷ [] ≡ (λ x 2 * (x + 1)) ∷ []
40+
lem₂ = {!!}
4041

4142
-- In such a case it is impossible to prove the two lists equal with
4243
-- refl as the two functions are not propositionally equal. In the
@@ -56,6 +57,7 @@ open import Relation.Binary.PropositionalEquality using (_≗_)
5657
open import Data.List.Relation.Binary.Pointwise using (Pointwise)
5758

5859
lem₃ : Pointwise _≗_ ((λ x x + 1) ∷ []) ((λ x x + 21) ∷ [])
60+
lem₃ = {!!}
5961

6062
-- the library provides some nicer wrappers and infix notation in the
6163
-- folder "Data.List.Relation.Binary.Equality".

README/Design/Hierarchies.agda

+3-1
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@
44
-- An explanation about how mathematical hierarchies are laid out.
55
------------------------------------------------------------------------
66

7-
{-# OPTIONS --warning noMissingDefinitions #-}
7+
{-# OPTIONS --allow-unsolved-metas #-}
88

99
module README.Design.Hierarchies where
1010

@@ -261,9 +261,11 @@ record Semigroup : Set (suc (a ⊔ ℓ)) where
261261
-- one to translate between left and right identities.
262262

263263
total⇒refl : {_∼_ : Rel A ℓ} Total _∼_ Reflexive _∼_
264+
total⇒refl = {!!}
264265

265266
idˡ+comm⇒idʳ : {_≈_ : Rel A ℓ} {e _∙_} Commutative _≈_ _∙_
266267
LeftIdentity _≈_ e _∙_ RightIdentity _≈_ e _∙_
268+
idˡ+comm⇒idʳ = {!!}
267269

268270
------------------------------------------------------------------------
269271
-- X.Construct

0 commit comments

Comments
 (0)