File tree Expand file tree Collapse file tree 1 file changed +10
-5
lines changed Expand file tree Collapse file tree 1 file changed +10
-5
lines changed Original file line number Diff line number Diff line change @@ -618,14 +618,19 @@ fun NOT_EQ_SYM th =
618
618
* *
619
619
* [TFM 90.05.08] *
620
620
* --------------------------------------------------------------------------*)
621
-
622
621
local
623
- val Fth = ASSUME F
622
+ val eq_F = el 4 $ CONJUNCTS $ SPEC_ALL EQ_CLAUSES;
623
+ val eq_F' = SYM eq_F
624
+ val t = (dest_neg o fst o dest_eq) (concl eq_F')
625
+ (* ∀t. ¬t ⇔ (t ⇔ F) *)
626
+ val eq_F' = GEN t eq_F'
624
627
in
625
628
fun EQF_INTRO th =
626
- IMP_ANTISYM_RULE (NOT_ELIM th)
627
- (DISCH F (CONTR (dest_neg (concl th)) Fth))
628
- handle HOL_ERR _ => raise ERR " EQF_INTRO" " "
629
+ let val t' = dest_neg (concl th)
630
+ in
631
+ EQ_MP (SPEC t' eq_F') th
632
+ end
633
+ handle HOL_ERR _ => raise ERR " EQF_INTRO" " "
629
634
end
630
635
631
636
(* --------------------------------------------------------------------------*
You can’t perform that action at this time.
0 commit comments