File tree Expand file tree Collapse file tree 22 files changed +70
-50
lines changed
Binary/Sublist/Propositional/Example Expand file tree Collapse file tree 22 files changed +70
-50
lines changed Original file line number Diff line number Diff line change @@ -1238,6 +1238,12 @@ Major improvements
1238
1238
pre-existing ` Reasoning ` module in just a couple of lines
1239
1239
(e.g. see ` ∣-Reasoning ` in ` Data.Nat.Divisibility ` )
1240
1240
1241
+ * One pre-requisite for that is that ` ≡-Reasoning ` has been moved from
1242
+ ` Relation.Binary.PropositionalEquality.Core ` (which shouldn't be
1243
+ imported anyway as it's a ` Core ` module) to
1244
+ ` Relation.Binary.PropositionalEquality.Properties ` .
1245
+ It is still exported by ` Relation.Binary.PropositionalEquality ` .
1246
+
1241
1247
Deprecated modules
1242
1248
------------------
1243
1249
Original file line number Diff line number Diff line change @@ -21,6 +21,8 @@ open import Data.Vec.Base as Vec using (Vec; _∷_)
21
21
open import Function.Base using (const; flip; id; _∘′_; _$′_; _⟨_⟩_; _∘₂′_)
22
22
open import Level using (Level)
23
23
open import Relation.Binary.PropositionalEquality.Core as P using (_≡_; cong; cong₂)
24
+ open import Relation.Binary.PropositionalEquality.Properties
25
+ using (module ≡-Reasoning )
24
26
25
27
private
26
28
variable
@@ -218,7 +220,7 @@ lookup-transpose n (as ∷ ass) = begin
218
220
lookup as n ∷ lookup (transpose ass) n ≡⟨ cong (lookup as n ∷_) (lookup-transpose n ass) ⟩
219
221
lookup as n ∷ List.map (flip lookup n) ass ≡⟨⟩
220
222
List.map (flip lookup n) (as ∷ ass) ∎
221
- where open P. ≡-Reasoning
223
+ where open ≡-Reasoning
222
224
223
225
lookup-transpose⁺ : ∀ n (ass : List⁺ (Stream A)) →
224
226
lookup (transpose⁺ ass) n ≡ List⁺.map (flip lookup n) ass
@@ -228,7 +230,7 @@ lookup-transpose⁺ n (as ∷ ass) = begin
228
230
lookup as n ∷ lookup (transpose ass) n ≡⟨ cong (lookup as n ∷_) (lookup-transpose n ass) ⟩
229
231
lookup as n ∷ List.map (flip lookup n) ass ≡⟨⟩
230
232
List⁺.map (flip lookup n) (as ∷ ass) ∎
231
- where open P. ≡-Reasoning
233
+ where open ≡-Reasoning
232
234
233
235
lookup-tails : ∀ n (as : Stream A) → lookup (tails as) n ≈ ℕ.iterate tail as n
234
236
lookup-tails zero as = B.refl
Original file line number Diff line number Diff line change @@ -26,6 +26,8 @@ open import Level
26
26
open import Relation.Unary using (Pred)
27
27
import Induction.WellFounded as WF
28
28
open import Relation.Binary.PropositionalEquality.Core as P using (_≡_)
29
+ open import Relation.Binary.PropositionalEquality.Properties
30
+ using (module ≡-Reasoning )
29
31
import Relation.Binary.Construct.On as On
30
32
31
33
private
@@ -132,7 +134,7 @@ merge xss = ⟦ merge′ xss ⟧P
132
134
Any-merge : ∀ xss → Any P (merge xss) ↔ Any (λ { (x , xs) → P x ⊎ Any P xs }) xss
133
135
Any-merge {P = P} xss = mk↔ₛ′ (proj₁ ∘ to xss) from to∘from (proj₂ ∘ to xss)
134
136
where
135
- open P. ≡-Reasoning
137
+ open ≡-Reasoning
136
138
137
139
-- The from function.
138
140
Original file line number Diff line number Diff line change @@ -25,6 +25,8 @@ open import Data.Vec.Base as Vec using (_∷_)
25
25
26
26
open import Function.Base using (id; _$_; _∘′_; const)
27
27
open import Relation.Binary.PropositionalEquality.Core as P using (_≡_; _≢_)
28
+ open import Relation.Binary.PropositionalEquality.Properties
29
+ using (module ≡-Reasoning )
28
30
29
31
private
30
32
variable
@@ -116,7 +118,7 @@ lookup-iterate-identity (suc n) f a = begin
116
118
lookup (iterate f (f a)) n ≡⟨ lookup-iterate-identity n f (f a) ⟩
117
119
fold (f a) f n ≡⟨ fold-pull a f (const ∘′ f) (f a) P.refl (λ _ → P.refl) n ⟩
118
120
f (fold a f n) ≡⟨⟩
119
- fold a f (suc n) ∎ where open P. ≡-Reasoning
121
+ fold a f (suc n) ∎ where open ≡-Reasoning
120
122
121
123
------------------------------------------------------------------------
122
124
-- DEPRECATED
Original file line number Diff line number Diff line change @@ -16,6 +16,8 @@ module Data.Fin.Relation.Unary.Top where
16
16
open import Data.Nat.Base using (ℕ; zero; suc)
17
17
open import Data.Fin.Base using (Fin; zero; suc; fromℕ; inject₁)
18
18
open import Relation.Binary.PropositionalEquality.Core
19
+ open import Relation.Binary.PropositionalEquality.Properties
20
+ using (module ≡-Reasoning )
19
21
20
22
private
21
23
variable
Original file line number Diff line number Diff line change @@ -16,9 +16,11 @@ import Data.Vec.Properties as VecProp
16
16
open import Function.Base as Fun using (_∘_; _$_; flip)
17
17
open import Relation.Binary.PropositionalEquality.Core as PropEq
18
18
using (_≡_; refl; sym; cong; cong₂)
19
+ open import Relation.Binary.PropositionalEquality.Properties
20
+ using (module ≡-Reasoning )
19
21
open import Relation.Binary.Construct.Closure.ReflexiveTransitive
20
22
using (Star; ε; _◅_; _▻_)
21
- open PropEq. ≡-Reasoning
23
+ open ≡-Reasoning
22
24
open import Level using (Level; _⊔_)
23
25
open import Relation.Unary using (Pred)
24
26
Original file line number Diff line number Diff line change @@ -31,8 +31,8 @@ open import Relation.Nullary
31
31
open import Relation.Nullary.Decidable using (dec-true; dec-false)
32
32
open import Relation.Binary.PropositionalEquality.Core as PropEq
33
33
using (_≡_; _≢_; refl; cong)
34
- open PropEq.≡-Reasoning
35
34
import Relation.Binary.PropositionalEquality.Properties as PropEq
35
+ open PropEq.≡-Reasoning
36
36
37
37
private
38
38
open module D = DecSetoid D
Original file line number Diff line number Diff line change 10
10
11
11
module Data.List.Relation.Binary.Sublist.Propositional.Example.UniqueBoundVariables (Base : Set ) where
12
12
13
- open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; sym; cong; subst; module ≡-Reasoning )
13
+ open import Relation.Binary.PropositionalEquality
14
+ using (_≡_; refl; sym; cong; subst; module ≡-Reasoning )
14
15
open ≡-Reasoning
15
16
16
17
open import Data.List.Base using (List; []; _∷_; [_])
Original file line number Diff line number Diff line change @@ -16,7 +16,9 @@ open import Data.List.Relation.Ternary.Interleaving hiding (map)
16
16
open import Function.Base using (_$_)
17
17
open import Relation.Binary.Core using (REL)
18
18
open import Relation.Binary.PropositionalEquality.Core
19
- using (_≡_; refl; sym; cong; module ≡-Reasoning )
19
+ using (_≡_; refl; sym; cong)
20
+ open import Relation.Binary.PropositionalEquality.Properties
21
+ using (module ≡-Reasoning )
20
22
open ≡-Reasoning
21
23
22
24
------------------------------------------------------------------------
Original file line number Diff line number Diff line change @@ -43,6 +43,8 @@ open import Relation.Binary.Core using (Rel; REL)
43
43
open import Relation.Binary.Definitions as B
44
44
open import Relation.Binary.PropositionalEquality.Core as P
45
45
using (_≡_; refl)
46
+ open import Relation.Binary.PropositionalEquality.Properties
47
+ using (module ≡-Reasoning )
46
48
open import Relation.Unary as U
47
49
using (Pred; _⟨×⟩_; _⟨→⟩_) renaming (_⊆_ to _⋐_)
48
50
open import Relation.Nullary using (¬_; _because_; does; ofʸ; ofⁿ; yes; no)
@@ -219,7 +221,7 @@ Any-×⁻ pq with Prod.map₂ (Prod.map₂ find) (find pq)
219
221
(Any P xs × Any Q ys) ↔ Any (λ x → Any (λ y → P x × Q y) ys) xs
220
222
×↔ {P = P} {Q = Q} {xs} {ys} = mk↔ₛ′ Any-×⁺ Any-×⁻ to∘from from∘to
221
223
where
222
- open P. ≡-Reasoning
224
+ open ≡-Reasoning
223
225
224
226
from∘to : ∀ pq → Any-×⁻ (Any-×⁺ pq) ≡ pq
225
227
from∘to (p , q) =
You can’t perform that action at this time.
0 commit comments