src/HOL/Hyperreal/HyperArith.thy
author paulson
Mon, 22 Dec 2003 12:50:22 +0100
changeset 14309 f508492af9b4
parent 10751 a81ea5d3dd41
child 14329 ff3210fe968f
permissions -rw-r--r--
moving HyperArith0.ML to other theories
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
14309
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
     1
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     2
theory HyperArith = HyperArith0
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     3
files "hypreal_arith.ML":
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     4
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     5
setup hypreal_arith_setup
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
     6
14309
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
     7
subsubsection{*Division By @{term 1} and @{term "-1"}*}
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
     8
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
     9
lemma hypreal_divide_minus1 [simp]: "x/-1 = -(x::hypreal)"
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    10
by simp
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    11
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    12
lemma hypreal_minus1_divide [simp]: "-1/(x::hypreal) = - (1/x)"
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    13
by (simp add: hypreal_divide_def hypreal_minus_inverse)
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    14
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    15
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    16
(*
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    17
FIXME: we should have this, as for type int, but many proofs would break.
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    18
It replaces x+-y by x-y.
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    19
Addsimps [symmetric hypreal_diff_def]
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    20
*)
f508492af9b4 moving HyperArith0.ML to other theories
paulson
parents: 10751
diff changeset
    21
10751
a81ea5d3dd41 separation of HOL-Hyperreal from HOL-Real
paulson
parents:
diff changeset
    22
end