2014-07-27 19:17:38 +00:00
|
|
|
import logic
|
2014-09-05 01:41:06 +00:00
|
|
|
open eq
|
2014-09-17 21:39:05 +00:00
|
|
|
definition subsets (P : Type) := P → Prop.
|
2014-07-27 19:17:38 +00:00
|
|
|
|
2015-04-22 02:33:21 +00:00
|
|
|
section
|
2014-07-27 19:17:38 +00:00
|
|
|
|
|
|
|
hypothesis A : Type.
|
|
|
|
|
|
|
|
hypothesis r : A → subsets A.
|
|
|
|
|
|
|
|
hypothesis i : subsets A → A.
|
|
|
|
|
|
|
|
hypothesis retract {P : subsets A} {a : A} : r (i P) a = P a.
|
|
|
|
|
|
|
|
definition delta (a:A) : Prop := ¬ (r a a).
|
|
|
|
|
2015-04-22 02:33:21 +00:00
|
|
|
local notation `δ` := delta.
|
2014-07-27 19:17:38 +00:00
|
|
|
|
|
|
|
theorem delta_aux : ¬ (δ (i delta))
|
|
|
|
:= assume H : δ (i delta),
|
|
|
|
H (subst (symm retract) H).
|
|
|
|
|
2014-08-08 00:08:59 +00:00
|
|
|
check delta_aux.
|
|
|
|
|
2014-09-05 01:41:06 +00:00
|
|
|
end
|