Added R^1 = R
authornipkow
Sat, 27 Apr 1996 12:05:58 +0200
changeset 1693 7083f6b05423
parent 1692 5324be24a5fa
child 1694 3452958f85a8
Added R^1 = R
src/HOL/RelPow.ML
--- a/src/HOL/RelPow.ML	Fri Apr 26 13:33:51 1996 +0200
+++ b/src/HOL/RelPow.ML	Sat Apr 27 12:05:58 1996 +0200
@@ -9,6 +9,11 @@
 val [rel_pow_0, rel_pow_Suc] = nat_recs rel_pow_def;
 Addsimps [rel_pow_0];
 
+goal RelPow.thy "R^1 = R";
+by(simp_tac (!simpset addsimps [rel_pow_Suc]) 1);
+qed "rel_pow_1";
+Addsimps [rel_pow_1];
+
 goal RelPow.thy "(x,x) : R^0";
 by (Simp_tac 1);
 qed "rel_pow_0_I";