2014-07-27 20:18:33 +00:00
|
|
|
|
--- Copyright (c) 2014 Jeremy Avigad. All rights reserved.
|
|
|
|
|
--- Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
|
--- Author: Jeremy Avigad, Leonardo de Moura
|
|
|
|
|
import logic funext bool
|
|
|
|
|
using eq_proofs bool
|
|
|
|
|
|
|
|
|
|
namespace set
|
|
|
|
|
definition set (T : Type) := T → bool
|
2014-07-29 02:58:57 +00:00
|
|
|
|
definition mem {T : Type} (x : T) (s : set T) := (s x) = tt
|
2014-07-27 20:18:33 +00:00
|
|
|
|
infix `∈`:50 := mem
|
|
|
|
|
|
|
|
|
|
section
|
|
|
|
|
parameter {T : Type}
|
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
definition empty : set T := λx, ff
|
2014-07-27 20:18:33 +00:00
|
|
|
|
notation `∅`:max := empty
|
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem mem_empty (x : T) : ¬ (x ∈ ∅) :=
|
|
|
|
|
assume H : x ∈ ∅, absurd H ff_ne_tt
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
definition univ : set T := λx, tt
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem mem_univ (x : T) : x ∈ univ := refl _
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
|
|
|
|
definition inter (A B : set T) : set T := λx, A x && B x
|
|
|
|
|
infixl `∩`:70 := inter
|
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem mem_inter (x : T) (A B : set T) : x ∈ A ∩ B ↔ (x ∈ A ∧ x ∈ B) :=
|
|
|
|
|
iff_intro
|
|
|
|
|
(assume H, and_intro (band_eq_tt_elim_left H) (band_eq_tt_elim_right H))
|
|
|
|
|
(assume H,
|
|
|
|
|
have e1 : A x = tt, from and_elim_left H,
|
|
|
|
|
have e2 : B x = tt, from and_elim_right H,
|
|
|
|
|
show A x && B x = tt, from e1⁻¹ ▸ e2⁻¹ ▸ band_tt_left tt)
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem inter_comm (A B : set T) : A ∩ B = B ∩ A :=
|
|
|
|
|
funext (λx, band_comm (A x) (B x))
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem inter_assoc (A B C : set T) : (A ∩ B) ∩ C = A ∩ (B ∩ C) :=
|
|
|
|
|
funext (λx, band_assoc (A x) (B x) (C x))
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
|
|
|
|
definition union (A B : set T) : set T := λx, A x || B x
|
|
|
|
|
infixl `∪`:65 := union
|
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem mem_union (x : T) (A B : set T) : x ∈ A ∪ B ↔ (x ∈ A ∨ x ∈ B) :=
|
|
|
|
|
iff_intro
|
|
|
|
|
(assume H, bor_to_or H)
|
|
|
|
|
(assume H, or_elim H
|
|
|
|
|
(assume Ha : A x = tt,
|
|
|
|
|
show A x || B x = tt, from Ha⁻¹ ▸ bor_tt_left (B x))
|
|
|
|
|
(assume Hb : B x = tt,
|
|
|
|
|
show A x || B x = tt, from Hb⁻¹ ▸ bor_tt_right (A x)))
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem union_comm (A B : set T) : A ∪ B = B ∪ A :=
|
|
|
|
|
funext (λx, bor_comm (A x) (B x))
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
2014-07-29 02:58:57 +00:00
|
|
|
|
theorem union_assoc (A B C : set T) : (A ∪ B) ∪ C = A ∪ (B ∪ C) :=
|
|
|
|
|
funext (λx, bor_assoc (A x) (B x) (C x))
|
2014-07-27 20:18:33 +00:00
|
|
|
|
|
|
|
|
|
end
|
|
|
|
|
end
|