diff src/LEMC.agda @ 1096:55ab5de1ae02

recovery
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Fri, 23 Dec 2022 12:54:05 +0900
parents d1c9f5ae5d0a
children e086a266c6b7
line wrap: on
line diff
--- a/src/LEMC.agda	Thu Dec 22 15:10:31 2022 +0900
+++ b/src/LEMC.agda	Fri Dec 23 12:54:05 2022 +0900
@@ -32,8 +32,6 @@
 
 open HOD
 
-open _⊆_
-
 decp : ( p : Set n ) → Dec p   -- assuming axiom of choice    
 decp  p with p∨¬p p
 decp  p | case1 x = yes x
@@ -50,8 +48,8 @@
 ... | no ¬p = ⊥-elim ( notnot ¬p )
 
 power→⊆ :  ( A t : HOD) → Power A ∋ t → t ⊆ A
-power→⊆ A t  PA∋t = record { incl = λ {x} t∋x → double-neg-eilm (λ not → t1 t∋x (λ x → not x) ) } where
-   t1 : {x : HOD }  → t ∋ x → ¬ ¬ (A ∋ x)
+power→⊆ A t  PA∋t t∋x = subst (λ k → odef A k ) &iso ( t1 (subst (λ k → odef t k ) (sym &iso) t∋x))  where
+   t1 : {x : HOD }  → t ∋ x → A ∋ x
    t1 = power→ A t PA∋t
 
 --- With assuption of HOD is ordered,  p ∨ ( ¬ p ) <=> axiom of choice