src/HOL/Hyperreal/HyperPow.thy
author wenzelm
Fri, 02 Jun 2006 23:22:29 +0200
changeset 19765 dfe940911617
parent 17429 e8d6ed3aacfe
child 20541 f614c619b1e1
permissions -rw-r--r--
misc cleanup;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     1
(*  Title       : HyperPow.thy
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     2
    Author      : Jacques D. Fleuriot  
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     3
    Copyright   : 1998  University of Cambridge
14387
e96d5c42c4b0 Polymorphic treatment of binary arithmetic using axclasses
paulson
parents: 14378
diff changeset
     4
    Conversion to Isar and new proofs by Lawrence C Paulson, 2003/4
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     5
*)
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     6
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
     7
header{*Exponentials on the Hyperreals*}
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
     8
15131
c69542757a4d New theory header syntax.
nipkow
parents: 15085
diff changeset
     9
theory HyperPow
15360
300e09825d8b Added "ALL x > y" and relatives.
nipkow
parents: 15229
diff changeset
    10
imports HyperArith HyperNat
15131
c69542757a4d New theory header syntax.
nipkow
parents: 15085
diff changeset
    11
begin
10778
2c6605049646 more tidying, especially to remove real_of_posnat
paulson
parents: 10751
diff changeset
    12
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    13
(* consts hpowr :: "[hypreal,nat] => hypreal" *)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    14
17298
ad73fb6144cf replace type hypreal with real star
huffman
parents: 16924
diff changeset
    15
lemma hpowr_0 [simp]:   "r ^ 0       = (1::hypreal)"
ad73fb6144cf replace type hypreal with real star
huffman
parents: 16924
diff changeset
    16
by (rule power_0)
ad73fb6144cf replace type hypreal with real star
huffman
parents: 16924
diff changeset
    17
ad73fb6144cf replace type hypreal with real star
huffman
parents: 16924
diff changeset
    18
lemma hpowr_Suc [simp]: "r ^ (Suc n) = (r::hypreal) * (r ^ n)"
ad73fb6144cf replace type hypreal with real star
huffman
parents: 16924
diff changeset
    19
by (rule power_Suc)
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
    20
19765
dfe940911617 misc cleanup;
wenzelm
parents: 17429
diff changeset
    21
definition
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
    22
  (* hypernatural powers of hyperreals *)
19765
dfe940911617 misc cleanup;
wenzelm
parents: 17429
diff changeset
    23
  pow :: "[hypreal,hypnat] => hypreal"     (infixr "pow" 80)
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
    24
  hyperpow_def [transfer_unfold]:
19765
dfe940911617 misc cleanup;
wenzelm
parents: 17429
diff changeset
    25
  "(R::hypreal) pow (N::hypnat) = ( *f2* op ^) R N"
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    26
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    27
lemma hrealpow_two: "(r::hypreal) ^ Suc (Suc 0) = r * r"
14443
75910c7557c5 generic theorems about exponentials; general tidying up
paulson
parents: 14435
diff changeset
    28
by simp
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    29
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
    30
lemma hrealpow_two_le [simp]: "(0::hypreal) \<le> r ^ Suc (Suc 0)"
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
    31
by (auto simp add: zero_le_mult_iff)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    32
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
    33
lemma hrealpow_two_le_add_order [simp]:
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    34
     "(0::hypreal) \<le> u ^ Suc (Suc 0) + v ^ Suc (Suc 0)"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    35
by (simp only: hrealpow_two_le add_nonneg_nonneg)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    36
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
    37
lemma hrealpow_two_le_add_order2 [simp]:
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    38
     "(0::hypreal) \<le> u ^ Suc (Suc 0) + v ^ Suc (Suc 0) + w ^ Suc (Suc 0)"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    39
by (simp only: hrealpow_two_le add_nonneg_nonneg)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    40
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    41
lemma hypreal_add_nonneg_eq_0_iff:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    42
     "[| 0 \<le> x; 0 \<le> y |] ==> (x+y = 0) = (x = 0 & y = (0::hypreal))"
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
    43
by arith
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
    44
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    45
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    46
text{*FIXME: DELETE THESE*}
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    47
lemma hypreal_three_squares_add_zero_iff:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    48
     "(x*x + y*y + z*z = 0) = (x = 0 & y = 0 & z = (0::hypreal))"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    49
apply (simp only: zero_le_square add_nonneg_nonneg hypreal_add_nonneg_eq_0_iff, auto)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    50
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    51
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    52
lemma hrealpow_three_squares_add_zero_iff [simp]:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    53
     "(x ^ Suc (Suc 0) + y ^ Suc (Suc 0) + z ^ Suc (Suc 0) = (0::hypreal)) = 
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    54
      (x = 0 & y = 0 & z = 0)"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    55
by (simp only: hypreal_three_squares_add_zero_iff hrealpow_two)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    56
16924
04246269386e removed the dependence on abs_mult
paulson
parents: 15539
diff changeset
    57
(*FIXME: This and RealPow.abs_realpow_two should be replaced by an abstract
04246269386e removed the dependence on abs_mult
paulson
parents: 15539
diff changeset
    58
  result proved in Ring_and_Field*)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    59
lemma hrabs_hrealpow_two [simp]:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    60
     "abs(x ^ Suc (Suc 0)) = (x::hypreal) ^ Suc (Suc 0)"
16924
04246269386e removed the dependence on abs_mult
paulson
parents: 15539
diff changeset
    61
by (simp add: abs_mult)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    62
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    63
lemma two_hrealpow_ge_one [simp]: "(1::hypreal) \<le> 2 ^ n"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    64
by (insert power_increasing [of 0 n "2::hypreal"], simp)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    65
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
    66
lemma two_hrealpow_gt [simp]: "hypreal_of_nat n < 2 ^ n"
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    67
apply (induct_tac "n")
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    68
apply (auto simp add: hypreal_of_nat_Suc left_distrib)
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
    69
apply (cut_tac n = n in two_hrealpow_ge_one, arith)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    70
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    71
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    72
lemma hrealpow:
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    73
    "star_n X ^ m = star_n (%n. (X n::real) ^ m)"
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    74
apply (induct_tac "m")
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    75
apply (auto simp add: star_n_one_num star_n_mult power_0)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    76
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    77
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    78
lemma hrealpow_sum_square_expand:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    79
     "(x + (y::hypreal)) ^ Suc (Suc 0) =
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    80
      x ^ Suc (Suc 0) + y ^ Suc (Suc 0) + (hypreal_of_nat (Suc (Suc 0)))*x*y"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    81
by (simp add: right_distrib left_distrib hypreal_of_nat_Suc)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    82
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    83
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    84
subsection{*Literal Arithmetic Involving Powers and Type @{typ hypreal}*}
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    85
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    86
lemma power_hypreal_of_real_number_of:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    87
     "(number_of v :: hypreal) ^ n = hypreal_of_real ((number_of v) ^ n)"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    88
by simp
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
    89
(* why is this a simp rule? - BH *)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    90
declare power_hypreal_of_real_number_of [of _ "number_of w", standard, simp]
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    91
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    92
lemma hrealpow_HFinite: "x \<in> HFinite ==> x ^ n \<in> HFinite"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    93
apply (induct_tac "n")
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    94
apply (auto intro: HFinite_mult)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    95
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    96
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    97
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    98
subsection{*Powers with Hypernatural Exponents*}
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
    99
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   100
lemma hyperpow: "star_n X pow star_n Y = star_n (%n. X n ^ Y n)"
17429
e8d6ed3aacfe merged Transfer.thy and StarType.thy into StarDef.thy; renamed Ifun2_of to starfun2; cleaned up
huffman
parents: 17332
diff changeset
   101
by (simp add: hyperpow_def starfun2_star_n)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   102
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   103
lemma hyperpow_zero [simp]: "!!n. (0::hypreal) pow (n + (1::hypnat)) = 0"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   104
by (transfer, simp)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   105
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   106
lemma hyperpow_not_zero: "!!r n. r \<noteq> (0::hypreal) ==> r pow n \<noteq> 0"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   107
by (transfer, simp)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   108
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   109
lemma hyperpow_inverse:
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   110
     "!!r n. r \<noteq> (0::hypreal) ==> inverse(r pow n) = (inverse r) pow n"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   111
by (transfer, rule power_inverse)
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   112
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   113
lemma hyperpow_hrabs: "!!r n. abs r pow n = abs (r pow n)"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   114
by (transfer, rule power_abs [symmetric])
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   115
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   116
lemma hyperpow_add: "!!r n m. r pow (n + m) = (r pow n) * (r pow m)"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   117
by (transfer, rule power_add)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   118
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   119
lemma hyperpow_one [simp]: "!!r. r pow (1::hypnat) = r"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   120
by (transfer, simp)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   121
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   122
lemma hyperpow_two:
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   123
     "!!r. r pow ((1::hypnat) + (1::hypnat)) = r * r"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   124
by (transfer, simp)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   125
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   126
lemma hyperpow_gt_zero: "!!r n. (0::hypreal) < r ==> 0 < r pow n"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   127
by (transfer, rule zero_less_power)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   128
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   129
lemma hyperpow_ge_zero: "!!r n. (0::hypreal) \<le> r ==> 0 \<le> r pow n"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   130
by (transfer, rule zero_le_power)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   131
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   132
lemma hyperpow_le:
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   133
  "!!x y n. [|(0::hypreal) < x; x \<le> y|] ==> x pow n \<le> y pow n"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   134
by (transfer, rule power_mono [OF _ order_less_imp_le])
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   135
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   136
lemma hyperpow_eq_one [simp]: "!!n. 1 pow n = (1::hypreal)"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   137
by (transfer, simp)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   138
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   139
lemma hrabs_hyperpow_minus_one [simp]: "!!n. abs(-1 pow n) = (1::hypreal)"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   140
by (transfer, simp)
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   141
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   142
lemma hyperpow_mult: "!!r s n. (r * s) pow n = (r pow n) * (s pow n)"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   143
by (transfer, rule power_mult_distrib)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   144
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   145
lemma hyperpow_two_le [simp]: "0 \<le> r pow (1 + 1)"
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   146
by (auto simp add: hyperpow_two zero_le_mult_iff)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   147
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   148
lemma hrabs_hyperpow_two [simp]: "abs(x pow (1 + 1)) = x pow (1 + 1)"
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   149
by (simp add: abs_if hyperpow_two_le linorder_not_less)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   150
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   151
lemma hyperpow_two_hrabs [simp]: "abs(x) pow (1 + 1)  = x pow (1 + 1)"
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   152
by (simp add: hyperpow_hrabs)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   153
15229
1eb23f805c06 new simprules for abs and for things like a/b<1
paulson
parents: 15169
diff changeset
   154
text{*The precondition could be weakened to @{term "0\<le>x"}*}
1eb23f805c06 new simprules for abs and for things like a/b<1
paulson
parents: 15169
diff changeset
   155
lemma hypreal_mult_less_mono:
1eb23f805c06 new simprules for abs and for things like a/b<1
paulson
parents: 15169
diff changeset
   156
     "[| u<v;  x<y;  (0::hypreal) < v;  0 < x |] ==> u*x < v* y"
1eb23f805c06 new simprules for abs and for things like a/b<1
paulson
parents: 15169
diff changeset
   157
 by (simp add: Ring_and_Field.mult_strict_mono order_less_imp_le)
1eb23f805c06 new simprules for abs and for things like a/b<1
paulson
parents: 15169
diff changeset
   158
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   159
lemma hyperpow_two_gt_one: "1 < r ==> 1 < r pow (1 + 1)"
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   160
apply (auto simp add: hyperpow_two)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   161
apply (rule_tac y = "1*1" in order_le_less_trans)
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   162
apply (rule_tac [2] hypreal_mult_less_mono, auto)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   163
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   164
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   165
lemma hyperpow_two_ge_one:
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   166
     "1 \<le> r ==> 1 \<le> r pow (1 + 1)"
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   167
by (auto dest!: order_le_imp_less_or_eq intro: hyperpow_two_gt_one order_less_imp_le)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   168
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   169
lemma two_hyperpow_ge_one [simp]: "(1::hypreal) \<le> 2 pow n"
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   170
apply (rule_tac y = "1 pow n" in order_trans)
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   171
apply (rule_tac [2] hyperpow_le, auto)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   172
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   173
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   174
lemma hyperpow_minus_one2 [simp]:
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   175
     "!!n. -1 pow ((1 + 1)*n) = (1::hypreal)"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   176
by (transfer, simp)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   177
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   178
lemma hyperpow_less_le:
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   179
     "!!r n N. [|(0::hypreal) \<le> r; r \<le> 1; n < N|] ==> r pow N \<le> r pow n"
17332
4910cf8c0cd2 added theorem attributes transfer_intro, transfer_unfold, transfer_refold; simplified some proofs; some rearranging
huffman
parents: 17318
diff changeset
   180
by (transfer, rule power_decreasing [OF order_less_imp_le])
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   181
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   182
lemma hyperpow_SHNat_le:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   183
     "[| 0 \<le> r;  r \<le> (1::hypreal);  N \<in> HNatInfinite |]
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   184
      ==> ALL n: Nats. r pow N \<le> r pow n"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   185
by (auto intro!: hyperpow_less_le simp add: HNatInfinite_iff)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   186
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   187
lemma hyperpow_realpow:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   188
      "(hypreal_of_real r) pow (hypnat_of_nat n) = hypreal_of_real (r ^ n)"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   189
by (simp add: star_of_def hypnat_of_nat_eq hyperpow)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   190
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   191
lemma hyperpow_SReal [simp]:
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   192
     "(hypreal_of_real r) pow (hypnat_of_nat n) \<in> Reals"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   193
by (simp del: star_of_power add: hyperpow_realpow SReal_def)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   194
15003
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   195
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   196
lemma hyperpow_zero_HNatInfinite [simp]:
6145dd7538d7 replaced monomorphic abs definitions by abs_if
paulson
parents: 14468
diff changeset
   197
     "N \<in> HNatInfinite ==> (0::hypreal) pow N = 0"
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   198
by (drule HNatInfinite_is_Suc, auto)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   199
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   200
lemma hyperpow_le_le:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   201
     "[| (0::hypreal) \<le> r; r \<le> 1; n \<le> N |] ==> r pow N \<le> r pow n"
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   202
apply (drule order_le_less [of n, THEN iffD1])
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   203
apply (auto intro: hyperpow_less_le)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   204
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   205
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   206
lemma hyperpow_Suc_le_self2:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   207
     "[| (0::hypreal) \<le> r; r < 1 |] ==> r pow (n + (1::hypnat)) \<le> r"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   208
apply (drule_tac n = " (1::hypnat) " in hyperpow_le_le)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   209
apply auto
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   210
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   211
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   212
lemma lemma_Infinitesimal_hyperpow:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   213
     "[| x \<in> Infinitesimal; 0 < N |] ==> abs (x pow N) \<le> abs x"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   214
apply (unfold Infinitesimal_def)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   215
apply (auto intro!: hyperpow_Suc_le_self2 
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   216
          simp add: hyperpow_hrabs [symmetric] hypnat_gt_zero_iff2 abs_ge_zero)
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   217
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   218
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   219
lemma Infinitesimal_hyperpow:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   220
     "[| x \<in> Infinitesimal; 0 < N |] ==> x pow N \<in> Infinitesimal"
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   221
apply (rule hrabs_le_Infinitesimal)
14371
c78c7da09519 Conversion of HyperNat to Isar format and its declaration as a semiring
paulson
parents: 14348
diff changeset
   222
apply (rule_tac [2] lemma_Infinitesimal_hyperpow, auto)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   223
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   224
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   225
lemma hrealpow_hyperpow_Infinitesimal_iff:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   226
     "(x ^ n \<in> Infinitesimal) = (x pow (hypnat_of_nat n) \<in> Infinitesimal)"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   227
apply (cases x)
14378
69c4d5997669 generic of_nat and of_int functions, and generalization of iszero
paulson
parents: 14371
diff changeset
   228
apply (simp add: hrealpow hyperpow hypnat_of_nat_eq)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   229
done
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   230
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   231
lemma Infinitesimal_hrealpow:
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   232
     "[| x \<in> Infinitesimal; 0 < n |] ==> x ^ n \<in> Infinitesimal"
17318
bc1c75855f3d starfun, starset, and other functions on NS types are now polymorphic;
huffman
parents: 17299
diff changeset
   233
by (simp add: hrealpow_hyperpow_Infinitesimal_iff Infinitesimal_hyperpow)
14348
744c868ee0b7 Defining the type class "ringpower" and deleting superseded theorems for
paulson
parents: 11713
diff changeset
   234
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
   235
end