File tree Expand file tree Collapse file tree 5 files changed +6
-6
lines changed Expand file tree Collapse file tree 5 files changed +6
-6
lines changed Original file line number Diff line number Diff line change @@ -383,8 +383,8 @@ New modules
383
383
Reflection.Meta
384
384
Reflection.Name
385
385
Reflection.Pattern
386
- Reflection.TCMonadSyntax
387
386
Reflection.Term
387
+ Reflection.TypeChecking.MonadSyntax
388
388
```
389
389
390
390
* New tactics for monoid and ring solvers. See ` README.Tactic.MonoidSolver/RingSolver ` for details
Original file line number Diff line number Diff line change @@ -71,7 +71,7 @@ open Builtin public
71
71
72
72
-- Standard monad operators
73
73
74
- open import Reflection.TCMonadSyntax public
74
+ open import Reflection.TypeChecking.MonadSyntax public
75
75
using (_>>=_; _>>_)
76
76
77
77
newMeta : Type → TC Term
Original file line number Diff line number Diff line change 6
6
7
7
{-# OPTIONS --without-K --safe #-}
8
8
9
- module Reflection.TCMonadSyntax where
9
+ module Reflection.TypeChecking.MonadSyntax where
10
10
11
11
open import Agda.Builtin.Reflection
12
12
open import Level using (Level)
Original file line number Diff line number Diff line change @@ -82,9 +82,9 @@ open import Data.Nat as ℕ using (ℕ; suc; zero)
82
82
open import Data.Product as Product using (_×_; _,_)
83
83
84
84
open import Agda.Builtin.Reflection
85
- open import Reflection.TCMonadSyntax
86
- open import Reflection.Term using (getName; _⋯⟅∷⟆_)
87
85
open import Reflection.Argument
86
+ open import Reflection.Term using (getName; _⋯⟅∷⟆_)
87
+ open import Reflection.TypeChecking.MonadSyntax
88
88
89
89
import Relation.Binary.Reasoning.Setoid as SetoidReasoning
90
90
Original file line number Diff line number Diff line change @@ -23,9 +23,9 @@ open import Data.Unit using (⊤)
23
23
open import Data.String using (String)
24
24
open import Data.Product using (_,_)
25
25
open import Function
26
- open import Reflection.TCMonadSyntax
27
26
open import Reflection.Argument
28
27
open import Reflection.Term
28
+ open import Reflection.TypeChecking.MonadSyntax
29
29
30
30
open import Tactic.RingSolver.NonReflective renaming (solve to solve-fn)
31
31
open import Tactic.RingSolver.Core.AlmostCommutativeRing
You can’t perform that action at this time.
0 commit comments