src/ZF/CardinalArith.thy
changeset 13328 703de709a64b
parent 13269 3ba9be497c33
child 13356 c9cfe1638bf2
--- a/src/ZF/CardinalArith.thy	Tue Jul 09 23:03:21 2002 +0200
+++ b/src/ZF/CardinalArith.thy	Tue Jul 09 23:05:26 2002 +0200
@@ -3,13 +3,9 @@
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1994  University of Cambridge
 
-Cardinal arithmetic -- WITHOUT the Axiom of Choice
+*)
 
-Note: Could omit proving the algebraic laws for cardinal addition and
-multiplication.  On finite cardinals these operations coincide with
-addition and multiplication of natural numbers; on infinite cardinals they
-coincide with union (maximum).  Either way we get most laws for free.
-*)
+header{*Cardinal Arithmetic Without the Axiom of Choice*}
 
 theory CardinalArith = Cardinal + OrderArith + ArithSimp + Finite:
 
@@ -94,6 +90,11 @@
 
 (*** Cardinal addition ***)
 
+text{*Note: Could omit proving the algebraic laws for cardinal addition and
+multiplication.  On finite cardinals these operations coincide with
+addition and multiplication of natural numbers; on infinite cardinals they
+coincide with union (maximum).  Either way we get most laws for free.*}
+
 (** Cardinal addition is commutative **)
 
 lemma sum_commute_eqpoll: "A+B \<approx> B+A"