src/ZF/upair.thy
author wenzelm
Thu, 07 Sep 2000 21:12:49 +0200
changeset 9907 473a6604da94
parent 9570 e16e168984e1
child 11770 b6bb7a853dd2
permissions -rw-r--r--
tuned ML code (the_context, bind_thms(s));
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 124
diff changeset
     1
(*  Title:      ZF/upair.thy
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 124
diff changeset
     2
    ID:         $Id$
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 124
diff changeset
     3
    Author:     Lawrence C Paulson and Martin D Coen, CU Computer Laboratory
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 124
diff changeset
     4
    Copyright   1993  University of Cambridge
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 124
diff changeset
     5
*)
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 124
diff changeset
     6
9570
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents: 6153
diff changeset
     7
theory upair = ZF
e16e168984e1 installation of cancellation simprocs for the integers
paulson
parents: 6153
diff changeset
     8
files "Tools/typechk":
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 3924
diff changeset
     9
9907
473a6604da94 tuned ML code (the_context, bind_thms(s));
wenzelm
parents: 9570
diff changeset
    10
setup TypeCheck.setup
473a6604da94 tuned ML code (the_context, bind_thms(s));
wenzelm
parents: 9570
diff changeset
    11
setup Rulify.setup
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 3924
diff changeset
    12
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 3924
diff changeset
    13
end