src/HOL/ex/Tuple.thy
changeset 17388 495c799df31d
parent 16417 9bc16273c2d4
equal deleted inserted replaced
17387:40ce48cc45f7 17388:495c799df31d
     1 (*  Title:      HOL/ex/Tuple.thy
     1 (*  Title:      HOL/ex/Tuple.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Markus Wenzel, TU Muenchen
     3     Author:     Markus Wenzel, TU Muenchen
     4 
       
     5 Properly nested products (see also theory Prod).
       
     6 
       
     7 Unquestionably, this should be used as the standard representation of
       
     8 tuples in HOL, but it breaks many existing theories!
       
     9 *)
     4 *)
    10 
     5 
    11 header {* Properly nested products *}
     6 header {* Properly nested products *}
    12 
     7 
    13 theory Tuple imports HOL begin
     8 theory Tuple imports HOL begin