src/ZF/Rel.ML
changeset 5147 825877190618
parent 5137 60205b0de9b9
child 5321 f8848433d240
equal deleted inserted replaced
5146:1ea751ae62b2 5147:825877190618
     1 (*  Title:      ZF/Rel.ML
     1 (*  Title:      ZF/Rel.ML
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1994  University of Cambridge
     4     Copyright   1994  University of Cambridge
     5 
     5 
     6 For Rel.thy.  Relations in Zermelo-Fraenkel Set Theory 
     6 Relations in Zermelo-Fraenkel Set Theory 
     7 *)
     7 *)
     8 
     8 
     9 open Rel;
     9 open Rel;
    10 
    10 
    11 (*** Some properties of relations -- useful? ***)
    11 (*** Some properties of relations -- useful? ***)
    47 qed "antisymE";
    47 qed "antisymE";
    48 
    48 
    49 (* transitivity *)
    49 (* transitivity *)
    50 
    50 
    51 Goalw [trans_def]
    51 Goalw [trans_def]
    52     "!!r. [| trans(r);  <a,b>:r;  <b,c>:r |] ==> <a,c>:r";
    52     "[| trans(r);  <a,b>:r;  <b,c>:r |] ==> <a,c>:r";
    53 by (Blast_tac 1);
    53 by (Blast_tac 1);
    54 qed "transD";
    54 qed "transD";
    55 
    55 
    56 Goalw [trans_on_def]
    56 Goalw [trans_on_def]
    57     "!!r. [| trans[A](r);  <a,b>:r;  <b,c>:r;  a:A;  b:A;  c:A |] ==> <a,c>:r";
    57     "[| trans[A](r);  <a,b>:r;  <b,c>:r;  a:A;  b:A;  c:A |] ==> <a,c>:r";
    58 by (Blast_tac 1);
    58 by (Blast_tac 1);
    59 qed "trans_onD";
    59 qed "trans_onD";
    60 
    60