playground/coq/unfinished/nofixpoint-fn-real.v

13 lines
197 B
Coq
Raw Normal View History

2023-05-23 17:08:33 +00:00
Require Import Coq.Reals.Reals.
Require Export Coq.Reals.RIneq.
(*Require Import Raxioms.*)
Definition f (x:R) : R := x + 1.
Theorem fnofix : forall x:R,
f x <> x.
Proof.
intros.
field.