Skip to content

Commit

Permalink
Refactor directory names
Browse files Browse the repository at this point in the history
Signed-off-by: zeramorphic <[email protected]>
  • Loading branch information
zeramorphic committed Dec 3, 2024
1 parent dc51a7e commit 6fdc87c
Show file tree
Hide file tree
Showing 16 changed files with 29 additions and 29 deletions.
24 changes: 12 additions & 12 deletions ConNF.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,25 +8,13 @@ import ConNF.Basic.Set
import ConNF.Basic.Transfer
import ConNF.Basic.WellOrder
import ConNF.Construction.Code
import ConNF.Construction.ConstructHypothesis
import ConNF.Construction.ConstructMotive
import ConNF.Construction.Externalise
import ConNF.Construction.Hailperin
import ConNF.Construction.InductionStatement
import ConNF.Construction.NewModelData
import ConNF.Construction.RaiseStrong
import ConNF.Construction.Result
import ConNF.Construction.RunInduction
import ConNF.Construction.TTT
import ConNF.Counting.BaseCoding
import ConNF.Counting.BaseCounting
import ConNF.Counting.CodingFunction
import ConNF.Counting.Conclusions
import ConNF.Counting.CountSupportOrbit
import ConNF.Counting.Recode
import ConNF.Counting.SMulSpec
import ConNF.Counting.Spec
import ConNF.Counting.SpecSame
import ConNF.Counting.Strong
import ConNF.Counting.Twist
import ConNF.FOA.BaseAction
Expand All @@ -38,6 +26,15 @@ import ConNF.FOA.StrAction
import ConNF.FOA.StrActionFOA
import ConNF.FOA.StrApprox
import ConNF.FOA.StrApproxFOA
import ConNF.Model.ConstructHypothesis
import ConNF.Model.ConstructMotive
import ConNF.Model.Externalise
import ConNF.Model.Hailperin
import ConNF.Model.InductionStatement
import ConNF.Model.RaiseStrong
import ConNF.Model.Result
import ConNF.Model.RunInduction
import ConNF.Model.TTT
import ConNF.Setup.Atom
import ConNF.Setup.BasePerm
import ConNF.Setup.BasePositions
Expand All @@ -59,3 +56,6 @@ import ConNF.Setup.StrSet
import ConNF.Setup.Support
import ConNF.Setup.Tree
import ConNF.Setup.TypeIndex
import ConNF.Strong.SMulSpec
import ConNF.Strong.Spec
import ConNF.Strong.SpecSame
2 changes: 1 addition & 1 deletion ConNF/Counting/BaseCoding.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Counting.SpecSame
import ConNF.Strong.SpecSame

/-!
# Coding the base type
Expand Down
4 changes: 2 additions & 2 deletions ConNF/Counting/CountSupportOrbit.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
import ConNF.Counting.SMulSpec
import ConNF.Counting.SpecSame
import ConNF.Strong.SMulSpec
import ConNF.Strong.SpecSame

/-!
# Counting support orbits
Expand Down
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.ConstructMotive
import ConNF.Model.ConstructMotive

/-!
# New file
Expand Down
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.InductionStatement
import ConNF.Model.InductionStatement
import ConNF.Construction.NewModelData
import ConNF.Counting.Conclusions

Expand Down
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.RunInduction
import ConNF.Model.RunInduction

/-!
# Externalisation
Expand Down
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.TTT
import ConNF.Model.TTT

/-!
# New file
Expand Down
File renamed without changes.
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.Externalise
import ConNF.Model.Externalise

/-!
# New file
Expand Down
2 changes: 1 addition & 1 deletion ConNF/Construction/Result.lean → ConNF/Model/Result.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.Hailperin
import ConNF.Model.Hailperin

/-!
# New file
Expand Down
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
import ConNF.Basic.InductiveConstruction
import ConNF.Construction.ConstructHypothesis
import ConNF.Model.ConstructHypothesis

/-!
# New file
Expand Down
2 changes: 1 addition & 1 deletion ConNF/Construction/TTT.lean → ConNF/Model/TTT.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Construction.RaiseStrong
import ConNF.Model.RaiseStrong

/-!
# New file
Expand Down
Original file line number Diff line number Diff line change
@@ -1,4 +1,4 @@
import ConNF.Counting.Spec
import ConNF.Strong.Spec

/-!
# Action on specifications
Expand Down
File renamed without changes.
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
import ConNF.FOA.StrActionFOA
import ConNF.Counting.Strong
import ConNF.Counting.Spec
import ConNF.Strong.Spec

/-!
# Supports with the same specification
Expand Down
8 changes: 4 additions & 4 deletions DependencyGraph.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,7 @@ elab "#deptree " : command => do
for (gp, _) in groups imports do
h.write ("subgraph cluster_" ++ nameCode gp ++ " {\n").toUTF8
for (k, v) in imports do
if (`ConNF).isPrefixOf k && group k = gp then do
if (`ConNF).isPrefixOf k && k != `ConNF && group k = gp then do
printDeps₁ k v (fun s => h.write s.toUTF8)
h.write ("label = \"" ++ gp.toString ++ "\";\n").toUTF8
h.write ("margin = 32;\n").toUTF8
Expand All @@ -52,7 +52,7 @@ elab "#deptree " : command => do
h.write ("color = cyan4;\n").toUTF8
h.write "}\n".toUTF8
for (k, v) in imports do
if (`ConNF).isPrefixOf k then do
if (`ConNF).isPrefixOf k && k != `ConNF then do
printDeps₂ k v (fun s => h.write s.toUTF8)
h.write "}\n".toUTF8

Expand All @@ -77,10 +77,10 @@ def allFiles (env : Environment) : List Name :=
(toString · < toString ·)

def allDecls (env : Environment) : Elab.Command.CommandElabM NameSet :=
(fun l => RBTree.ofList (l.map (fun a => a.toList)).join) <$>
(fun l => RBTree.ofList (l.map (fun a => a.toList)).flatten) <$>
(mapM allDeclsIn (allFiles env))

/-- `#index` computes an index of the declations in the project and saves it to `index.csv`. -/
/-- `#index` computes an index of the declarations in the project and saves it to `index.csv`. -/
elab "#index " : command => do
let env ← getEnv
let allDecls ← allDecls env
Expand Down

0 comments on commit 6fdc87c

Please sign in to comment.