Skip to content

Commit

Permalink
introduce top level dir order: move algebra.order and content of …
Browse files Browse the repository at this point in the history
…`algebra.lattice`
  • Loading branch information
johoelzl committed Aug 11, 2017
1 parent 218c1dd commit e27aae8
Show file tree
Hide file tree
Showing 17 changed files with 15 additions and 35 deletions.
20 changes: 0 additions & 20 deletions algebra/lattice/README.md

This file was deleted.

3 changes: 0 additions & 3 deletions algebra/lattice/default.lean

This file was deleted.

2 changes: 1 addition & 1 deletion data/set/lattice.lean
Expand Up @@ -6,7 +6,7 @@ Authors Jeremy Avigad, Leonardo de Moura, Johannes Hölzl
-- QUESTION: can make the first argument in ∀ x ∈ a, ... implicit?
-/
import logic.basic data.set.basic
import algebra.lattice algebra.order algebra.lattice.complete_boolean_algebra category.basic
import order.complete_boolean_algebra category.basic
import tactic.finish

open function tactic set lattice auto
Expand Down
File renamed without changes.
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl
Type class hierarchy for Boolean algebras.
-/
import algebra.lattice.bounded_lattice
import order.bounded_lattice

set_option old_structure_cmd true

Expand Down
Expand Up @@ -8,7 +8,7 @@ Defines bounded lattice type class hierarchy.
Includes the Prop and fun instances.
-/

import algebra.lattice.basic
import order.lattice

set_option old_structure_cmd true

Expand Down
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl
Theory of complete Boolean algebras.
-/
import algebra.lattice.complete_lattice algebra.lattice.boolean_algebra data.set.basic
import order.complete_lattice order.boolean_algebra data.set.basic

set_option old_structure_cmd true

Expand Down
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl
Theory of complete lattices.
-/
import algebra.lattice.bounded_lattice data.set.basic
import order.bounded_lattice data.set.basic

set_option old_structure_cmd true

Expand Down
3 changes: 3 additions & 0 deletions order/default.lean
@@ -0,0 +1,3 @@
import order.basic order.lattice order.bounded_lattice
order.boolean_algebra order.complete_lattice

2 changes: 1 addition & 1 deletion algebra/lattice/filter.lean → order/filter.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl
Theory of filters on sets.
-/
import algebra.lattice.complete_lattice data.set algebra.lattice.zorn
import order.complete_lattice data.set order.zorn
open lattice set

universes u v w x y
Expand Down
Expand Up @@ -6,7 +6,7 @@ Authors: Johannes Hölzl
Fixed point construction on complete lattices.
-/

import algebra.lattice.complete_lattice
import order.complete_lattice

universes u v w
variables {α : Type u} {β : Type v} {γ : Type w}
Expand Down
2 changes: 1 addition & 1 deletion algebra/lattice/basic.lean → order/lattice.lean
Expand Up @@ -6,7 +6,7 @@ Authors: Johannes Hölzl
Defines the inf/sup (semi)-lattice with optionally top/bot type class hierarchy.
-/

import algebra.order tactic.finish
import order.basic tactic.finish
open auto

set_option old_structure_cmd true
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion tactic/converter/binders.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Johannes Hölzl
Binder elimination
-/
import algebra.lattice tactic.converter.old_conv
import order tactic.converter.old_conv

namespace old_conv
open tactic monad
Expand Down
2 changes: 1 addition & 1 deletion topology/real.lean
Expand Up @@ -22,7 +22,7 @@ generalizations:
-/

import topology.uniform_space data.rat algebra.field algebra.order
import topology.uniform_space data.rat algebra.field
noncomputable theory
open classical set lattice filter
local attribute [instance] decidable_inhabited prop_decidable
Expand Down
2 changes: 1 addition & 1 deletion topology/topological_space.lean
Expand Up @@ -10,7 +10,7 @@ Parts of the formalization is based on the books:
I. M. James: Topologies and Uniformities
A major difference is that this formalization is heavily based on the filter library.
-/
import algebra.lattice.filter
import order.filter
open set filter lattice classical
local attribute [instance] decidable_inhabited prop_decidable

Expand Down
2 changes: 1 addition & 1 deletion topology/uniform_space.lean
Expand Up @@ -27,7 +27,7 @@ The formalization is mostly based on the books:
I. M. James: Topologies and Uniformities
A major difference is that this formalization is heavily based on the filter library.
-/
import algebra.lattice.filter topology.topological_space topology.continuity
import order.filter topology.topological_space topology.continuity
open set lattice filter classical
local attribute [instance] decidable_inhabited prop_decidable

Expand Down

0 comments on commit e27aae8

Please sign in to comment.