src/ZF/Cardinal.ML
changeset 3891 3a05a7f549bd
parent 3840 e0baea4d485a
child 3894 8b9f0bc6dc1a
equal deleted inserted replaced
3890:2a2a86b57fed 3891:3a05a7f549bd
   752 by (dres_inst_tac [("x", "Z")] spec 1);
   752 by (dres_inst_tac [("x", "Z")] spec 1);
   753 by (Blast.depth_tac (!claset) 4 1);
   753 by (Blast.depth_tac (!claset) 4 1);
   754 qed "nat_wf_on_converse_Memrel";
   754 qed "nat_wf_on_converse_Memrel";
   755 
   755 
   756 goal Cardinal.thy "!!n. n:nat ==> well_ord(n,converse(Memrel(n)))";
   756 goal Cardinal.thy "!!n. n:nat ==> well_ord(n,converse(Memrel(n)))";
   757 by (forward_tac [Ord_nat RS Ord_in_Ord RS well_ord_Memrel] 1);
   757 by (forward_tac [transfer thy Ord_nat RS Ord_in_Ord RS well_ord_Memre] 1);
   758 by (rewtac well_ord_def);
   758 by (rewtac well_ord_def);
   759 by (blast_tac (!claset addSIs [tot_ord_converse, 
   759 by (blast_tac (!claset addSIs [tot_ord_converse, 
   760 			       nat_wf_on_converse_Memrel]) 1);
   760 			       nat_wf_on_converse_Memrel]) 1);
   761 qed "nat_well_ord_converse_Memrel";
   761 qed "nat_well_ord_converse_Memrel";
   762 
   762