Skip to content

Commit

Permalink
chore(category): rename to control (#2516)
Browse files Browse the repository at this point in the history
This is parallel to leanprover-community/lean#202 for community Lean (now merged).

It seems the changes are actually completely independent; this compiles against current community Lean, and that PR. (I'm surprised, but I guess it's just that everything is in the root namespace, and in `init/`.)

This PR anticipates then renaming `category_theory/` to `category/`.

Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
semorrison and semorrison committed Apr 28, 2020
1 parent c435b1c commit d12db89
Show file tree
Hide file tree
Showing 35 changed files with 34 additions and 34 deletions.
2 changes: 0 additions & 2 deletions src/category/traversable/default.lean

This file was deleted.

2 changes: 1 addition & 1 deletion src/category_theory/core.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import category_theory.groupoid
import category.equiv_functor
import control.equiv_functor
import category_theory.types

namespace category_theory
Expand Down
Expand Up @@ -5,7 +5,7 @@ Author: Simon Hudon
Instances for identity and composition functors
-/
import category.functor
import control.functor

universe variables u v w

Expand Down
File renamed without changes.
File renamed without changes.
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: Simon Hudon
-/
import category.bifunctor
import control.bifunctor

/-!
# Bitraversable type class
Expand Down
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2019 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author(s): Simon Hudon
-/
import category.bitraversable.lemmas
import category.traversable.lemmas
import control.bitraversable.lemmas
import control.traversable.lemmas

/-!
# bitraversable instances
Expand Down
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author(s): Simon Hudon
-/
import category.bitraversable.basic
import control.bitraversable.basic

/-!
# Bitraversable Lemmas
Expand Down
File renamed without changes.
File renamed without changes.
4 changes: 2 additions & 2 deletions src/category/fold.lean → src/control/fold.lean
Expand Up @@ -43,8 +43,8 @@ but the author cannot think of instances of `foldable` that are not also
-/
import algebra.free_monoid
import algebra.opposites
import category.traversable.instances
import category.traversable.lemmas
import control.traversable.instances
import control.traversable.lemmas
import category_theory.category
import category_theory.endomorphism
import category_theory.types
Expand Down
File renamed without changes.
File renamed without changes.
Expand Up @@ -7,7 +7,7 @@ Monad encapsulating continuation passing programming style, similar to
Haskell's `Cont`, `ContT` and `MonadCont`:
<http://hackage.haskell.org/package/mtl-2.2.2/docs/Control-Monad-Cont.html>
-/
import category.monad.writer
import control.monad.writer

universes u v w

Expand Down
Expand Up @@ -5,7 +5,7 @@ Authors: Simon Hudon
The writer monad transformer for passing immutable state.
-/
import category.monad.basic
import control.monad.basic
universes u v w

structure writer_t (ω : Type u) (m : Type u → Type v) (α : Type u) : Type (max u v) :=
Expand Down
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: Simon Hudon
-/
import category.applicative
import control.applicative

/-!
# Traversable type class
Expand Down
2 changes: 2 additions & 0 deletions src/control/traversable/default.lean
@@ -0,0 +1,2 @@
import control.traversable.instances
import control.traversable.lemmas
Expand Up @@ -5,7 +5,7 @@ Author: Simon Hudon
Automation to construct `traversable` instances
-/
import category.traversable.lemmas
import control.traversable.lemmas
import data.list.basic

namespace tactic.interactive
Expand Down
Expand Up @@ -6,7 +6,7 @@ Authors: Simon Hudon
Transferring `traversable` instances using isomorphisms.
-/
import data.equiv.basic
import category.traversable.lemmas
import control.traversable.lemmas

universes u

Expand Down
File renamed without changes.
Expand Up @@ -12,7 +12,7 @@ Inspired by:
In Journal of Functional Programming. Vol. 19. No. 3&4. Pages 377−402. 2009.
<http://www.cs.ox.ac.uk/jeremy.gibbons/publications/iterator.pdf>
-/
import category.traversable.basic
import control.traversable.basic

universe variables u

Expand Down
2 changes: 1 addition & 1 deletion src/data/array/lemmas.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2017 Microsoft Corporation. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Leonardo de Moura, Mario Carneiro
-/
import category.traversable.equiv
import control.traversable.equiv
import data.vector2

universes u v w
Expand Down
2 changes: 1 addition & 1 deletion src/data/buffer/basic.lean
Expand Up @@ -7,7 +7,7 @@ Traversable instance for buffers.
-/
import data.buffer
import data.array.lemmas
import category.traversable.instances
import control.traversable.instances

namespace buffer

Expand Down
4 changes: 2 additions & 2 deletions src/data/dlist/instances.lean
Expand Up @@ -6,8 +6,8 @@ Authors: Simon Hudon
Traversable instance for dlists.
-/
import data.dlist
import category.traversable.equiv
import category.traversable.instances
import control.traversable.equiv
import control.traversable.instances

namespace dlist

Expand Down
2 changes: 1 addition & 1 deletion src/data/equiv/functor.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johan Commelin, Simon Hudon, Scott Morrison
-/
import data.equiv.basic
import category.bifunctor
import control.bifunctor

/-!
# Functor and bifunctors can be applied to `equiv`s.
Expand Down
2 changes: 1 addition & 1 deletion src/data/fin_enum.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author(s): Simon Hudon
-/
import category.monad.basic
import control.monad.basic
import data.fintype.basic

/-!
Expand Down
4 changes: 2 additions & 2 deletions src/data/lazy_list2.lean
Expand Up @@ -5,8 +5,8 @@ Authors: Simon Hudon
Traversable instance for lazy_lists.
-/
import category.traversable.equiv
import category.traversable.instances
import control.traversable.equiv
import control.traversable.instances
import data.lazy_list

universes u
Expand Down
4 changes: 2 additions & 2 deletions src/data/multiset.lean
Expand Up @@ -10,8 +10,8 @@ import data.list.intervals
import data.list.antidiagonal
import data.string.basic
import algebra.group_power
import category.traversable.lemmas
import category.traversable.instances
import control.traversable.lemmas
import control.traversable.instances

open list subtype nat

Expand Down
2 changes: 1 addition & 1 deletion src/tactic/converter/old_conv.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Leonardo de Moura
Converter monad for building simplifiers.
-/
import category.basic
import control.basic
open tactic

meta structure old_conv_result (α : Type) :=
Expand Down
2 changes: 1 addition & 1 deletion src/tactic/core.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro, Simon Hudon, Scott Morrison, Keeley Hoek
-/
import data.dlist.basic
import category.basic
import control.basic
import meta.expr
import meta.rb_map
import data.bool
Expand Down
2 changes: 1 addition & 1 deletion src/tactic/equiv_rw.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import category.equiv_functor
import control.equiv_functor

/-!
# The `equiv_rw` tactic transports goals or hypotheses along equivalences.
Expand Down
4 changes: 2 additions & 2 deletions src/tactic/monotonicity/interactive.lean
Expand Up @@ -4,8 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Author: Simon Hudon
-/
import tactic.monotonicity.basic
import category.traversable
import category.traversable.derive
import control.traversable
import control.traversable.derive
import data.dlist

variables {a b c p : Prop}
Expand Down
2 changes: 1 addition & 1 deletion src/tactic/squeeze.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2019 Simon Hudon. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: Simon Hudon
-/
import category.traversable.basic
import control.traversable.basic
import tactic.simpa

open interactive interactive.types lean.parser
Expand Down
2 changes: 1 addition & 1 deletion test/equiv_rw.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Scott Morrison
-/
import tactic.equiv_rw
import category.equiv_functor.instances -- these make equiv_rw more powerful!
import control.equiv_functor.instances -- these make equiv_rw more powerful!

-- Uncomment this line to observe the steps of constructing appropriate equivalences.
-- set_option trace.equiv_rw_type true
Expand Down
2 changes: 1 addition & 1 deletion test/traversable.lean
@@ -1,4 +1,4 @@
import category.traversable.derive
import control.traversable.derive
import tactic

universes u
Expand Down

0 comments on commit d12db89

Please sign in to comment.