comparison src/LEMC.agda @ 440:d1c9f5ae5d0a

give up this generic filter definition
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Tue, 01 Mar 2022 14:31:31 +0900
parents a5f8084b8368
children 55ab5de1ae02
comparison
equal deleted inserted replaced
439:fdcbf23ba2f9 440:d1c9f5ae5d0a
129 -- 129 --
130 -- axiom regurality from ε-induction (using axiom of choice above) 130 -- axiom regurality from ε-induction (using axiom of choice above)
131 -- 131 --
132 -- from https://math.stackexchange.com/questions/2973777/is-it-possible-to-prove-regularity-with-transfinite-induction-only 132 -- from https://math.stackexchange.com/questions/2973777/is-it-possible-to-prove-regularity-with-transfinite-induction-only
133 -- 133 --
134 -- FIXME : don't use HOD make this level n, so we can remove ε-induction1
135 record Minimal (x : HOD) : Set (suc n) where 134 record Minimal (x : HOD) : Set (suc n) where
136 field 135 field
137 min : HOD 136 min : HOD
138 x∋min : x ∋ min 137 x∋min : x ∋ min
139 min-empty : (y : HOD ) → ¬ ( min ∋ y) ∧ (x ∋ y) 138 min-empty : (y : HOD ) → ¬ ( min ∋ y) ∧ (x ∋ y)